src/HOL/Tools/typecopy_package.ML
author wenzelm
Tue, 02 Sep 2008 14:10:45 +0200
changeset 28083 103d9282a946
parent 28054 2b84d34c5d02
child 28084 a05ca48ef263
permissions -rw-r--r--
explicit type Name.binding for higher-specification elements;
     1 (*  Title:      HOL/Tools/typecopy_package.ML
     2     ID:         $Id$
     3     Author:     Florian Haftmann, TU Muenchen
     4 
     5 Introducing copies of types using trivial typedefs; datatype-like abstraction.
     6 *)
     7 
     8 signature TYPECOPY_PACKAGE =
     9 sig
    10   type info = {
    11     vs: (string * sort) list,
    12     constr: string,
    13     typ: typ,
    14     inject: thm,
    15     proj: string * typ,
    16     proj_def: thm
    17   }
    18   val add_typecopy: bstring * string list -> typ -> (bstring * bstring) option
    19     -> theory -> (string * info) * theory
    20   val get_typecopies: theory -> string list
    21   val get_info: theory -> string -> info option
    22   val interpretation: (string -> theory -> theory) -> theory -> theory
    23   val print_typecopies: theory -> unit
    24   val setup: theory -> theory
    25 end;
    26 
    27 structure TypecopyPackage: TYPECOPY_PACKAGE =
    28 struct
    29 
    30 (* theory data *)
    31 
    32 type info = {
    33   vs: (string * sort) list,
    34   constr: string,
    35   typ: typ,
    36   inject: thm,
    37   proj: string * typ,
    38   proj_def: thm
    39 };
    40 
    41 structure TypecopyData = TheoryDataFun
    42 (
    43   type T = info Symtab.table;
    44   val empty = Symtab.empty;
    45   val copy = I;
    46   val extend = I;
    47   fun merge _ = Symtab.merge (K true);
    48 );
    49 
    50 fun print_typecopies thy =
    51   let
    52     val tab = TypecopyData.get thy;
    53     fun mk (tyco, { vs, constr, typ, proj = (proj, _), ... } : info) =
    54       (Pretty.block o Pretty.breaks) [
    55         Syntax.pretty_typ_global thy (Type (tyco, map TFree vs)),
    56         Pretty.str "=",
    57         (Pretty.str o Sign.extern_const thy) constr,
    58         Syntax.pretty_typ_global thy typ,
    59         Pretty.block [Pretty.str "(", (Pretty.str o Sign.extern_const thy) proj, Pretty.str  ")"]];
    60     in
    61       (Pretty.writeln o Pretty.block o Pretty.fbreaks)
    62         (Pretty.str "type copies:" :: map mk (Symtab.dest tab))
    63     end;
    64 
    65 val get_typecopies = Symtab.keys o TypecopyData.get;
    66 val get_info = Symtab.lookup o TypecopyData.get;
    67 
    68 
    69 (* interpretation of type copies *)
    70 
    71 structure TypecopyInterpretation = InterpretationFun(type T = string val eq = op =);
    72 val interpretation = TypecopyInterpretation.interpretation;
    73 
    74 
    75 (* add a type copy *)
    76 
    77 local
    78 
    79 fun gen_add_typecopy prep_typ (raw_tyco, raw_vs) raw_ty constr_proj thy =
    80   let
    81     val ty = prep_typ thy raw_ty;
    82     val vs = AList.make (the_default HOLogic.typeS o AList.lookup (op =) (typ_tfrees ty)) raw_vs;
    83     val tac = Tactic.rtac UNIV_witness 1;
    84     fun add_info tyco ( { abs_type = ty_abs, rep_type = ty_rep, Abs_name = c_abs,
    85       Rep_name = c_rep, Abs_inject = inject,
    86       Abs_inverse = inverse, ... } : TypedefPackage.info ) thy =
    87         let
    88           val exists_thm =
    89             UNIV_I
    90             |> Drule.instantiate' [SOME (ctyp_of thy (Logic.varifyT ty_rep))] [];
    91           val inject' = inject OF [exists_thm, exists_thm];
    92           val proj_def = inverse OF [exists_thm];
    93           val info = {
    94             vs = vs,
    95             constr = c_abs,
    96             typ = ty_rep,
    97             inject = inject',
    98             proj = (c_rep, ty_abs --> ty_rep),
    99             proj_def = proj_def
   100           };
   101         in
   102           thy
   103           |> (TypecopyData.map o Symtab.update_new) (tyco, info)
   104           |> TypecopyInterpretation.data tyco
   105           |> pair (tyco, info)
   106         end
   107   in
   108     thy
   109     |> TypedefPackage.add_typedef_i false (SOME raw_tyco) (raw_tyco, map fst vs, NoSyn)
   110       (HOLogic.mk_UNIV ty) (Option.map swap constr_proj) tac
   111     |-> (fn (tyco, info) => add_info tyco info)
   112   end;
   113 
   114 in
   115 
   116 val add_typecopy = gen_add_typecopy Sign.certify_typ;
   117 
   118 end;
   119 
   120 
   121 (* code generator setup *)
   122 
   123 fun add_typecopy_spec tyco thy =
   124   let
   125     val SOME { constr, proj_def, inject, vs, ... } = get_info thy tyco;
   126     val vs' = (map o apsnd) (curry (Sorts.inter_sort (Sign.classes_of thy)) [HOLogic.class_eq]) vs;
   127     val ty = Logic.unvarifyT (Sign.the_const_type thy constr);
   128     fun add_def tyco lthy =
   129       let
   130         val ty = Type (tyco, map TFree vs');
   131         fun mk_side const_name = Const (const_name, ty --> ty --> HOLogic.boolT)
   132           $ Free ("x", ty) $ Free ("y", ty);
   133         val def = HOLogic.mk_Trueprop (HOLogic.mk_eq
   134           (mk_side @{const_name eq_class.eq}, mk_side @{const_name "op ="}));
   135         val def' = Syntax.check_term lthy def;
   136         val ((_, (_, thm)), lthy') = Specification.definition
   137           (NONE, ((Name.no_binding, []), def')) lthy;
   138         val ctxt_thy = ProofContext.init (ProofContext.theory_of lthy);
   139         val thm' = singleton (ProofContext.export lthy' ctxt_thy) thm;
   140       in (thm', lthy') end;
   141     fun tac thms = Class.intro_classes_tac []
   142       THEN ALLGOALS (ProofContext.fact_tac thms);
   143     fun add_eq_thm thy = 
   144       let
   145         val eq = inject
   146           |> Code_Unit.constrain_thm [HOLogic.class_eq]
   147           |> Simpdata.mk_eq
   148           |> MetaSimplifier.rewrite_rule [Thm.transfer thy @{thm equals_eq}];
   149       in Code.add_func eq thy end;
   150   in
   151     thy
   152     |> Code.add_datatype [(constr, ty)]
   153     |> Code.add_func proj_def
   154     |> TheoryTarget.instantiation ([tyco], vs', [HOLogic.class_eq])
   155     |> add_def tyco
   156     |-> (fn thm => Class.prove_instantiation_instance (K (tac [thm]))
   157     #> LocalTheory.exit
   158     #> ProofContext.theory_of
   159     #> Code.del_func thm
   160     #> add_eq_thm)
   161   end;
   162 
   163 val setup =
   164   TypecopyInterpretation.init
   165   #> interpretation add_typecopy_spec
   166 
   167 end;