author | wenzelm |
Thu, 30 Jul 2009 12:20:43 +0200 | |
changeset 32283 | 3bebc195c124 |
parent 32212 | 21d7b4524395 |
child 32335 | 41fe1c93f218 |
permissions | -rw-r--r-- |
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
1 |
(* Title: HOL/Tools/record.ML |
14579 | 2 |
Author: Wolfgang Naraschewski, Norbert Schirmer and Markus Wenzel, TU Muenchen |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
3 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
4 |
Extensible records with structural subtyping in HOL. |
5698 | 5 |
*) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
6 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
7 |
|
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
8 |
signature BASIC_RECORD = |
5698 | 9 |
sig |
7178 | 10 |
val record_simproc: simproc |
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
11 |
val record_eq_simproc: simproc |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
12 |
val record_upd_simproc: simproc |
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
13 |
val record_split_simproc: (term -> int) -> simproc |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
14 |
val record_ex_sel_eq_simproc: simproc |
5698 | 15 |
val record_split_tac: int -> tactic |
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
16 |
val record_split_simp_tac: thm list -> (term -> int) -> int -> tactic |
5713 | 17 |
val record_split_name: string |
5698 | 18 |
val record_split_wrapper: string * wrapper |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
19 |
val print_record_type_abbr: bool ref |
17261 | 20 |
val print_record_type_as_fields: bool ref |
5698 | 21 |
end; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
22 |
|
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
23 |
signature RECORD = |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
24 |
sig |
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
25 |
include BASIC_RECORD |
25179 | 26 |
val timing: bool ref |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
27 |
val record_quick_and_dirty_sensitive: bool ref |
8574 | 28 |
val updateN: string |
21363 | 29 |
val updN: string |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
30 |
val ext_typeN: string |
21363 | 31 |
val extN: string |
32 |
val makeN: string |
|
33 |
val moreN: string |
|
34 |
val ext_dest: string |
|
35 |
||
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
36 |
val last_extT: typ -> (string * typ list) option |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
37 |
val dest_recTs : typ -> (string * typ list) list |
26088 | 38 |
val get_extT_fields: theory -> typ -> (string * typ) list * (string * typ) |
39 |
val get_recT_fields: theory -> typ -> (string * typ) list * (string * typ) |
|
40 |
val get_parent: theory -> string -> (typ list * string) option |
|
41 |
val get_extension: theory -> string -> (string * typ list) option |
|
16458 | 42 |
val get_extinjects: theory -> thm list |
43 |
val get_simpset: theory -> simpset |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
44 |
val print_records: theory -> unit |
27278
129574589734
export read_typ/cert_typ -- version with regular context operations;
wenzelm
parents:
27239
diff
changeset
|
45 |
val read_typ: Proof.context -> string -> (string * sort) list -> typ * (string * sort) list |
129574589734
export read_typ/cert_typ -- version with regular context operations;
wenzelm
parents:
27239
diff
changeset
|
46 |
val cert_typ: Proof.context -> typ -> (string * sort) list -> typ * (string * sort) list |
26477
ecf06644f6cb
eliminated quiete_mode ref (turned into proper argument);
wenzelm
parents:
26423
diff
changeset
|
47 |
val add_record: bool -> string list * string -> string option -> (string * string * mixfix) list |
16458 | 48 |
-> theory -> theory |
26477
ecf06644f6cb
eliminated quiete_mode ref (turned into proper argument);
wenzelm
parents:
26423
diff
changeset
|
49 |
val add_record_i: bool -> string list * string -> (typ list * string) option |
16458 | 50 |
-> (string * typ * mixfix) list -> theory -> theory |
18708 | 51 |
val setup: theory -> theory |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
52 |
end; |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
53 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
54 |
|
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
55 |
structure Record: RECORD = |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
56 |
struct |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
57 |
|
21546 | 58 |
val eq_reflection = thm "eq_reflection"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
59 |
val rec_UNIV_I = thm "rec_UNIV_I"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
60 |
val rec_True_simp = thm "rec_True_simp"; |
27104
791607529f6d
rep_datatype command now takes list of constructors as input arguments
haftmann
parents:
26957
diff
changeset
|
61 |
val Pair_eq = thm "Product_Type.prod.inject"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
62 |
val atomize_all = thm "HOL.atomize_all"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
63 |
val atomize_imp = thm "HOL.atomize_imp"; |
17960 | 64 |
val meta_allE = thm "Pure.meta_allE"; |
65 |
val prop_subst = thm "prop_subst"; |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
66 |
val Pair_sel_convs = [fst_conv,snd_conv]; |
26359 | 67 |
val K_record_comp = @{thm "K_record_comp"}; |
68 |
val K_comp_convs = [@{thm o_apply}, K_record_comp] |
|
11832 | 69 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
70 |
(** name components **) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
71 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
72 |
val rN = "r"; |
15215 | 73 |
val wN = "w"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
74 |
val moreN = "more"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
75 |
val schemeN = "_scheme"; |
17261 | 76 |
val ext_typeN = "_ext_type"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
77 |
val extN ="_ext"; |
15215 | 78 |
val casesN = "_cases"; |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
79 |
val ext_dest = "_sel"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
80 |
val updateN = "_update"; |
15215 | 81 |
val updN = "_upd"; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
82 |
val makeN = "make"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
83 |
val fields_selN = "fields"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
84 |
val extendN = "extend"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
85 |
val truncateN = "truncate"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
86 |
|
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
87 |
(*see typedef.ML*) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
88 |
val RepN = "Rep_"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
89 |
val AbsN = "Abs_"; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
90 |
|
4894 | 91 |
(*** utilities ***) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
92 |
|
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
93 |
fun but_last xs = fst (split_last xs); |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
94 |
|
19748 | 95 |
fun varifyT midx = |
96 |
let fun varify (a, S) = TVar ((a, midx + 1), S); |
|
97 |
in map_type_tfree varify end; |
|
98 |
||
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
99 |
fun domain_type' T = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
100 |
domain_type T handle Match => T; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
101 |
|
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
102 |
fun range_type' T = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
103 |
range_type T handle Match => T; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
104 |
|
5698 | 105 |
(* messages *) |
106 |
||
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
107 |
fun trace_thm str thm = |
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
31902
diff
changeset
|
108 |
tracing (str ^ (Pretty.string_of (Display.pretty_thm_without_context thm))); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
109 |
|
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
110 |
fun trace_thms str thms = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
111 |
(tracing str; map (trace_thm "") thms); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
112 |
|
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
113 |
fun trace_term str t = |
26957 | 114 |
tracing (str ^ Syntax.string_of_term_global Pure.thy t); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
115 |
|
15012
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
schirmer
parents:
14981
diff
changeset
|
116 |
(* timing *) |
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
schirmer
parents:
14981
diff
changeset
|
117 |
|
25179 | 118 |
val timing = ref false; |
15012
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
schirmer
parents:
14981
diff
changeset
|
119 |
fun timeit_msg s x = if !timing then (warning s; timeit x) else x (); |
16379 | 120 |
fun timing_msg s = if !timing then warning s else (); |
17261 | 121 |
|
12255 | 122 |
(* syntax *) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
123 |
|
12247 | 124 |
fun prune n xs = Library.drop (n, xs); |
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
125 |
fun prefix_base s = Long_Name.map_base_name (fn bname => s ^ bname); |
11832 | 126 |
|
11927
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
127 |
val Trueprop = HOLogic.mk_Trueprop; |
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
128 |
fun All xs t = Term.list_all_free (xs, t); |
4894 | 129 |
|
11934
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm
parents:
11927
diff
changeset
|
130 |
infix 9 $$; |
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm
parents:
11927
diff
changeset
|
131 |
infix 0 :== ===; |
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm
parents:
11927
diff
changeset
|
132 |
infixr 0 ==>; |
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm
parents:
11927
diff
changeset
|
133 |
|
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm
parents:
11927
diff
changeset
|
134 |
val (op $$) = Term.list_comb; |
24255 | 135 |
val (op :==) = PrimitiveDefs.mk_defpair; |
11927
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
136 |
val (op ===) = Trueprop o HOLogic.mk_eq; |
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
137 |
val (op ==>) = Logic.mk_implies; |
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
138 |
|
11832 | 139 |
(* morphisms *) |
140 |
||
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
141 |
fun mk_RepN name = suffix ext_typeN (prefix_base RepN name); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
142 |
fun mk_AbsN name = suffix ext_typeN (prefix_base AbsN name); |
11832 | 143 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
144 |
fun mk_Rep name repT absT = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
145 |
Const (suffix ext_typeN (prefix_base RepN name),absT --> repT); |
11832 | 146 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
147 |
fun mk_Abs name repT absT = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
148 |
Const (mk_AbsN name,repT --> absT); |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
149 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
150 |
(* constructor *) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
151 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
152 |
fun mk_extC (name,T) Ts = (suffix extN name, Ts ---> T); |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
153 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
154 |
fun mk_ext (name,T) ts = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
155 |
let val Ts = map fastype_of ts |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
156 |
in list_comb (Const (mk_extC (name,T) Ts),ts) end; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
157 |
|
15215 | 158 |
(* cases *) |
159 |
||
160 |
fun mk_casesC (name,T,vT) Ts = (suffix casesN name, (Ts ---> vT) --> T --> vT) |
|
161 |
||
162 |
fun mk_cases (name,T,vT) f = |
|
17261 | 163 |
let val Ts = binder_types (fastype_of f) |
15215 | 164 |
in Const (mk_casesC (name,T,vT) Ts) $ f end; |
17261 | 165 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
166 |
(* selector *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
167 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
168 |
fun mk_selC sT (c,T) = (c,sT --> T); |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
169 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
170 |
fun mk_sel s (c,T) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
171 |
let val sT = fastype_of s |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
172 |
in Const (mk_selC sT (c,T)) $ s end; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
173 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
174 |
(* updates *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
175 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
176 |
fun mk_updC sfx sT (c,T) = (suffix sfx c, (T --> T) --> sT --> sT); |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
177 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
178 |
fun mk_upd' sfx c v sT = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
179 |
let val vT = domain_type (fastype_of v); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
180 |
in Const (mk_updC sfx sT (c, vT)) $ v end; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
181 |
|
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
182 |
fun mk_upd sfx c v s = mk_upd' sfx c v (fastype_of s) $ s |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
183 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
184 |
(* types *) |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
185 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
186 |
fun dest_recT (typ as Type (c_ext_type, Ts as (T::_))) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
187 |
(case try (unsuffix ext_typeN) c_ext_type of |
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
188 |
NONE => raise TYPE ("Record.dest_recT", [typ], []) |
15570 | 189 |
| SOME c => ((c, Ts), List.last Ts)) |
31723
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents:
31136
diff
changeset
|
190 |
| dest_recT typ = raise TYPE ("Record.dest_recT", [typ], []); |
5197 | 191 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
192 |
fun is_recT T = |
17261 | 193 |
(case try dest_recT T of NONE => false | SOME _ => true); |
11833 | 194 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
195 |
fun dest_recTs T = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
196 |
let val ((c, Ts), U) = dest_recT T |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
197 |
in (c, Ts) :: dest_recTs U |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
198 |
end handle TYPE _ => []; |
14255 | 199 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
200 |
fun last_extT T = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
201 |
let val ((c, Ts), U) = dest_recT T |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
202 |
in (case last_extT U of |
15531 | 203 |
NONE => SOME (c,Ts) |
204 |
| SOME l => SOME l) |
|
205 |
end handle TYPE _ => NONE |
|
14255 | 206 |
|
17261 | 207 |
fun rec_id i T = |
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
208 |
let val rTs = dest_recTs T |
15570 | 209 |
val rTs' = if i < 0 then rTs else Library.take (i,rTs) |
210 |
in Library.foldl (fn (s,(c,T)) => s ^ c) ("",rTs') end; |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
211 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
212 |
(*** extend theory by record definition ***) |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
213 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
214 |
(** record info **) |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
215 |
|
14255 | 216 |
(* type record_info and parent_info *) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
217 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
218 |
type record_info = |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
219 |
{args: (string * sort) list, |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
220 |
parent: (typ list * string) option, |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
221 |
fields: (string * typ) list, |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
222 |
extension: (string * typ list), |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
223 |
induct: thm |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
224 |
}; |
11927
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
225 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
226 |
fun make_record_info args parent fields extension induct = |
17261 | 227 |
{args = args, parent = parent, fields = fields, extension = extension, |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
228 |
induct = induct}: record_info; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
229 |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
230 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
231 |
type parent_info = |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
232 |
{name: string, |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
233 |
fields: (string * typ) list, |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
234 |
extension: (string * typ list), |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
235 |
induct: thm |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
236 |
}; |
11927
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
wenzelm
parents:
11923
diff
changeset
|
237 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
238 |
fun make_parent_info name fields extension induct = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
239 |
{name = name, fields = fields, extension = extension, induct = induct}: parent_info; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
240 |
|
22846 | 241 |
|
242 |
(* theory data *) |
|
5001 | 243 |
|
7178 | 244 |
type record_data = |
245 |
{records: record_info Symtab.table, |
|
246 |
sel_upd: |
|
247 |
{selectors: unit Symtab.table, |
|
248 |
updates: string Symtab.table, |
|
249 |
simpset: Simplifier.simpset}, |
|
14255 | 250 |
equalities: thm Symtab.table, |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
251 |
extinjects: thm list, |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
252 |
extsplit: thm Symtab.table, (* maps extension name to split rule *) |
17261 | 253 |
splits: (thm*thm*thm*thm) Symtab.table, (* !!,!,EX - split-equalities,induct rule *) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
254 |
extfields: (string*typ) list Symtab.table, (* maps extension to its fields *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
255 |
fieldext: (string*typ list) Symtab.table (* maps field to its extension *) |
14255 | 256 |
}; |
7178 | 257 |
|
17261 | 258 |
fun make_record_data |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
259 |
records sel_upd equalities extinjects extsplit splits extfields fieldext = |
17261 | 260 |
{records = records, sel_upd = sel_upd, |
261 |
equalities = equalities, extinjects=extinjects, extsplit = extsplit, splits = splits, |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
262 |
extfields = extfields, fieldext = fieldext }: record_data; |
7178 | 263 |
|
16458 | 264 |
structure RecordsData = TheoryDataFun |
22846 | 265 |
( |
7178 | 266 |
type T = record_data; |
267 |
val empty = |
|
268 |
make_record_data Symtab.empty |
|
269 |
{selectors = Symtab.empty, updates = Symtab.empty, simpset = HOL_basic_ss} |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
270 |
Symtab.empty [] Symtab.empty Symtab.empty Symtab.empty Symtab.empty; |
7178 | 271 |
|
6556 | 272 |
val copy = I; |
16458 | 273 |
val extend = I; |
274 |
fun merge _ |
|
7178 | 275 |
({records = recs1, |
276 |
sel_upd = {selectors = sels1, updates = upds1, simpset = ss1}, |
|
14255 | 277 |
equalities = equalities1, |
17261 | 278 |
extinjects = extinjects1, |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
279 |
extsplit = extsplit1, |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
280 |
splits = splits1, |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
281 |
extfields = extfields1, |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
282 |
fieldext = fieldext1}, |
7178 | 283 |
{records = recs2, |
284 |
sel_upd = {selectors = sels2, updates = upds2, simpset = ss2}, |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
285 |
equalities = equalities2, |
17261 | 286 |
extinjects = extinjects2, |
287 |
extsplit = extsplit2, |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
288 |
splits = splits2, |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
289 |
extfields = extfields2, |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
290 |
fieldext = fieldext2}) = |
17261 | 291 |
make_record_data |
7178 | 292 |
(Symtab.merge (K true) (recs1, recs2)) |
293 |
{selectors = Symtab.merge (K true) (sels1, sels2), |
|
294 |
updates = Symtab.merge (K true) (upds1, upds2), |
|
295 |
simpset = Simplifier.merge_ss (ss1, ss2)} |
|
22634 | 296 |
(Symtab.merge Thm.eq_thm_prop (equalities1, equalities2)) |
297 |
(Library.merge Thm.eq_thm_prop (extinjects1, extinjects2)) |
|
298 |
(Symtab.merge Thm.eq_thm_prop (extsplit1,extsplit2)) |
|
17261 | 299 |
(Symtab.merge (fn ((a,b,c,d),(w,x,y,z)) |
300 |
=> Thm.eq_thm (a,w) andalso Thm.eq_thm (b,x) andalso |
|
301 |
Thm.eq_thm (c,y) andalso Thm.eq_thm (d,z)) |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
302 |
(splits1, splits2)) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
303 |
(Symtab.merge (K true) (extfields1,extfields2)) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
304 |
(Symtab.merge (K true) (fieldext1,fieldext2)); |
22846 | 305 |
); |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
306 |
|
22846 | 307 |
fun print_records thy = |
308 |
let |
|
309 |
val {records = recs, ...} = RecordsData.get thy; |
|
26943
aec0d97a01c4
moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents:
26626
diff
changeset
|
310 |
val prt_typ = Syntax.pretty_typ_global thy; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
311 |
|
22846 | 312 |
fun pretty_parent NONE = [] |
313 |
| pretty_parent (SOME (Ts, name)) = |
|
314 |
[Pretty.block [prt_typ (Type (name, Ts)), Pretty.str " +"]]; |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
315 |
|
22846 | 316 |
fun pretty_field (c, T) = Pretty.block |
317 |
[Pretty.str (Sign.extern_const thy c), Pretty.str " ::", |
|
318 |
Pretty.brk 1, Pretty.quote (prt_typ T)]; |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
319 |
|
22846 | 320 |
fun pretty_record (name, {args, parent, fields, ...}: record_info) = |
321 |
Pretty.block (Pretty.fbreaks (Pretty.block |
|
322 |
[prt_typ (Type (name, map TFree args)), Pretty.str " = "] :: |
|
323 |
pretty_parent parent @ map pretty_field fields)); |
|
324 |
in map pretty_record (Symtab.dest recs) |> Pretty.chunks |> Pretty.writeln end; |
|
5006 | 325 |
|
16458 | 326 |
|
7178 | 327 |
(* access 'records' *) |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
328 |
|
17412 | 329 |
val get_record = Symtab.lookup o #records o RecordsData.get; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
330 |
|
4890 | 331 |
fun put_record name info thy = |
7178 | 332 |
let |
17261 | 333 |
val {records, sel_upd, equalities, extinjects,extsplit,splits,extfields,fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
334 |
RecordsData.get thy; |
17412 | 335 |
val data = make_record_data (Symtab.update (name, info) records) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
336 |
sel_upd equalities extinjects extsplit splits extfields fieldext; |
7178 | 337 |
in RecordsData.put data thy end; |
338 |
||
22846 | 339 |
|
7178 | 340 |
(* access 'sel_upd' *) |
341 |
||
16458 | 342 |
val get_sel_upd = #sel_upd o RecordsData.get; |
7178 | 343 |
|
17510 | 344 |
val is_selector = Symtab.defined o #selectors o get_sel_upd; |
17412 | 345 |
val get_updates = Symtab.lookup o #updates o get_sel_upd; |
17892 | 346 |
fun get_simpset thy = Simplifier.theory_context thy (#simpset (get_sel_upd thy)); |
7178 | 347 |
|
29004 | 348 |
fun put_sel_upd names simps = RecordsData.map (fn {records, |
349 |
sel_upd = {selectors, updates, simpset}, |
|
350 |
equalities, extinjects, extsplit, splits, extfields, fieldext} => |
|
351 |
make_record_data records |
|
352 |
{selectors = fold (fn name => Symtab.update (name, ())) names selectors, |
|
353 |
updates = fold (fn name => Symtab.update ((suffix updateN) name, name)) names updates, |
|
354 |
simpset = Simplifier.addsimps (simpset, simps)} |
|
355 |
equalities extinjects extsplit splits extfields fieldext); |
|
7178 | 356 |
|
22846 | 357 |
|
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
358 |
(* access 'equalities' *) |
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
359 |
|
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
360 |
fun add_record_equalities name thm thy = |
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
361 |
let |
17261 | 362 |
val {records, sel_upd, equalities, extinjects, extsplit, splits, extfields,fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
363 |
RecordsData.get thy; |
17261 | 364 |
val data = make_record_data records sel_upd |
17412 | 365 |
(Symtab.update_new (name, thm) equalities) extinjects extsplit |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
366 |
splits extfields fieldext; |
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
367 |
in RecordsData.put data thy end; |
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
368 |
|
17412 | 369 |
val get_equalities =Symtab.lookup o #equalities o RecordsData.get; |
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
370 |
|
22846 | 371 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
372 |
(* access 'extinjects' *) |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
373 |
|
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
374 |
fun add_extinjects thm thy = |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
375 |
let |
17261 | 376 |
val {records, sel_upd, equalities, extinjects, extsplit, splits, extfields,fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
377 |
RecordsData.get thy; |
22846 | 378 |
val data = |
379 |
make_record_data records sel_upd equalities (insert Thm.eq_thm_prop thm extinjects) extsplit |
|
380 |
splits extfields fieldext; |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
381 |
in RecordsData.put data thy end; |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
382 |
|
22634 | 383 |
val get_extinjects = rev o #extinjects o RecordsData.get; |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
384 |
|
22846 | 385 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
386 |
(* access 'extsplit' *) |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
387 |
|
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
388 |
fun add_extsplit name thm thy = |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
389 |
let |
17261 | 390 |
val {records, sel_upd, equalities, extinjects, extsplit, splits, extfields,fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
391 |
RecordsData.get thy; |
17261 | 392 |
val data = make_record_data records sel_upd |
17412 | 393 |
equalities extinjects (Symtab.update_new (name, thm) extsplit) splits |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
394 |
extfields fieldext; |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
395 |
in RecordsData.put data thy end; |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
396 |
|
17412 | 397 |
val get_extsplit = Symtab.lookup o #extsplit o RecordsData.get; |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
398 |
|
26088 | 399 |
|
14255 | 400 |
(* access 'splits' *) |
401 |
||
402 |
fun add_record_splits name thmP thy = |
|
403 |
let |
|
17261 | 404 |
val {records, sel_upd, equalities, extinjects, extsplit, splits, extfields,fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
405 |
RecordsData.get thy; |
17261 | 406 |
val data = make_record_data records sel_upd |
17412 | 407 |
equalities extinjects extsplit (Symtab.update_new (name, thmP) splits) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
408 |
extfields fieldext; |
14255 | 409 |
in RecordsData.put data thy end; |
410 |
||
17412 | 411 |
val get_splits = Symtab.lookup o #splits o RecordsData.get; |
14255 | 412 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
413 |
|
26088 | 414 |
(* parent/extension of named record *) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
415 |
|
26088 | 416 |
val get_parent = (Option.join o Option.map #parent) oo (Symtab.lookup o #records o RecordsData.get); |
417 |
val get_extension = Option.map #extension oo (Symtab.lookup o #records o RecordsData.get); |
|
17261 | 418 |
|
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
419 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
420 |
(* access 'extfields' *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
421 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
422 |
fun add_extfields name fields thy = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
423 |
let |
17261 | 424 |
val {records, sel_upd, equalities, extinjects, extsplit,splits, extfields, fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
425 |
RecordsData.get thy; |
17261 | 426 |
val data = make_record_data records sel_upd |
427 |
equalities extinjects extsplit splits |
|
17412 | 428 |
(Symtab.update_new (name, fields) extfields) fieldext; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
429 |
in RecordsData.put data thy end; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
430 |
|
17412 | 431 |
val get_extfields = Symtab.lookup o #extfields o RecordsData.get; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
432 |
|
18858 | 433 |
fun get_extT_fields thy T = |
15059 | 434 |
let |
435 |
val ((name,Ts),moreT) = dest_recT T; |
|
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
436 |
val recname = let val (nm::recn::rst) = rev (Long_Name.explode name) |
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
437 |
in Long_Name.implode (rev (nm::rst)) end; |
15059 | 438 |
val midx = maxidx_of_typs (moreT::Ts); |
19748 | 439 |
val varifyT = varifyT midx; |
18858 | 440 |
val {records,extfields,...} = RecordsData.get thy; |
18931 | 441 |
val (flds,(more,_)) = split_last (Symtab.lookup_list extfields name); |
17412 | 442 |
val args = map varifyT (snd (#extension (the (Symtab.lookup records recname)))); |
15058 | 443 |
|
19748 | 444 |
val subst = fold (Sign.typ_match thy) (but_last args ~~ but_last Ts) (Vartab.empty); |
15059 | 445 |
val flds' = map (apsnd ((Envir.norm_type subst) o varifyT)) flds; |
446 |
in (flds',(more,moreT)) end; |
|
15058 | 447 |
|
18858 | 448 |
fun get_recT_fields thy T = |
17261 | 449 |
let |
18858 | 450 |
val (root_flds,(root_more,root_moreT)) = get_extT_fields thy T; |
17261 | 451 |
val (rest_flds,rest_more) = |
18858 | 452 |
if is_recT root_moreT then get_recT_fields thy root_moreT |
15059 | 453 |
else ([],(root_more,root_moreT)); |
454 |
in (root_flds@rest_flds,rest_more) end; |
|
455 |
||
15058 | 456 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
457 |
(* access 'fieldext' *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
458 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
459 |
fun add_fieldext extname_types fields thy = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
460 |
let |
17261 | 461 |
val {records, sel_upd, equalities, extinjects, extsplit, splits, extfields, fieldext} = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
462 |
RecordsData.get thy; |
17261 | 463 |
val fieldext' = |
17412 | 464 |
fold (fn field => Symtab.update_new (field, extname_types)) fields fieldext; |
17261 | 465 |
val data=make_record_data records sel_upd equalities extinjects extsplit |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
466 |
splits extfields fieldext'; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
467 |
in RecordsData.put data thy end; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
468 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
469 |
|
17412 | 470 |
val get_fieldext = Symtab.lookup o #fieldext o RecordsData.get; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
471 |
|
21962 | 472 |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
473 |
(* parent records *) |
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
474 |
|
15531 | 475 |
fun add_parents thy NONE parents = parents |
476 |
| add_parents thy (SOME (types, name)) parents = |
|
12247 | 477 |
let |
478 |
fun err msg = error (msg ^ " parent record " ^ quote name); |
|
12255 | 479 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
480 |
val {args, parent, fields, extension, induct} = |
15531 | 481 |
(case get_record thy name of SOME info => info | NONE => err "Unknown"); |
12247 | 482 |
val _ = if length types <> length args then err "Bad number of arguments for" else (); |
12255 | 483 |
|
12247 | 484 |
fun bad_inst ((x, S), T) = |
22578 | 485 |
if Sign.of_sort thy (T, S) then NONE else SOME x |
15570 | 486 |
val bads = List.mapPartial bad_inst (args ~~ types); |
21962 | 487 |
val _ = null bads orelse err ("Ill-sorted instantiation of " ^ commas bads ^ " in"); |
12255 | 488 |
|
12247 | 489 |
val inst = map fst args ~~ types; |
17377 | 490 |
val subst = Term.map_type_tfree (the o AList.lookup (op =) inst o fst); |
15570 | 491 |
val parent' = Option.map (apfst (map subst)) parent; |
12247 | 492 |
val fields' = map (apsnd subst) fields; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
493 |
val extension' = apsnd (map subst) extension; |
12247 | 494 |
in |
12255 | 495 |
add_parents thy parent' |
21962 | 496 |
(make_parent_info name fields' extension' induct :: parents) |
12247 | 497 |
end; |
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
498 |
|
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
499 |
|
21962 | 500 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
501 |
(** concrete syntax for records **) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
502 |
|
22693 | 503 |
(* decode type *) |
504 |
||
505 |
fun decode_type thy t = |
|
506 |
let |
|
23578 | 507 |
fun get_sort xs n = AList.lookup (op =) xs (n: indexname) |> the_default (Sign.defaultS thy); |
22693 | 508 |
val map_sort = Sign.intern_sort thy; |
509 |
in |
|
510 |
Syntax.typ_of_term (get_sort (Syntax.term_sorts map_sort t)) map_sort t |
|
511 |
|> Sign.intern_tycons thy |
|
512 |
end; |
|
513 |
||
514 |
||
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
515 |
(* parse translations *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
516 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
517 |
fun gen_field_tr mark sfx (t as Const (c, _) $ Const (name, _) $ arg) = |
25705 | 518 |
if c = mark then Syntax.const (suffix sfx name) $ (Abs ("_",dummyT, arg)) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
519 |
else raise TERM ("gen_field_tr: " ^ mark, [t]) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
520 |
| gen_field_tr mark _ t = raise TERM ("gen_field_tr: " ^ mark, [t]); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
521 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
522 |
fun gen_fields_tr sep mark sfx (tm as Const (c, _) $ t $ u) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
523 |
if c = sep then gen_field_tr mark sfx t :: gen_fields_tr sep mark sfx u |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
524 |
else [gen_field_tr mark sfx tm] |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
525 |
| gen_fields_tr _ mark sfx tm = [gen_field_tr mark sfx tm]; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
526 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
527 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
528 |
fun record_update_tr [t, u] = |
21078 | 529 |
Library.foldr (op $) (rev (gen_fields_tr "_updates" "_update" updateN u), t) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
530 |
| record_update_tr ts = raise TERM ("record_update_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
531 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
532 |
fun update_name_tr (Free (x, T) :: ts) = Free (suffix updateN x, T) $$ ts |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
533 |
| update_name_tr (Const (x, T) :: ts) = Const (suffix updateN x, T) $$ ts |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
534 |
| update_name_tr (((c as Const ("_constrain", _)) $ t $ ty) :: ts) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
535 |
(c $ update_name_tr [t] $ (Syntax.const "fun" $ ty $ Syntax.const "dummy")) $$ ts |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
536 |
| update_name_tr ts = raise TERM ("update_name_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
537 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
538 |
fun dest_ext_field mark (t as (Const (c,_) $ Const (name,_) $ arg)) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
539 |
if c = mark then (name,arg) else raise TERM ("dest_ext_field: " ^ mark, [t]) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
540 |
| dest_ext_field _ t = raise TERM ("dest_ext_field", [t]) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
541 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
542 |
fun dest_ext_fields sep mark (trm as (Const (c,_) $ t $ u)) = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
543 |
if c = sep then dest_ext_field mark t::dest_ext_fields sep mark u |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
544 |
else [dest_ext_field mark trm] |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
545 |
| dest_ext_fields _ mark t = [dest_ext_field mark t] |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
546 |
|
21772 | 547 |
fun gen_ext_fields_tr sep mark sfx more ctxt t = |
17261 | 548 |
let |
21772 | 549 |
val thy = ProofContext.theory_of ctxt; |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
550 |
val msg = "error in record input: "; |
17261 | 551 |
val fieldargs = dest_ext_fields sep mark t; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
552 |
fun splitargs (field::fields) ((name,arg)::fargs) = |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
553 |
if can (unsuffix name) field |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
554 |
then let val (args,rest) = splitargs fields fargs |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
555 |
in (arg::args,rest) end |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
556 |
else raise TERM (msg ^ "expecting field " ^ field ^ " but got " ^ name, [t]) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
557 |
| splitargs [] (fargs as (_::_)) = ([],fargs) |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
558 |
| splitargs (_::_) [] = raise TERM (msg ^ "expecting more fields", [t]) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
559 |
| splitargs _ _ = ([],[]); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
560 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
561 |
fun mk_ext (fargs as (name,arg)::_) = |
18858 | 562 |
(case get_fieldext thy (Sign.intern_const thy name) of |
563 |
SOME (ext,_) => (case get_extfields thy ext of |
|
17261 | 564 |
SOME flds |
565 |
=> let val (args,rest) = |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
566 |
splitargs (map fst (but_last flds)) fargs; |
17261 | 567 |
val more' = mk_ext rest; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
568 |
in list_comb (Syntax.const (suffix sfx ext),args@[more']) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
569 |
end |
15531 | 570 |
| NONE => raise TERM(msg ^ "no fields defined for " |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
571 |
^ ext,[t])) |
15531 | 572 |
| NONE => raise TERM (msg ^ name ^" is no proper field",[t])) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
573 |
| mk_ext [] = more |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
574 |
|
17261 | 575 |
in mk_ext fieldargs end; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
576 |
|
21772 | 577 |
fun gen_ext_type_tr sep mark sfx more ctxt t = |
17261 | 578 |
let |
21772 | 579 |
val thy = ProofContext.theory_of ctxt; |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
580 |
val msg = "error in record-type input: "; |
17261 | 581 |
val fieldargs = dest_ext_fields sep mark t; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
582 |
fun splitargs (field::fields) ((name,arg)::fargs) = |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
583 |
if can (unsuffix name) field |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
584 |
then let val (args,rest) = splitargs fields fargs |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
585 |
in (arg::args,rest) end |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
586 |
else raise TERM (msg ^ "expecting field " ^ field ^ " but got " ^ name, [t]) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
587 |
| splitargs [] (fargs as (_::_)) = ([],fargs) |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
588 |
| splitargs (_::_) [] = raise TERM (msg ^ "expecting more fields", [t]) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
589 |
| splitargs _ _ = ([],[]); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
590 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
591 |
fun mk_ext (fargs as (name,arg)::_) = |
18858 | 592 |
(case get_fieldext thy (Sign.intern_const thy name) of |
17261 | 593 |
SOME (ext,alphas) => |
18858 | 594 |
(case get_extfields thy ext of |
17261 | 595 |
SOME flds |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
596 |
=> (let |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
597 |
val flds' = but_last flds; |
17261 | 598 |
val types = map snd flds'; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
599 |
val (args,rest) = splitargs (map fst flds') fargs; |
22693 | 600 |
val argtypes = map (Sign.certify_typ thy o decode_type thy) args; |
24867 | 601 |
val midx = fold (fn T => fn i => Int.max (maxidx_of_typ T, i)) |
19748 | 602 |
argtypes 0; |
603 |
val varifyT = varifyT midx; |
|
604 |
val vartypes = map varifyT types; |
|
605 |
||
606 |
val subst = fold (Sign.typ_match thy) (vartypes ~~ argtypes) |
|
607 |
Vartab.empty; |
|
17261 | 608 |
val alphas' = map ((Syntax.term_of_typ (! Syntax.show_sorts)) o |
19748 | 609 |
Envir.norm_type subst o varifyT) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
610 |
(but_last alphas); |
17261 | 611 |
|
612 |
val more' = mk_ext rest; |
|
613 |
in list_comb (Syntax.const (suffix sfx ext),alphas'@[more']) |
|
19750 | 614 |
end handle TYPE_MATCH => raise |
14709
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
schirmer
parents:
14702
diff
changeset
|
615 |
TERM (msg ^ "type is no proper record (extension)", [t])) |
15531 | 616 |
| NONE => raise TERM (msg ^ "no fields defined for " ^ ext,[t])) |
617 |
| NONE => raise TERM (msg ^ name ^" is no proper field",[t])) |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
618 |
| mk_ext [] = more |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
619 |
|
17261 | 620 |
in mk_ext fieldargs end; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
621 |
|
21772 | 622 |
fun gen_adv_record_tr sep mark sfx unit ctxt [t] = |
623 |
gen_ext_fields_tr sep mark sfx unit ctxt t |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
624 |
| gen_adv_record_tr _ _ _ _ _ ts = raise TERM ("gen_record_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
625 |
|
21772 | 626 |
fun gen_adv_record_scheme_tr sep mark sfx ctxt [t, more] = |
627 |
gen_ext_fields_tr sep mark sfx more ctxt t |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
628 |
| gen_adv_record_scheme_tr _ _ _ _ ts = raise TERM ("gen_record_scheme_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
629 |
|
21772 | 630 |
fun gen_adv_record_type_tr sep mark sfx unit ctxt [t] = |
631 |
gen_ext_type_tr sep mark sfx unit ctxt t |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
632 |
| gen_adv_record_type_tr _ _ _ _ _ ts = raise TERM ("gen_record_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
633 |
|
21772 | 634 |
fun gen_adv_record_type_scheme_tr sep mark sfx ctxt [t, more] = |
635 |
gen_ext_type_tr sep mark sfx more ctxt t |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
636 |
| gen_adv_record_type_scheme_tr _ _ _ _ ts = raise TERM ("gen_record_scheme_tr", ts); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
637 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
638 |
val adv_record_tr = gen_adv_record_tr "_fields" "_field" extN HOLogic.unit; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
639 |
val adv_record_scheme_tr = gen_adv_record_scheme_tr "_fields" "_field" extN; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
640 |
|
17261 | 641 |
val adv_record_type_tr = |
642 |
gen_adv_record_type_tr "_field_types" "_field_type" ext_typeN |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
643 |
(Syntax.term_of_typ false (HOLogic.unitT)); |
17261 | 644 |
val adv_record_type_scheme_tr = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
645 |
gen_adv_record_type_scheme_tr "_field_types" "_field_type" ext_typeN; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
646 |
|
15215 | 647 |
|
24867 | 648 |
val parse_translation = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
649 |
[("_record_update", record_update_tr), |
17261 | 650 |
("_update_name", update_name_tr)]; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
651 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
652 |
|
24867 | 653 |
val adv_parse_translation = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
654 |
[("_record",adv_record_tr), |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
655 |
("_record_scheme",adv_record_scheme_tr), |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
656 |
("_record_type",adv_record_type_tr), |
17261 | 657 |
("_record_type_scheme",adv_record_type_scheme_tr)]; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
658 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
659 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
660 |
(* print translations *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
661 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
662 |
val print_record_type_abbr = ref true; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
663 |
val print_record_type_as_fields = ref true; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
664 |
|
25705 | 665 |
fun gen_field_upds_tr' mark sfx (tm as Const (name_field, _) $ k $ u) = |
666 |
let val t = (case k of (Abs (_,_,(Abs (_,_,t)$Bound 0))) |
|
667 |
=> if null (loose_bnos t) then t else raise Match |
|
668 |
| Abs (x,_,t) => if null (loose_bnos t) then t else raise Match |
|
669 |
| _ => raise Match) |
|
670 |
||
671 |
(* (case k of (Const ("K_record",_)$t) => t |
|
672 |
| Abs (x,_,Const ("K_record",_)$t$Bound 0) => t |
|
673 |
| _ => raise Match)*) |
|
674 |
in |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
675 |
(case try (unsuffix sfx) name_field of |
15531 | 676 |
SOME name => |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
677 |
apfst (cons (Syntax.const mark $ Syntax.free name $ t)) (gen_field_upds_tr' mark sfx u) |
15531 | 678 |
| NONE => ([], tm)) |
25705 | 679 |
end |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
680 |
| gen_field_upds_tr' _ _ tm = ([], tm); |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
681 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
682 |
fun record_update_tr' tm = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
683 |
let val (ts, u) = gen_field_upds_tr' "_update" updateN tm in |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
684 |
if null ts then raise Match |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
685 |
else Syntax.const "_record_update" $ u $ |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
686 |
foldr1 (fn (v, w) => Syntax.const "_updates" $ v $ w) (rev ts) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
687 |
end; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
688 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
689 |
fun gen_field_tr' sfx tr' name = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
690 |
let val name_sfx = suffix sfx name |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
691 |
in (name_sfx, fn [t, u] => tr' (Syntax.const name_sfx $ t $ u) | _ => raise Match) end; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
692 |
|
21772 | 693 |
fun record_tr' sep mark record record_scheme unit ctxt t = |
17261 | 694 |
let |
21772 | 695 |
val thy = ProofContext.theory_of ctxt; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
696 |
fun field_lst t = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
697 |
(case strip_comb t of |
17600 | 698 |
(Const (ext,_),args as (_::_)) |
18858 | 699 |
=> (case try (unsuffix extN) (Sign.intern_const thy ext) of |
17261 | 700 |
SOME ext' |
18858 | 701 |
=> (case get_extfields thy ext' of |
17261 | 702 |
SOME flds |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
703 |
=> (let |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
704 |
val (f::fs) = but_last (map fst flds); |
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
705 |
val flds' = Sign.extern_const thy f :: map Long_Name.base_name fs; |
17261 | 706 |
val (args',more) = split_last args; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
707 |
in (flds'~~args')@field_lst more end |
19841 | 708 |
handle Library.UnequalLengths => [("",t)]) |
15531 | 709 |
| NONE => [("",t)]) |
710 |
| NONE => [("",t)]) |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
711 |
| _ => [("",t)]) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
712 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
713 |
val (flds,(_,more)) = split_last (field_lst t); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
714 |
val _ = if null flds then raise Match else (); |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
715 |
val flds' = map (fn (n,t)=>Syntax.const mark$Syntax.const n$t) flds; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
716 |
val flds'' = foldr1 (fn (x,y) => Syntax.const sep$x$y) flds'; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
717 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
718 |
in if unit more |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
719 |
then Syntax.const record$flds'' |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
720 |
else Syntax.const record_scheme$flds''$more |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
721 |
end |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
722 |
|
17261 | 723 |
fun gen_record_tr' name = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
724 |
let val name_sfx = suffix extN name; |
26065 | 725 |
val unit = (fn Const (@{const_syntax "Product_Type.Unity"},_) => true | _ => false); |
21772 | 726 |
fun tr' ctxt ts = record_tr' "_fields" "_field" "_record" "_record_scheme" unit ctxt |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
727 |
(list_comb (Syntax.const name_sfx,ts)) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
728 |
in (name_sfx,tr') |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
729 |
end |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
730 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
731 |
fun print_translation names = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
732 |
map (gen_field_tr' updateN record_update_tr') names; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
733 |
|
19748 | 734 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
735 |
(* record_type_abbr_tr' tries to reconstruct the record name type abbreviation from *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
736 |
(* the (nested) extension types. *) |
21772 | 737 |
fun record_type_abbr_tr' default_tr' abbr alphas zeta lastExt schemeT ctxt tm = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
738 |
let |
21772 | 739 |
val thy = ProofContext.theory_of ctxt; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
740 |
(* tm is term representation of a (nested) field type. We first reconstruct the *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
741 |
(* type from tm so that we can continue on the type level rather then the term level.*) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
742 |
|
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
743 |
(* WORKAROUND: |
17261 | 744 |
* If a record type occurs in an error message of type inference there |
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
745 |
* may be some internal frees donoted by ??: |
17261 | 746 |
* (Const "_tfree",_)$Free ("??'a",_). |
747 |
||
748 |
* This will unfortunately be translated to Type ("??'a",[]) instead of |
|
749 |
* TFree ("??'a",_) by typ_of_term, which will confuse unify below. |
|
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
750 |
* fixT works around. |
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
751 |
*) |
17261 | 752 |
fun fixT (T as Type (x,[])) = |
18858 | 753 |
if String.isPrefix "??'" x then TFree (x,Sign.defaultS thy) else T |
15273
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
754 |
| fixT (Type (x,xs)) = Type (x,map fixT xs) |
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
schirmer
parents:
15258
diff
changeset
|
755 |
| fixT T = T; |
17261 | 756 |
|
22693 | 757 |
val T = fixT (decode_type thy tm); |
19748 | 758 |
val midx = maxidx_of_typ T; |
759 |
val varifyT = varifyT midx; |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
760 |
|
17261 | 761 |
fun mk_type_abbr subst name alphas = |
19748 | 762 |
let val abbrT = Type (name, map (fn a => varifyT (TFree (a, Sign.defaultS thy))) alphas); |
17261 | 763 |
in Syntax.term_of_typ (! Syntax.show_sorts) |
18858 | 764 |
(Sign.extern_typ thy (Envir.norm_type subst abbrT)) end; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
765 |
|
24867 | 766 |
fun match rT T = (Sign.typ_match thy (varifyT rT,T) |
19748 | 767 |
Vartab.empty); |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
768 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
769 |
in if !print_record_type_abbr |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
770 |
then (case last_extT T of |
17261 | 771 |
SOME (name,_) |
772 |
=> if name = lastExt |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
773 |
then |
17261 | 774 |
(let |
19748 | 775 |
val subst = match schemeT T |
17261 | 776 |
in |
19748 | 777 |
if HOLogic.is_unitT (Envir.norm_type subst (varifyT (TFree(zeta,Sign.defaultS thy)))) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
778 |
then mk_type_abbr subst abbr alphas |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
779 |
else mk_type_abbr subst (suffix schemeN abbr) (alphas@[zeta]) |
21772 | 780 |
end handle TYPE_MATCH => default_tr' ctxt tm) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
781 |
else raise Match (* give print translation of specialised record a chance *) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
782 |
| _ => raise Match) |
21772 | 783 |
else default_tr' ctxt tm |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
784 |
end |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
785 |
|
21772 | 786 |
fun record_type_tr' sep mark record record_scheme ctxt t = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
787 |
let |
21772 | 788 |
val thy = ProofContext.theory_of ctxt; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
789 |
|
22693 | 790 |
val T = decode_type thy t; |
791 |
val varifyT = varifyT (Term.maxidx_of_typ T); |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
792 |
|
18858 | 793 |
fun term_of_type T = Syntax.term_of_typ (!Syntax.show_sorts) (Sign.extern_typ thy T); |
17261 | 794 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
795 |
fun field_lst T = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
796 |
(case T of |
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
797 |
Type (ext, args) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
798 |
=> (case try (unsuffix ext_typeN) ext of |
17261 | 799 |
SOME ext' |
18858 | 800 |
=> (case get_extfields thy ext' of |
17261 | 801 |
SOME flds |
18858 | 802 |
=> (case get_fieldext thy (fst (hd flds)) of |
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
803 |
SOME (_, alphas) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
804 |
=> (let |
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
805 |
val (f :: fs) = but_last flds; |
18858 | 806 |
val flds' = apfst (Sign.extern_const thy) f |
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
807 |
:: map (apfst Long_Name.base_name) fs; |
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
808 |
val (args', more) = split_last args; |
19748 | 809 |
val alphavars = map varifyT (but_last alphas); |
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
810 |
val subst = fold2 (curry (Sign.typ_match thy)) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
811 |
alphavars args' Vartab.empty; |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
812 |
val flds'' = (map o apsnd) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
813 |
(Envir.norm_type subst o varifyT) flds'; |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
814 |
in flds'' @ field_lst more end |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
815 |
handle TYPE_MATCH => [("", T)] |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
816 |
| Library.UnequalLengths => [("", T)]) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
817 |
| NONE => [("", T)]) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
818 |
| NONE => [("", T)]) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
819 |
| NONE => [("", T)]) |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
820 |
| _ => [("", T)]) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
821 |
|
22219
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
822 |
val (flds, (_, moreT)) = split_last (field_lst T); |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
823 |
val flds' = map (fn (n, T) => Syntax.const mark $ Syntax.const n $ term_of_type T) flds; |
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
haftmann
parents:
21962
diff
changeset
|
824 |
val flds'' = foldr1 (fn (x, y) => Syntax.const sep $ x $ y) flds' handle Empty => raise Match; |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
825 |
|
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
826 |
in if not (!print_record_type_as_fields) orelse null flds then raise Match |
17261 | 827 |
else if moreT = HOLogic.unitT |
828 |
then Syntax.const record$flds'' |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
829 |
else Syntax.const record_scheme$flds''$term_of_type moreT |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
830 |
end |
17261 | 831 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
832 |
|
17261 | 833 |
fun gen_record_type_tr' name = |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
834 |
let val name_sfx = suffix ext_typeN name; |
21772 | 835 |
fun tr' ctxt ts = record_type_tr' "_field_types" "_field_type" |
836 |
"_record_type" "_record_type_scheme" ctxt |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
837 |
(list_comb (Syntax.const name_sfx,ts)) |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
838 |
in (name_sfx,tr') |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
839 |
end |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
840 |
|
17261 | 841 |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
842 |
fun gen_record_type_abbr_tr' abbr alphas zeta lastExt schemeT name = |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
843 |
let val name_sfx = suffix ext_typeN name; |
17261 | 844 |
val default_tr' = record_type_tr' "_field_types" "_field_type" |
845 |
"_record_type" "_record_type_scheme" |
|
21772 | 846 |
fun tr' ctxt ts = |
847 |
record_type_abbr_tr' default_tr' abbr alphas zeta lastExt schemeT ctxt |
|
18858 | 848 |
(list_comb (Syntax.const name_sfx,ts)) |
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
849 |
in (name_sfx, tr') end; |
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
850 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
851 |
(** record simprocs **) |
14358 | 852 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
853 |
val record_quick_and_dirty_sensitive = ref false; |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
854 |
|
15215 | 855 |
|
18858 | 856 |
fun quick_and_dirty_prove stndrd thy asms prop tac = |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
857 |
if !record_quick_and_dirty_sensitive andalso !quick_and_dirty |
20049 | 858 |
then Goal.prove (ProofContext.init thy) [] [] |
859 |
(Logic.list_implies (map Logic.varify asms,Logic.varify prop)) |
|
29064 | 860 |
(K (SkipProof.cheat_tac @{theory HOL})) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
861 |
(* standard can take quite a while for large records, thats why |
17261 | 862 |
* we varify the proposition manually here.*) |
20049 | 863 |
else let val prf = Goal.prove (ProofContext.init thy) [] asms prop tac; |
17261 | 864 |
in if stndrd then standard prf else prf end; |
15215 | 865 |
|
17261 | 866 |
fun quick_and_dirty_prf noopt opt () = |
867 |
if !record_quick_and_dirty_sensitive andalso !quick_and_dirty |
|
15215 | 868 |
then noopt () |
869 |
else opt (); |
|
4867
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
wenzelm
parents:
diff
changeset
|
870 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
871 |
local |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
872 |
fun abstract_over_fun_app (Abs (f,fT,t)) = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
873 |
let |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
874 |
val (f',t') = Term.dest_abs (f,fT,t); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
875 |
val T = domain_type fT; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
876 |
val (x,T') = hd (Term.variant_frees t' [("x",T)]); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
877 |
val f_x = Free (f',fT)$(Free (x,T')); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
878 |
fun is_constr (Const (c,_)$_) = can (unsuffix extN) c |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
879 |
| is_constr _ = false; |
24867 | 880 |
fun subst (t as u$w) = if Free (f',fT)=u |
881 |
then if is_constr w then f_x |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
882 |
else raise TERM ("abstract_over_fun_app",[t]) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
883 |
else subst u$subst w |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
884 |
| subst (Abs (x,T,t)) = (Abs (x,T,subst t)) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
885 |
| subst t = t |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
886 |
val t'' = abstract_over (f_x,subst t'); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
887 |
val vars = strip_qnt_vars "all" t''; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
888 |
val bdy = strip_qnt_body "all" t''; |
24867 | 889 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
890 |
in list_abs ((x,T')::vars,bdy) end |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
891 |
| abstract_over_fun_app t = raise TERM ("abstract_over_fun_app",[t]); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
892 |
(* Generates a theorem of the kind: |
24867 | 893 |
* !!f x*. PROP P (f ( r x* ) x* == !!r x*. PROP P r x* |
894 |
*) |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
895 |
fun mk_fun_apply_eq (Abs (f, fT, t)) thy = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
896 |
let |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
897 |
val rT = domain_type fT; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
898 |
val vars = Term.strip_qnt_vars "all" t; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
899 |
val Ts = map snd vars; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
900 |
val n = length vars; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
901 |
fun app_bounds 0 t = t$Bound 0 |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
902 |
| app_bounds n t = if n > 0 then app_bounds (n-1) (t$Bound n) else t |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
903 |
|
24867 | 904 |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
905 |
val [P,r] = Term.variant_frees t [("P",rT::Ts--->Term.propT),("r",Ts--->rT)]; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
906 |
val prop = Logic.mk_equals |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
907 |
(list_all ((f,fT)::vars, |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
908 |
app_bounds (n - 1) ((Free P)$(Bound n$app_bounds (n-1) (Free r)))), |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
909 |
list_all ((fst r,rT)::vars, |
24867 | 910 |
app_bounds (n - 1) ((Free P)$Bound n))); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
911 |
val prove_standard = quick_and_dirty_prove true thy; |
27217 | 912 |
val thm = prove_standard [] prop (fn _ => |
24867 | 913 |
EVERY [rtac equal_intr_rule 1, |
21687 | 914 |
Goal.norm_hhf_tac 1,REPEAT (etac meta_allE 1), atac 1, |
915 |
Goal.norm_hhf_tac 1,REPEAT (etac meta_allE 1), atac 1]); |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
916 |
in thm end |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
917 |
| mk_fun_apply_eq t thy = raise TERM ("mk_fun_apply_eq",[t]); |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
918 |
|
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
919 |
in |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
920 |
(* During proof of theorems produced by record_simproc you can end up in |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
921 |
* situations like "!!f ... . ... f r ..." where f is an extension update function. |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
922 |
* In order to split "f r" we transform this to "!!r ... . ... r ..." so that the |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
923 |
* usual split rules for extensions can apply. |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
924 |
*) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
925 |
val record_split_f_more_simproc = |
29064 | 926 |
Simplifier.simproc @{theory HOL} "record_split_f_more_simp" ["x"] |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
927 |
(fn thy => fn _ => fn t => |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
928 |
(case t of (Const ("all", Type (_, [Type (_, [Type("fun",[T,T']), _]), _])))$ |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
929 |
(trm as Abs _) => |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
930 |
(case rec_id (~1) T of |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
931 |
"" => NONE |
24867 | 932 |
| n => if T=T' |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
933 |
then (let |
24867 | 934 |
val P=cterm_of thy (abstract_over_fun_app trm); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
935 |
val thm = mk_fun_apply_eq trm thy; |
29265
5b4247055bd7
moved old add_term_vars, add_term_frees etc. to structure OldTerm;
wenzelm
parents:
29064
diff
changeset
|
936 |
val PV = cterm_of thy (hd (OldTerm.term_vars (prop_of thm))); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
937 |
val thm' = cterm_instantiate [(PV,P)] thm; |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
938 |
in SOME thm' end handle TERM _ => NONE) |
24867 | 939 |
else NONE) |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
940 |
| _ => NONE)) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
941 |
end |
14255 | 942 |
|
18858 | 943 |
fun prove_split_simp thy ss T prop = |
17261 | 944 |
let |
18858 | 945 |
val {sel_upd={simpset,...},extsplit,...} = RecordsData.get thy; |
17261 | 946 |
val extsplits = |
17412 | 947 |
Library.foldl (fn (thms,(n,_)) => the_list (Symtab.lookup extsplit n) @ thms) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
948 |
([],dest_recTs T); |
18858 | 949 |
val thms = (case get_splits thy (rec_id (~1) T) of |
17261 | 950 |
SOME (all_thm,_,_,_) => |
15203 | 951 |
all_thm::(case extsplits of [thm] => [] | _ => extsplits) |
952 |
(* [thm] is the same as all_thm *) |
|
17261 | 953 |
| NONE => extsplits) |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
954 |
val thms'=K_comp_convs@thms; |
24867 | 955 |
val ss' = (Simplifier.inherit_context ss simpset |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
956 |
addsimps thms' |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
957 |
addsimprocs [record_split_f_more_simproc]); |
16973 | 958 |
in |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
959 |
quick_and_dirty_prove true thy [] prop (fn _ => simp_tac ss' 1) |
15203 | 960 |
end; |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
961 |
|
15215 | 962 |
|
15059 | 963 |
local |
16822 | 964 |
fun eq (s1:string) (s2:string) = (s1 = s2); |
965 |
fun has_field extfields f T = |
|
18931 | 966 |
exists (fn (eN,_) => exists (eq f o fst) (Symtab.lookup_list extfields eN)) |
16822 | 967 |
(dest_recTs T); |
25705 | 968 |
|
969 |
fun K_skeleton n (T as Type (_,[_,kT])) (b as Bound i) (Abs (x,xT,t)) = |
|
970 |
if null (loose_bnos t) then ((n,kT),(Abs (x,xT,Bound (i+1)))) else ((n,T),b) |
|
971 |
| K_skeleton n T b _ = ((n,T),b); |
|
972 |
||
973 |
(* |
|
974 |
fun K_skeleton n _ b ((K_rec as Const ("Record.K_record",Type (_,[kT,_])))$_) = |
|
975 |
((n,kT),K_rec$b) |
|
976 |
| K_skeleton n _ (Bound i) |
|
977 |
(Abs (x,T,(K_rec as Const ("Record.K_record",Type (_,[kT,_])))$_$Bound 0)) = |
|
978 |
((n,kT),Abs (x,T,(K_rec$Bound (i+1)$Bound 0))) |
|
979 |
| K_skeleton n T b _ = ((n,T),b); |
|
980 |
*) |
|
981 |
||
982 |
fun normalize_rhs thm = |
|
983 |
let |
|
984 |
val ss = HOL_basic_ss addsimps K_comp_convs; |
|
985 |
val rhs = thm |> Thm.cprop_of |> Thm.dest_comb |> snd; |
|
986 |
val rhs' = (Simplifier.rewrite ss rhs); |
|
987 |
in Thm.transitive thm rhs' end; |
|
15059 | 988 |
in |
14255 | 989 |
(* record_simproc *) |
990 |
(* Simplifies selections of an record update: |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
991 |
* (1) S (S_update k r) = k (S r) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
992 |
* (2) S (X_update k r) = S r |
14255 | 993 |
* The simproc skips multiple updates at once, eg: |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
994 |
* S (X_update x (Y_update y (S_update k r))) = k (S r) |
14255 | 995 |
* But be careful in (2) because of the extendibility of records. |
996 |
* - If S is a more-selector we have to make sure that the update on component |
|
997 |
* X does not affect the selected subrecord. |
|
998 |
* - If X is a more-selector we have to make sure that S is not in the updated |
|
17261 | 999 |
* subrecord. |
14255 | 1000 |
*) |
13462 | 1001 |
val record_simproc = |
29064 | 1002 |
Simplifier.simproc @{theory HOL} "record_simp" ["x"] |
18858 | 1003 |
(fn thy => fn ss => fn t => |
16872 | 1004 |
(case t of (sel as Const (s, Type (_,[domS,rangeS])))$ |
1005 |
((upd as Const (u,Type(_,[_,Type (_,[rT,_])]))) $ k $ r)=> |
|
18858 | 1006 |
if is_selector thy s then |
1007 |
(case get_updates thy u of SOME u_name => |
|
13462 | 1008 |
let |
18858 | 1009 |
val {sel_upd={updates,...},extfields,...} = RecordsData.get thy; |
17261 | 1010 |
|
16872 | 1011 |
fun mk_eq_terms ((upd as Const (u,Type(_,[kT,_]))) $ k $ r) = |
17412 | 1012 |
(case Symtab.lookup updates u of |
15531 | 1013 |
NONE => NONE |
17261 | 1014 |
| SOME u_name |
14255 | 1015 |
=> if u_name = s |
24867 | 1016 |
then (case mk_eq_terms r of |
1017 |
NONE => |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1018 |
let |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1019 |
val rv = ("r",rT) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1020 |
val rb = Bound 0 |
25705 | 1021 |
val (kv,kb) = K_skeleton "k" kT (Bound 1) k; |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1022 |
in SOME (upd$kb$rb,kb$(sel$rb),[kv,rv]) end |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1023 |
| SOME (trm,trm',vars) => |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1024 |
let |
25705 | 1025 |
val (kv,kb) = K_skeleton "k" kT (Bound (length vars)) k; |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1026 |
in SOME (upd$kb$trm,kb$trm',kv::vars) end) |
16822 | 1027 |
else if has_field extfields u_name rangeS |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1028 |
orelse has_field extfields s (domain_type kT) |
15531 | 1029 |
then NONE |
17261 | 1030 |
else (case mk_eq_terms r of |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1031 |
SOME (trm,trm',vars) |
17261 | 1032 |
=> let |
25705 | 1033 |
val (kv,kb) = |
1034 |
K_skeleton "k" kT (Bound (length vars)) k; |
|
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1035 |
in SOME (upd$kb$trm,trm',kv::vars) end |
15531 | 1036 |
| NONE |
17261 | 1037 |
=> let |
1038 |
val rv = ("r",rT) |
|
14255 | 1039 |
val rb = Bound 0 |
25705 | 1040 |
val (kv,kb) = K_skeleton "k" kT (Bound 1) k; |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1041 |
in SOME (upd$kb$rb,sel$rb,[kv,rv]) end)) |
17261 | 1042 |
| mk_eq_terms r = NONE |
13462 | 1043 |
in |
17261 | 1044 |
(case mk_eq_terms (upd$k$r) of |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1045 |
SOME (trm,trm',vars) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1046 |
=> SOME (prove_split_simp thy ss domS |
27330 | 1047 |
(list_all(vars, Logic.mk_equals (sel $ trm, trm')))) |
15531 | 1048 |
| NONE => NONE) |
13462 | 1049 |
end |
15531 | 1050 |
| NONE => NONE) |
17510 | 1051 |
else NONE |
15531 | 1052 |
| _ => NONE)); |
7178 | 1053 |
|
17261 | 1054 |
(* record_upd_simproc *) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1055 |
(* simplify multiple updates: |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1056 |
* (1) "N_update y (M_update g (N_update x (M_update f r))) = |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1057 |
(N_update (y o x) (M_update (g o f) r))" |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1058 |
* (2) "r(|M:= M r|) = r" |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1059 |
* For (2) special care of "more" updates has to be taken: |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1060 |
* r(|more := m; A := A r|) |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1061 |
* If A is contained in the fields of m we cannot remove the update A := A r! |
17261 | 1062 |
* (But r(|more := r; A := A (r(|more := r|))|) = r(|more := r|) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1063 |
*) |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1064 |
val record_upd_simproc = |
29064 | 1065 |
Simplifier.simproc @{theory HOL} "record_upd_simp" ["x"] |
18858 | 1066 |
(fn thy => fn ss => fn t => |
16872 | 1067 |
(case t of ((upd as Const (u, Type(_,[_,Type(_,[rT,_])]))) $ k $ r) => |
17261 | 1068 |
let datatype ('a,'b) calc = Init of 'b | Inter of 'a |
18858 | 1069 |
val {sel_upd={selectors,updates,...},extfields,...} = RecordsData.get thy; |
17261 | 1070 |
|
1071 |
(*fun mk_abs_var x t = (x, fastype_of t);*) |
|
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30345
diff
changeset
|
1072 |
fun sel_name u = Long_Name.base_name (unsuffix updateN u); |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1073 |
|
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1074 |
fun seed s (upd as Const (more,Type(_,[mT,_]))$ k $ r) = |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1075 |
if has_field extfields s (domain_type' mT) then upd else seed s r |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1076 |
| seed _ r = r; |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1077 |
|
17261 | 1078 |
fun grow u uT k kT vars (sprout,skeleton) = |
1079 |
if sel_name u = moreN |
|
25705 | 1080 |
then let val (kv,kb) = K_skeleton "k" kT (Bound (length vars)) k; |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1081 |
in ((Const (u,uT)$k$sprout,Const (u,uT)$kb$skeleton),kv::vars) end |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1082 |
else ((sprout,skeleton),vars); |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1083 |
|
25705 | 1084 |
|
1085 |
fun dest_k (Abs (x,T,((sel as Const (s,_))$r))) = |
|
1086 |
if null (loose_bnos r) then SOME (x,T,sel,s,r) else NONE |
|
1087 |
| dest_k (Abs (_,_,(Abs (x,T,((sel as Const (s,_))$r)))$Bound 0)) = |
|
1088 |
(* eta expanded variant *) |
|
1089 |
if null (loose_bnos r) then SOME (x,T,sel,s,r) else NONE |
|
1090 |
| dest_k _ = NONE; |
|
1091 |
||
1092 |
fun is_upd_same (sprout,skeleton) u k = |
|
1093 |
(case dest_k k of SOME (x,T,sel,s,r) => |
|
17261 | 1094 |
if (unsuffix updateN u) = s andalso (seed s sprout) = r |
25705 | 1095 |
then SOME (fn t => Abs (x,T,incr_boundvars 1 t),sel,seed s skeleton) |
15531 | 1096 |
else NONE |
25705 | 1097 |
| NONE => NONE); |
17261 | 1098 |
|
16872 | 1099 |
fun init_seed r = ((r,Bound 0), [("r", rT)]); |
17261 | 1100 |
|
24867 | 1101 |
fun add (n:string) f fmaps = |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1102 |
(case AList.lookup (op =) fmaps n of |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1103 |
NONE => AList.update (op =) (n,[f]) fmaps |
24867 | 1104 |
| SOME fs => AList.update (op =) (n,f::fs) fmaps) |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1105 |
|
24867 | 1106 |
fun comps (n:string) T fmaps = |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1107 |
(case AList.lookup (op =) fmaps n of |
24867 | 1108 |
SOME fs => |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1109 |
foldr1 (fn (f,g) => Const ("Fun.comp",(T-->T)-->(T-->T)-->(T-->T))$f$g) fs |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1110 |
| NONE => error ("record_upd_simproc.comps")) |
24867 | 1111 |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1112 |
(* mk_updterm returns either |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1113 |
* - Init (orig-term, orig-term-skeleton, vars) if no optimisation can be made, |
17261 | 1114 |
* where vars are the bound variables in the skeleton |
1115 |
* - Inter (orig-term-skeleton,simplified-term-skeleton, |
|
16872 | 1116 |
* vars, (term-sprout, skeleton-sprout)) |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1117 |
* where "All vars. orig-term-skeleton = simplified-term-skeleton" is |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1118 |
* the desired simplification rule, |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1119 |
* the sprouts accumulate the "more-updates" on the way from the seed |
17261 | 1120 |
* to the outermost update. It is only relevant to calculate the |
1121 |
* possible simplification for (2) |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1122 |
* The algorithm first walks down the updates to the seed-record while |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1123 |
* memorising the updates in the already-table. While walking up the |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1124 |
* updates again, the optimised term is constructed. |
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1125 |
*) |
17261 | 1126 |
fun mk_updterm upds already |
16872 | 1127 |
(t as ((upd as Const (u,uT as (Type (_,[kT,_])))) $ k $ r)) = |
17261 | 1128 |
if Symtab.defined upds u |
1129 |
then let |
|
1130 |
fun rest already = mk_updterm upds already |
|
1131 |
in if u mem_string already |
|
1132 |
then (case (rest already r) of |
|
1133 |
Init ((sprout,skel),vars) => |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1134 |
let |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1135 |
val n = sel_name u; |
25705 | 1136 |
val (kv,kb) = K_skeleton n kT (Bound (length vars)) k; |
16872 | 1137 |
val (sprout',vars')= grow u uT k kT (kv::vars) (sprout,skel); |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1138 |
in Inter (upd$kb$skel,skel,vars',add n kb [],sprout') end |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1139 |
| Inter (trm,trm',vars,fmaps,sprout) => |
17261 | 1140 |
let |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1141 |
val n = sel_name u; |
25705 | 1142 |
val (kv,kb) = K_skeleton n kT (Bound (length vars)) k; |
16872 | 1143 |
val (sprout',vars') = grow u uT k kT (kv::vars) sprout; |
24867 | 1144 |
in Inter(upd$kb$trm,trm',kv::vars',add n kb fmaps,sprout') |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1145 |
end) |
17261 | 1146 |
else |
1147 |
(case rest (u::already) r of |
|
1148 |
Init ((sprout,skel),vars) => |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1149 |
(case is_upd_same (sprout,skel) u k of |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1150 |
SOME (K_rec,sel,skel') => |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1151 |
let |
17261 | 1152 |
val (sprout',vars') = grow u uT k kT vars (sprout,skel); |
25705 | 1153 |
in Inter(upd$(K_rec (sel$skel'))$skel,skel,vars',[],sprout') |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1154 |
end |
17261 | 1155 |
| NONE => |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1156 |
let |
25705 | 1157 |
val n = sel_name u; |
1158 |
val (kv,kb) = K_skeleton n kT (Bound (length vars)) k; |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1159 |
in Init ((upd$k$sprout,upd$kb$skel),kv::vars) end) |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1160 |
| Inter (trm,trm',vars,fmaps,sprout) => |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1161 |
(case is_upd_same sprout u k of |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1162 |
SOME (K_rec,sel,skel) => |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1163 |
let |
16872 | 1164 |
val (sprout',vars') = grow u uT k kT vars sprout |
25705 | 1165 |
in Inter(upd$(K_rec (sel$skel))$trm,trm',vars',fmaps,sprout') |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1166 |
end |
15531 | 1167 |
| NONE => |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1168 |
let |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1169 |
val n = sel_name u |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1170 |
val T = domain_type kT |
25705 | 1171 |
val (kv,kb) = K_skeleton n kT (Bound (length vars)) k; |
16872 | 1172 |
val (sprout',vars') = grow u uT k kT (kv::vars) sprout |
24867 | 1173 |
val fmaps' = add n kb fmaps |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1174 |
in Inter (upd$kb$trm,upd$comps n T fmaps'$trm' |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1175 |
,vars',fmaps',sprout') end)) |
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1176 |
end |
17261 | 1177 |
else Init (init_seed t) |
1178 |
| mk_updterm _ _ t = Init (init_seed t); |
|
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1179 |
|
17261 | 1180 |
in (case mk_updterm updates [] t of |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1181 |
Inter (trm,trm',vars,_,_) |
25705 | 1182 |
=> SOME (normalize_rhs |
1183 |
(prove_split_simp thy ss rT |
|
27330 | 1184 |
(list_all(vars, Logic.mk_equals (trm, trm'))))) |
15531 | 1185 |
| _ => NONE) |
24867 | 1186 |
end |
21226
a607ae87ee81
field-update in records is generalised to take a function on the field
schirmer
parents:
21109
diff
changeset
|
1187 |
| _ => NONE)) |
15059 | 1188 |
end |
15015
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
schirmer
parents:
15012
diff
changeset
|
1189 |
|
14255 | 1190 |
(* record_eq_simproc *) |
1191 |
(* looks up the most specific record-equality. |
|
1192 |
* Note on efficiency: |
|
1193 |
* Testing equality of records boils down to the test of equality of all components. |
|
1194 |
* Therefore the complexity is: #components * complexity for single component. |
|
1195 |
* Especially if a record has a lot of components it may be better to split up |
|
1196 |
* the record first and do simplification on that (record_split_simp_tac). |
|
1197 |
* e.g. r(|lots of updates|) = x |
|
1198 |
* |
|
14700
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
schirmer
parents:
14643
diff
changeset
|
1199 |
* record_eq_simproc record_split_simp_tac |
17261 | 1200 |
* Complexity: #components * #updates #updates |
1201 |
* |
|
14255 | 1202 |
*) |
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
1203 |
val record_eq_simproc = |
29064 | 1204 |
Simplifier.simproc @{theory HOL} "record_eq_simp" ["r = s"] |
18858 | 1205 |
(fn thy => fn _ => fn t => |
14079
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
berghofe
parents:
13904
diff
changeset
|
1206 |
(case t of Const ("op =", Type (_, [T, _])) $ _ $ _ => |