src/HOL/Tools/typecopy_package.ML
author haftmann
Thu, 29 Nov 2007 23:01:18 +0100
changeset 25506 c9bea6426932
parent 25489 5b0625f6e324
child 25534 d0b74fdd6067
permissions -rw-r--r--
tuned
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     1
(*  Title:      HOL/Tools/typecopy_package.ML
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     2
    ID:         $Id$
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     3
    Author:     Florian Haftmann, TU Muenchen
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     4
20855
9f60d493c8fe clarified header comments
haftmann
parents: 20835
diff changeset
     5
Introducing copies of types using trivial typedefs; datatype-like abstraction.
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     6
*)
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     7
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     8
signature TYPECOPY_PACKAGE =
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
     9
sig
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    10
  type info = {
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    11
    vs: (string * sort) list,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    12
    constr: string,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    13
    typ: typ,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    14
    inject: thm,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    15
    proj: string * typ,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    16
    proj_def: thm
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    17
  }
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    18
  val add_typecopy: bstring * string list -> typ -> (bstring * bstring) option
20483
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
    19
    -> theory -> (string * info) * theory
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    20
  val get_typecopies: theory -> string list
25506
haftmann
parents: 25489
diff changeset
    21
  val get_info: theory -> string -> info option
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
    22
  val interpretation: (string -> theory -> theory) -> theory -> theory
20835
haftmann
parents: 20597
diff changeset
    23
  val get_eq: theory -> string -> thm
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    24
  val print_typecopies: theory -> unit
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    25
  val setup: theory -> theory
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    26
end;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    27
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    28
structure TypecopyPackage: TYPECOPY_PACKAGE =
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    29
struct
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    30
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    31
(* theory data *)
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    32
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    33
type info = {
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    34
  vs: (string * sort) list,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    35
  constr: string,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    36
  typ: typ,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    37
  inject: thm,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    38
  proj: string * typ,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    39
  proj_def: thm
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    40
};
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    41
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    42
structure TypecopyData = TheoryDataFun
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    43
(
24626
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
    44
  type T = info Symtab.table;
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
    45
  val empty = Symtab.empty;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    46
  val copy = I;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    47
  val extend = I;
24626
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
    48
  fun merge _ = Symtab.merge (K true);
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    49
);
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    50
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    51
fun print_typecopies thy =
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    52
  let
24626
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
    53
    val tab = TypecopyData.get thy;
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    54
    fun mk (tyco, { vs, constr, typ, proj = (proj, _), ... } : info) =
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    55
      (Pretty.block o Pretty.breaks) [
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    56
        Sign.pretty_typ thy (Type (tyco, map TFree vs)),
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    57
        Pretty.str "=",
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    58
        (Pretty.str o Sign.extern_const thy) constr,
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    59
        Sign.pretty_typ thy typ,
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    60
        Pretty.block [Pretty.str "(", (Pretty.str o Sign.extern_const thy) proj, Pretty.str  ")"]];
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    61
    in
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    62
      (Pretty.writeln o Pretty.block o Pretty.fbreaks)
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
    63
        (Pretty.str "type copies:" :: map mk (Symtab.dest tab))
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    64
    end;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    65
24626
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
    66
val get_typecopies = Symtab.keys o TypecopyData.get;
25506
haftmann
parents: 25489
diff changeset
    67
val get_info = Symtab.lookup o TypecopyData.get;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    68
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    69
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
    70
(* interpretation of type copies *)
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    71
24711
e8bba7723858 simplified interpretation setup;
wenzelm
parents: 24626
diff changeset
    72
structure TypecopyInterpretation = InterpretationFun(type T = string val eq = op =);
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
    73
val interpretation = TypecopyInterpretation.interpretation;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    74
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    75
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    76
(* add a type copy *)
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    77
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    78
local
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    79
20483
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
    80
fun gen_add_typecopy prep_typ (raw_tyco, raw_vs) raw_ty constr_proj thy =
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    81
  let
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    82
    val ty = prep_typ thy raw_ty;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    83
    val vs = AList.make (the_default HOLogic.typeS o AList.lookup (op =) (typ_tfrees ty)) raw_vs;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    84
    val tac = Tactic.rtac UNIV_witness 1;
20483
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
    85
    fun add_info tyco ( { abs_type = ty_abs, rep_type = ty_rep, Abs_name = c_abs,
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    86
      Rep_name = c_rep, Abs_inject = inject,
21708
45e7491bea47 reorganized structure Tactic vs. MetaSimplifier;
wenzelm
parents: 21675
diff changeset
    87
      Abs_inverse = inverse, ... } : TypedefPackage.info ) thy =
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    88
        let
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    89
          val exists_thm =
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    90
            UNIV_I
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    91
            |> Drule.instantiate' [SOME (ctyp_of thy (Logic.varifyT ty_rep))] [];
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    92
          val inject' = inject OF [exists_thm, exists_thm];
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    93
          val proj_def = inverse OF [exists_thm];
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    94
          val info = {
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    95
            vs = vs,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    96
            constr = c_abs,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    97
            typ = ty_rep,
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    98
            inject = inject',
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
    99
            proj = (c_rep, ty_abs --> ty_rep),
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   100
            proj_def = proj_def
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   101
          };
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   102
        in
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   103
          thy
24626
85eceef2edc7 introduced generic concepts for theory interpretators
haftmann
parents: 24624
diff changeset
   104
          |> (TypecopyData.map o Symtab.update_new) (tyco, info)
24711
e8bba7723858 simplified interpretation setup;
wenzelm
parents: 24626
diff changeset
   105
          |> TypecopyInterpretation.data tyco
20483
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
   106
          |> pair (tyco, info)
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   107
        end
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   108
  in
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   109
    thy
20483
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
   110
    |> setmp TypedefPackage.quiet_mode true
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
   111
        (TypedefPackage.add_typedef_i false (SOME raw_tyco) (raw_tyco, map fst vs, NoSyn)
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
   112
          (HOLogic.mk_UNIV ty) (Option.map swap constr_proj)) tac
04aa552a83bc TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents: 20426
diff changeset
   113
    |-> (fn (tyco, info) => add_info tyco info)
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   114
  end;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   115
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   116
in
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   117
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   118
val add_typecopy = gen_add_typecopy Sign.certify_typ;
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   119
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
   120
end;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   121
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   122
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   123
(* code generator setup *)
20835
haftmann
parents: 20597
diff changeset
   124
25506
haftmann
parents: 25489
diff changeset
   125
fun get_eq thy = #inject o the o get_info thy;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   126
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   127
fun add_typecopy_spec tyco thy =
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   128
  let
25506
haftmann
parents: 25489
diff changeset
   129
    val SOME { constr, proj_def, inject, ... } = get_info thy tyco;
haftmann
parents: 25489
diff changeset
   130
    val ty = Logic.unvarifyT (Sign.the_const_type thy constr);
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   131
  in
25506
haftmann
parents: 25489
diff changeset
   132
    thy
haftmann
parents: 25489
diff changeset
   133
    |> Code.add_datatype [(constr, ty)]
haftmann
parents: 25489
diff changeset
   134
    |> Code.add_func proj_def
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   135
  end;
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   136
25489
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   137
val setup =
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   138
  TypecopyInterpretation.init
5b0625f6e324 simplified interpretations
haftmann
parents: 24711
diff changeset
   139
  #> interpretation add_typecopy_spec
20426
9ffea7a8b31c added typecopy_package
haftmann
parents:
diff changeset
   140
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22484
diff changeset
   141
end;