author | wenzelm |
Thu, 07 Dec 2006 23:16:55 +0100 | |
changeset 21708 | 45e7491bea47 |
parent 21675 | 38f6cb45ce24 |
child 22423 | c1836b14c63a |
permissions | -rw-r--r-- |
20426 | 1 |
(* Title: HOL/Tools/typecopy_package.ML |
2 |
ID: $Id$ |
|
3 |
Author: Florian Haftmann, TU Muenchen |
|
4 |
||
20855 | 5 |
Introducing copies of types using trivial typedefs; datatype-like abstraction. |
20426 | 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 |
|
20483
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
19 |
-> theory -> (string * info) * theory |
20426 | 20 |
val get_typecopies: theory -> string list |
21 |
val get_typecopy_info: theory -> string -> info option |
|
20835 | 22 |
type hook = string * info -> theory -> theory |
23 |
val add_hook: hook -> theory -> theory |
|
24 |
val get_spec: theory -> string -> (string * sort) list * (string * typ list) list |
|
25 |
val get_cert: theory -> string -> thm |
|
26 |
val get_eq: theory -> string -> thm |
|
20426 | 27 |
val print: theory -> unit |
28 |
val setup: theory -> theory |
|
29 |
end; |
|
30 |
||
31 |
structure TypecopyPackage: TYPECOPY_PACKAGE = |
|
32 |
struct |
|
33 |
||
34 |
(* theory data *) |
|
35 |
||
36 |
type info = { |
|
37 |
vs: (string * sort) list, |
|
38 |
constr: string, |
|
39 |
typ: typ, |
|
40 |
inject: thm, |
|
41 |
proj: string * typ, |
|
42 |
proj_def: thm |
|
43 |
}; |
|
44 |
||
45 |
type hook = string * info -> theory -> theory; |
|
46 |
||
47 |
structure TypecopyData = TheoryDataFun |
|
48 |
(struct |
|
49 |
val name = "HOL/typecopy_package"; |
|
50 |
type T = info Symtab.table * (serial * hook) list; |
|
51 |
val empty = (Symtab.empty, []); |
|
52 |
val copy = I; |
|
53 |
val extend = I; |
|
54 |
fun merge _ ((tab1, hooks1), (tab2, hooks2) : T) = |
|
55 |
(Symtab.merge (K true) (tab1, tab2), AList.merge (op =) (K true) (hooks1, hooks2)); |
|
56 |
fun print thy (tab, _) = |
|
57 |
let |
|
58 |
fun mk (tyco, { vs, constr, typ, proj = (proj, _), ... } : info) = |
|
59 |
(Pretty.block o Pretty.breaks) [ |
|
60 |
Sign.pretty_typ thy (Type (tyco, map TFree vs)), |
|
61 |
Pretty.str "=", |
|
62 |
(Pretty.str o Sign.extern_const thy) constr, |
|
63 |
Sign.pretty_typ thy typ, |
|
64 |
Pretty.block [Pretty.str "(", (Pretty.str o Sign.extern_const thy) proj, Pretty.str ")"] |
|
65 |
]; |
|
66 |
in |
|
67 |
(Pretty.writeln o Pretty.block o Pretty.fbreaks) ( |
|
68 |
Pretty.str "type copies:" |
|
69 |
:: map mk (Symtab.dest tab) |
|
70 |
) |
|
71 |
end; |
|
72 |
end); |
|
73 |
||
74 |
val print = TypecopyData.print; |
|
75 |
val get_typecopies = Symtab.keys o fst o TypecopyData.get; |
|
76 |
val get_typecopy_info = Symtab.lookup o fst o TypecopyData.get; |
|
77 |
||
78 |
||
79 |
(* hook management *) |
|
80 |
||
81 |
fun add_hook hook = |
|
82 |
(TypecopyData.map o apsnd o cons) (serial (), hook); |
|
83 |
||
84 |
fun invoke_hooks tyco_info thy = |
|
85 |
fold (fn (_, f) => f tyco_info) ((snd o TypecopyData.get) thy) thy; |
|
86 |
||
87 |
||
88 |
(* add a type copy *) |
|
89 |
||
90 |
local |
|
91 |
||
20483
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
92 |
fun gen_add_typecopy prep_typ (raw_tyco, raw_vs) raw_ty constr_proj thy = |
20426 | 93 |
let |
94 |
val ty = prep_typ thy raw_ty; |
|
95 |
val vs = AList.make (the_default HOLogic.typeS o AList.lookup (op =) (typ_tfrees ty)) raw_vs; |
|
96 |
val tac = Tactic.rtac UNIV_witness 1; |
|
20483
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
97 |
fun add_info tyco ( { abs_type = ty_abs, rep_type = ty_rep, Abs_name = c_abs, |
20426 | 98 |
Rep_name = c_rep, Abs_inject = inject, |
21708 | 99 |
Abs_inverse = inverse, ... } : TypedefPackage.info ) thy = |
20426 | 100 |
let |
101 |
val exists_thm = |
|
102 |
UNIV_I |
|
103 |
|> Drule.instantiate' [SOME (ctyp_of thy (Logic.varifyT ty_rep))] []; |
|
104 |
val inject' = inject OF [exists_thm, exists_thm]; |
|
105 |
val proj_def = inverse OF [exists_thm]; |
|
106 |
val info = { |
|
107 |
vs = vs, |
|
108 |
constr = c_abs, |
|
109 |
typ = ty_rep, |
|
110 |
inject = inject', |
|
111 |
proj = (c_rep, ty_abs --> ty_rep), |
|
112 |
proj_def = proj_def |
|
113 |
}; |
|
114 |
in |
|
115 |
thy |
|
20483
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
116 |
|> (TypecopyData.map o apfst o Symtab.update_new) (tyco, info) |
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
117 |
|> invoke_hooks (tyco, info) |
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
118 |
|> pair (tyco, info) |
20426 | 119 |
end |
120 |
in |
|
121 |
thy |
|
20483
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
122 |
|> setmp TypedefPackage.quiet_mode true |
04aa552a83bc
TypedefPackage.add_typedef_* now yields name of introduced type constructor
haftmann
parents:
20426
diff
changeset
|
123 |
(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
|
124 |
(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
|
125 |
|-> (fn (tyco, info) => add_info tyco info) |
20426 | 126 |
end; |
127 |
||
128 |
in |
|
129 |
||
130 |
val add_typecopy = gen_add_typecopy Sign.certify_typ; |
|
131 |
||
132 |
end; (*local*) |
|
133 |
||
134 |
||
20835 | 135 |
(* equality function equation *) |
136 |
||
137 |
fun get_eq thy tyco = |
|
138 |
(#inject o the o get_typecopy_info thy) tyco; |
|
139 |
||
140 |
||
141 |
(* datatype specification and certificate *) |
|
142 |
||
143 |
fun get_spec thy tyco = |
|
144 |
let |
|
145 |
val SOME { vs, constr, typ, ... } = get_typecopy_info thy tyco |
|
146 |
in (vs, [(constr, [typ])]) end; |
|
147 |
||
148 |
local |
|
21708 | 149 |
val bool_eq_implies = iffD1; |
20835 | 150 |
val rew_eq = thm "HOL.atomize_eq" |> Thm.symmetric; |
151 |
in fun get_cert thy tyco = |
|
21708 | 152 |
MetaSimplifier.rewrite_rule [rew_eq] (bool_eq_implies OF [get_eq thy tyco]) |
20835 | 153 |
end; (*local*) |
154 |
||
155 |
||
156 |
(* hook for projection function code *) |
|
20426 | 157 |
|
21708 | 158 |
fun add_project (_ , {proj_def, ...} : info) = |
20597 | 159 |
CodegenData.add_func proj_def; |
20426 | 160 |
|
161 |
val setup = |
|
162 |
TypecopyData.init |
|
20597 | 163 |
#> add_hook add_project; |
20426 | 164 |
|
165 |
end; (*struct*) |