| author | haftmann | 
| Tue, 12 May 2009 19:30:33 +0200 | |
| changeset 31125 | 80218ee73167 | 
| parent 30715 | e23e15f52d42 | 
| child 31136 | 85d04515abb3 | 
| permissions | -rw-r--r-- | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1 | (* Title: HOL/Tools/record_package.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: 
21109diff
changeset | 7 | |
| 5698 | 8 | signature BASIC_RECORD_PACKAGE = | 
| 9 | sig | |
| 7178 | 10 | val record_simproc: simproc | 
| 14079 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
changeset | 11 | val record_eq_simproc: simproc | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 12 | val record_upd_simproc: simproc | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 13 | val record_split_simproc: (term -> int) -> simproc | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15258diff
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: 
14643diff
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 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 23 | signature RECORD_PACKAGE = | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 24 | sig | 
| 5698 | 25 | include BASIC_RECORD_PACKAGE | 
| 25179 | 26 | val timing: bool ref | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
14643diff
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: 
14643diff
changeset | 36 | val last_extT: typ -> (string * typ list) option | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
27239diff
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: 
27239diff
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: 
26423diff
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: 
26423diff
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: 
14643diff
changeset | 54 | |
| 17960 | 55 | structure RecordPackage: RECORD_PACKAGE = | 
| 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: 
14643diff
changeset | 59 | val rec_UNIV_I = thm "rec_UNIV_I"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
26957diff
changeset | 61 | val Pair_eq = thm "Product_Type.prod.inject"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 62 | val atomize_all = thm "HOL.atomize_all"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 70 | (** name components **) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 71 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 72 | val rN = "r"; | 
| 15215 | 73 | val wN = "w"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 74 | val moreN = "more"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 77 | val extN ="_ext"; | 
| 15215 | 78 | val casesN = "_cases"; | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
changeset | 79 | val ext_dest = "_sel"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 80 | val updateN = "_update"; | 
| 15215 | 81 | val updN = "_upd"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 82 | val makeN = "make"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 83 | val fields_selN = "fields"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 84 | val extendN = "extend"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 85 | val truncateN = "truncate"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 86 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 87 | (*see typedef_package.ML*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 88 | val RepN = "Rep_"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 89 | val AbsN = "Abs_"; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14702diff
changeset | 93 | fun but_last xs = fst (split_last xs); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
21109diff
changeset | 99 | fun domain_type' T = | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 100 | domain_type T handle Match => T; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 101 | |
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 102 | fun range_type' T = | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 103 | range_type T handle Match => T; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 104 | |
| 5698 | 105 | (* messages *) | 
| 106 | ||
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 107 | fun trace_thm str thm = | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 108 | tracing (str ^ (Pretty.string_of (Display.pretty_thm thm))); | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 109 | |
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 110 | fun trace_thms str thms = | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 111 | (tracing str; map (trace_thm "") thms); | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 112 | |
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 115 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 116 | (* timing *) | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 117 | |
| 25179 | 118 | val timing = ref false; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
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: 
30345diff
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: 
11923diff
changeset | 127 | val Trueprop = HOLogic.mk_Trueprop; | 
| 
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
 wenzelm parents: 
11923diff
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: 
11927diff
changeset | 130 | infix 9 $$; | 
| 
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
 wenzelm parents: 
11927diff
changeset | 131 | infix 0 :== ===; | 
| 
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
 wenzelm parents: 
11927diff
changeset | 132 | infixr 0 ==>; | 
| 
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
 wenzelm parents: 
11927diff
changeset | 133 | |
| 
6c1bf72430b6
derived operations are now: make, extend, truncate (cf. derived_defs);
 wenzelm parents: 
11927diff
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: 
11923diff
changeset | 136 | val (op ===) = Trueprop o HOLogic.mk_eq; | 
| 
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
 wenzelm parents: 
11923diff
changeset | 137 | val (op ==>) = Logic.mk_implies; | 
| 
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
 wenzelm parents: 
11923diff
changeset | 138 | |
| 11832 | 139 | (* morphisms *) | 
| 140 | ||
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 144 | fun mk_Rep name repT absT = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 147 | fun mk_Abs name repT absT = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 154 | fun mk_ext (name,T) ts = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 155 | let val Ts = map fastype_of ts | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 166 | (* selector *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 167 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 170 | fun mk_sel s (c,T) = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 171 | let val sT = fastype_of s | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 174 | (* updates *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 175 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 181 | |
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
14643diff
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: 
14643diff
changeset | 187 | (case try (unsuffix ext_typeN) c_ext_type of | 
| 15531 | 188 |         NONE => raise TYPE ("RecordPackage.dest_recT", [typ], [])
 | 
| 15570 | 189 | | SOME c => ((c, Ts), List.last Ts)) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 190 |   | dest_recT typ = raise TYPE ("RecordPackage.dest_recT", [typ], []);
 | 
| 5197 | 191 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 195 | fun dest_recTs T = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 196 | let val ((c, Ts), U) = dest_recT T | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 197 | in (c, Ts) :: dest_recTs U | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 198 | end handle TYPE _ => []; | 
| 14255 | 199 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 200 | fun last_extT T = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 201 | let val ((c, Ts), U) = dest_recT T | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15258diff
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: 
14643diff
changeset | 222 | extension: (string * typ list), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 223 | induct: thm | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 224 | }; | 
| 11927 
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
 wenzelm parents: 
11923diff
changeset | 225 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 228 | induct = induct}: record_info; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 234 | extension: (string * typ list), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 235 | induct: thm | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 236 | }; | 
| 11927 
96f267adc029
provodes induct/cases for use with corresponding Isar methods;
 wenzelm parents: 
11923diff
changeset | 237 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 238 | fun make_parent_info name fields extension induct = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15012diff
changeset | 251 | extinjects: thm list, | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
14643diff
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: 
14643diff
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: 
15012diff
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: 
14643diff
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: 
15012diff
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: 
15012diff
changeset | 279 | extsplit = extsplit1, | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 280 | splits = splits1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 281 | extfields = extfields1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15012diff
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: 
14643diff
changeset | 288 | splits = splits2, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 289 | extfields = extfields2, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 302 | (splits1, splits2)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 303 | (Symtab.merge (K true) (extfields1,extfields2)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
26626diff
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: 
15012diff
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: 
15012diff
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: 
13904diff
changeset | 358 | (* access 'equalities' *) | 
| 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
changeset | 359 | |
| 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
changeset | 360 | fun add_record_equalities name thm thy = | 
| 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
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: 
15012diff
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: 
15012diff
changeset | 366 | splits extfields fieldext; | 
| 14079 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
changeset | 367 | in RecordsData.put data thy end; | 
| 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
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: 
13904diff
changeset | 370 | |
| 22846 | 371 | |
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 372 | (* access 'extinjects' *) | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 373 | |
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 374 | fun add_extinjects thm thy = | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
15012diff
changeset | 381 | in RecordsData.put data thy end; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 382 | |
| 22634 | 383 | val get_extinjects = rev o #extinjects o RecordsData.get; | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 384 | |
| 22846 | 385 | |
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 386 | (* access 'extsplit' *) | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 387 | |
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 388 | fun add_extsplit name thm thy = | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
15012diff
changeset | 394 | extfields fieldext; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 395 | in RecordsData.put data thy end; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
15012diff
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: 
15012diff
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: 
15012diff
changeset | 413 | |
| 26088 | 414 | (* parent/extension of named record *) | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
13904diff
changeset | 419 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 420 | (* access 'extfields' *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 421 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 422 | fun add_extfields name fields thy = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15012diff
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: 
14643diff
changeset | 429 | in RecordsData.put data thy end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
30345diff
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: 
30345diff
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: 
14643diff
changeset | 457 | (* access 'fieldext' *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 458 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 459 | fun add_fieldext extname_types fields thy = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
15012diff
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: 
15012diff
changeset | 466 | splits extfields fieldext'; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 467 | in RecordsData.put data thy end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 468 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 501 | (** concrete syntax for records **) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 515 | (* parse translations *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 516 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 519 |       else raise TERM ("gen_field_tr: " ^ mark, [t])
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 521 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 524 | else [gen_field_tr mark sfx tm] | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 526 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 527 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 531 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 537 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 541 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 544 | else [dest_ext_field mark trm] | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14702diff
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: 
14643diff
changeset | 552 | fun splitargs (field::fields) ((name,arg)::fargs) = | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
changeset | 553 | if can (unsuffix name) field | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 554 | then let val (args,rest) = splitargs fields fargs | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 555 | in (arg::args,rest) end | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
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: 
14643diff
changeset | 557 | | splitargs [] (fargs as (_::_)) = ([],fargs) | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
changeset | 558 | | splitargs (_::_) [] = raise TERM (msg ^ "expecting more fields", [t]) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 559 | | splitargs _ _ = ([],[]); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 560 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 573 | | mk_ext [] = more | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 574 | |
| 17261 | 575 | in mk_ext fieldargs end; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14702diff
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: 
14643diff
changeset | 582 | fun splitargs (field::fields) ((name,arg)::fargs) = | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
changeset | 583 | if can (unsuffix name) field | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 584 | then let val (args,rest) = splitargs fields fargs | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 585 | in (arg::args,rest) end | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
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: 
14643diff
changeset | 587 | | splitargs [] (fargs as (_::_)) = ([],fargs) | 
| 14709 
d01983034ded
tuned HOL/record package; enabled record_upd_simproc by default.
 schirmer parents: 
14702diff
changeset | 588 | | splitargs (_::_) [] = raise TERM (msg ^ "expecting more fields", [t]) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 589 | | splitargs _ _ = ([],[]); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 590 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 596 | => (let | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14702diff
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: 
14643diff
changeset | 618 | | mk_ext [] = more | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 619 | |
| 17261 | 620 | in mk_ext fieldargs end; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 637 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 646 | |
| 15215 | 647 | |
| 24867 | 648 | val parse_translation = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 651 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 652 | |
| 24867 | 653 | val adv_parse_translation = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 654 |  [("_record",adv_record_tr),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 655 |   ("_record_scheme",adv_record_scheme_tr),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 658 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 659 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 660 | (* print translations *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 661 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 662 | val print_record_type_abbr = ref true; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 663 | val print_record_type_as_fields = ref true; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 680 | | gen_field_upds_tr' _ _ tm = ([], tm); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 681 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 682 | fun record_update_tr' tm = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
21109diff
changeset | 684 | if null ts then raise Match | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 685 | else Syntax.const "_record_update" $ u $ | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
14643diff
changeset | 687 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 688 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 689 | fun gen_field_tr' sfx tr' name = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 690 | let val name_sfx = suffix sfx name | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 696 | fun field_lst t = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 703 | => (let | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
30345diff
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: 
14643diff
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: 
14643diff
changeset | 711 |        | _ => [("",t)])
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 712 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
21109diff
changeset | 714 | val _ = if null flds then raise Match else (); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 717 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 718 | in if unit more | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 719 | then Syntax.const record$flds'' | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 720 | else Syntax.const record_scheme$flds''$more | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 721 | end | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 722 | |
| 17261 | 723 | fun gen_record_tr' name = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 727 | (list_comb (Syntax.const name_sfx,ts)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 728 | in (name_sfx,tr') | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 729 | end | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 730 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 731 | fun print_translation names = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 732 | map (gen_field_tr' updateN record_update_tr') names; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 733 | |
| 19748 | 734 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 742 | |
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
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: 
15258diff
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: 
15258diff
changeset | 750 | * fixT works around. | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
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: 
15258diff
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: 
15258diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 768 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 769 | in if !print_record_type_abbr | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 778 | then mk_type_abbr subst abbr alphas | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 784 | end | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 795 | fun field_lst T = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
21962diff
changeset | 797 | Type (ext, args) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
21962diff
changeset | 803 | SOME (_, alphas) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 804 | => (let | 
| 22219 
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
 haftmann parents: 
21962diff
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: 
30345diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
21962diff
changeset | 817 |                          | NONE => [("", T)])
 | 
| 
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
 haftmann parents: 
21962diff
changeset | 818 |                    | NONE => [("", T)])
 | 
| 
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
 haftmann parents: 
21962diff
changeset | 819 |              | NONE => [("", T)])
 | 
| 
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
 haftmann parents: 
21962diff
changeset | 820 |         | _ => [("", T)])
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 821 | |
| 22219 
61b5bab471ce
print translation for record types with empty-sorted type variables raise Match instead of producing an error
 haftmann parents: 
21962diff
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: 
21962diff
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: 
21962diff
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: 
14643diff
changeset | 825 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 830 | end | 
| 17261 | 831 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 832 | |
| 17261 | 833 | fun gen_record_type_tr' name = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
changeset | 837 | (list_comb (Syntax.const name_sfx,ts)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 838 | in (name_sfx,tr') | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 839 | end | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 840 | |
| 17261 | 841 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
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: 
14643diff
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: 
14643diff
changeset | 849 | in (name_sfx, tr') end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 850 | |
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 851 | (** record simprocs **) | 
| 14358 | 852 | |
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 853 | val record_quick_and_dirty_sensitive = ref false; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
15012diff
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: 
21109diff
changeset | 871 | local | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 873 | let | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 875 | val T = domain_type fT; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 883 | else subst u$subst w | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 885 | | subst t = t | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 896 | let | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 897 | val rT = domain_type fT; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 899 | val Ts = map snd vars; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 900 | val n = length vars; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 903 | |
| 24867 | 904 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 906 | val prop = Logic.mk_equals | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 907 | (list_all ((f,fT)::vars, | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 916 | in thm end | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 918 | |
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 919 | in | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 924 | *) | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 927 | (fn thy => fn _ => fn t => | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 929 | (trm as Abs _) => | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 930 | (case rec_id (~1) T of | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
29064diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 940 | | _ => NONE)) | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
15012diff
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: 
21109diff
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: 
21109diff
changeset | 956 | addsimps thms' | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
15012diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 1018 | let | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1019 |                                    val rv = ("r",rT)
 | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 1023 | | SOME (trm,trm',vars) => | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 1045 | SOME (trm,trm',vars) | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
15012diff
changeset | 1055 | (* simplify multiple updates: | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
changeset | 1057 | (N_update (y o x) (M_update (g o f) r))" | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1058 | * (2) "r(|M:= M r|) = r" | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1059 | * For (2) special care of "more" updates has to be taken: | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1060 | * r(|more := m; A := A r|) | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
changeset | 1063 | *) | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
30345diff
changeset | 1072 | fun sel_name u = Long_Name.base_name (unsuffix updateN u); | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1073 | |
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
21109diff
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: 
15012diff
changeset | 1076 | | seed _ r = r; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
15012diff
changeset | 1082 | else ((sprout,skeleton),vars); | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 1110 |                 | NONE => error ("record_upd_simproc.comps"))
 | 
| 24867 | 1111 | |
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1112 | (* mk_updterm returns either | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
changeset | 1117 | * where "All vars. orig-term-skeleton = simplified-term-skeleton" is | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1118 | * the desired simplification rule, | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
changeset | 1122 | * The algorithm first walks down the updates to the seed-record while | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1123 | * memorising the updates in the already-table. While walking up the | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1124 | * updates again, the optimised term is constructed. | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
changeset | 1134 | let | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
21109diff
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: 
15012diff
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: 
21109diff
changeset | 1150 | SOME (K_rec,sel,skel') => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
21109diff
changeset | 1154 | end | 
| 17261 | 1155 | | NONE => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
15012diff
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: 
21109diff
changeset | 1160 | | Inter (trm,trm',vars,fmaps,sprout) => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
21109diff
changeset | 1162 | SOME (K_rec,sel,skel) => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
21109diff
changeset | 1166 | end | 
| 15531 | 1167 | | NONE => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1168 | let | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1169 | val n = sel_name u | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
21109diff
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: 
21109diff
changeset | 1175 | ,vars',fmaps',sprout') end)) | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
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: 
15012diff
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: 
21109diff
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: 
21109diff
changeset | 1187 | | _ => NONE)) | 
| 15059 | 1188 | end | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
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: 
14643diff
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: 
13904diff
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: 
13904diff
changeset | 1206 |       (case t of Const ("op =", Type (_, [T, _])) $ _ $ _ =>
 | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1207 | (case rec_id (~1) T of | 
| 15531 | 1208 | "" => NONE | 
| 18858 | 1209 | | name => (case get_equalities thy name of | 
| 15531 | 1210 | NONE => NONE | 
| 1211 | | SOME thm => SOME (thm RS Eq_TrueI))) | |
| 1212 | | _ => NONE)); | |
| 14079 
1c22e5499eeb
- record_split_tac now also works for object-level universal quantifier
 berghofe parents: 
13904diff
changeset | 1213 | |
| 14255 | 1214 | (* record_split_simproc *) | 
| 17261 | 1215 | (* splits quantified occurrences of records, for which P holds. P can peek on the | 
| 14255 | 1216 | * subterm starting at the quantified occurrence of the record (including the quantifier) | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1217 | * P t = 0: do not split | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1218 | * P t = ~1: completely split | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1219 | * P t > 0: split up to given bound of record extensions | 
| 14255 | 1220 | *) | 
| 1221 | fun record_split_simproc P = | |
| 29064 | 1222 |   Simplifier.simproc @{theory HOL} "record_split_simp" ["x"]
 | 
| 18858 | 1223 | (fn thy => fn _ => fn t => | 
| 14255 | 1224 | (case t of (Const (quantifier, Type (_, [Type (_, [T, _]), _])))$trm => | 
| 1225 | if quantifier = "All" orelse quantifier = "all" orelse quantifier = "Ex" | |
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1226 | then (case rec_id (~1) T of | 
| 15531 | 1227 | "" => NONE | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1228 | | name | 
| 17261 | 1229 | => let val split = P t | 
| 1230 | in if split <> 0 then | |
| 18858 | 1231 | (case get_splits thy (rec_id split T) of | 
| 15531 | 1232 | NONE => NONE | 
| 17261 | 1233 | | SOME (all_thm, All_thm, Ex_thm,_) | 
| 15531 | 1234 | => SOME (case quantifier of | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1235 | "all" => all_thm | 
| 21546 | 1236 | | "All" => All_thm RS eq_reflection | 
| 1237 | | "Ex" => Ex_thm RS eq_reflection | |
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1238 | | _ => error "record_split_simproc")) | 
| 15531 | 1239 | else NONE | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1240 | end) | 
| 15531 | 1241 | else NONE | 
| 1242 | | _ => NONE)) | |
| 7178 | 1243 | |
| 14427 | 1244 | val record_ex_sel_eq_simproc = | 
| 29064 | 1245 |   Simplifier.simproc @{theory HOL} "record_ex_sel_eq_simproc" ["Ex t"]
 | 
| 18858 | 1246 | (fn thy => fn ss => fn t => | 
| 17261 | 1247 | let | 
| 16973 | 1248 | fun prove prop = | 
| 18858 | 1249 | quick_and_dirty_prove true thy [] prop | 
| 1250 | (fn _ => simp_tac (Simplifier.inherit_context ss (get_simpset thy) | |
| 16973 | 1251 | addsimps simp_thms addsimprocs [record_split_simproc (K ~1)]) 1); | 
| 14959 | 1252 | |
| 1253 | fun mkeq (lr,Teq,(sel,Tsel),x) i = | |
| 18858 | 1254 | if is_selector thy sel then | 
| 17261 | 1255 | let val x' = if not (loose_bvar1 (x,0)) | 
| 1256 |                               then Free ("x" ^ string_of_int i, range_type Tsel)
 | |
| 14959 | 1257 |                               else raise TERM ("",[x]);
 | 
| 1258 | val sel' = Const (sel,Tsel)$Bound 0; | |
| 1259 | val (l,r) = if lr then (sel',x') else (x',sel'); | |
| 1260 |                   in Const ("op =",Teq)$l$r end
 | |
| 17510 | 1261 |               else raise TERM ("",[Const (sel,Tsel)]);
 | 
| 14959 | 1262 | |
| 17261 | 1263 |          fun dest_sel_eq (Const ("op =",Teq)$(Const (sel,Tsel)$Bound 0)$X) =
 | 
| 14959 | 1264 | (true,Teq,(sel,Tsel),X) | 
| 1265 |            | dest_sel_eq (Const ("op =",Teq)$X$(Const (sel,Tsel)$Bound 0)) =
 | |
| 1266 | (false,Teq,(sel,Tsel),X) | |
| 1267 |            | dest_sel_eq _ = raise TERM ("",[]);
 | |
| 1268 | ||
| 17261 | 1269 | in | 
| 1270 | (case t of | |
| 14959 | 1271 |            (Const ("Ex",Tex)$Abs(s,T,t)) =>
 | 
| 16872 | 1272 | (let val eq = mkeq (dest_sel_eq t) 0; | 
| 14959 | 1273 |                  val prop = list_all ([("r",T)],
 | 
| 1274 |                               Logic.mk_equals (Const ("Ex",Tex)$Abs(s,T,eq),
 | |
| 1275 | HOLogic.true_const)); | |
| 15531 | 1276 | in SOME (prove prop) end | 
| 16872 | 1277 | handle TERM _ => NONE) | 
| 17261 | 1278 | | _ => NONE) | 
| 14427 | 1279 | end) | 
| 1280 | ||
| 5698 | 1281 | |
| 17261 | 1282 | |
| 6358 | 1283 | |
| 14255 | 1284 | local | 
| 1285 | val inductive_atomize = thms "induct_atomize"; | |
| 18464 | 1286 | val inductive_rulify = thms "induct_rulify"; | 
| 14255 | 1287 | in | 
| 1288 | (* record_split_simp_tac *) | |
| 17261 | 1289 | (* splits (and simplifies) all records in the goal for which P holds. | 
| 14255 | 1290 | * For quantified occurrences of a record | 
| 1291 | * P can peek on the whole subterm (including the quantifier); for free variables P | |
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1292 | * can only peek on the variable itself. | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1293 | * P t = 0: do not split | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1294 | * P t = ~1: completely split | 
| 17261 | 1295 | * P t > 0: split up to given bound of record extensions | 
| 14255 | 1296 | *) | 
| 15248 
b436486091a6
record_split_simp_tac now can get simp rules as parameter
 schirmer parents: 
15215diff
changeset | 1297 | fun record_split_simp_tac thms P i st = | 
| 14255 | 1298 | let | 
| 18858 | 1299 | val thy = Thm.theory_of_thm st; | 
| 14255 | 1300 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1301 | val has_rec = exists_Const | 
| 14255 | 1302 | (fn (s, Type (_, [Type (_, [T, _]), _])) => | 
| 17261 | 1303 | (s = "all" orelse s = "All" orelse s = "Ex") andalso is_recT T | 
| 14255 | 1304 | | _ => false); | 
| 1305 | ||
| 18011 
685d95c793ff
cleaned up nth, nth_update, nth_map and nth_string functions
 haftmann parents: 
17960diff
changeset | 1306 | val goal = nth (Thm.prems_of st) (i - 1); | 
| 29265 
5b4247055bd7
moved old add_term_vars, add_term_frees etc. to structure OldTerm;
 wenzelm parents: 
29064diff
changeset | 1307 | val frees = List.filter (is_recT o type_of) (OldTerm.term_frees goal); | 
| 14255 | 1308 | |
| 17261 | 1309 | fun mk_split_free_tac free induct_thm i = | 
| 18858 | 1310 | let val cfree = cterm_of thy free; | 
| 14255 | 1311 | val (_$(_$r)) = concl_of induct_thm; | 
| 18858 | 1312 | val crec = cterm_of thy r; | 
| 14255 | 1313 | val thm = cterm_instantiate [(crec,cfree)] induct_thm; | 
| 1314 | in EVERY [simp_tac (HOL_basic_ss addsimps inductive_atomize) i, | |
| 1315 | rtac thm i, | |
| 18464 | 1316 | simp_tac (HOL_basic_ss addsimps inductive_rulify) i] | 
| 17261 | 1317 | end; | 
| 14255 | 1318 | |
| 17261 | 1319 | fun split_free_tac P i (free as Free (n,T)) = | 
| 1320 | (case rec_id (~1) T of | |
| 15531 | 1321 | "" => NONE | 
| 17261 | 1322 | | name => let val split = P free | 
| 1323 | in if split <> 0 then | |
| 18858 | 1324 | (case get_splits thy (rec_id split T) of | 
| 15531 | 1325 | NONE => NONE | 
| 1326 | | SOME (_,_,_,induct_thm) | |
| 1327 | => SOME (mk_split_free_tac free induct_thm i)) | |
| 1328 | else NONE | |
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1329 | end) | 
| 15531 | 1330 | | split_free_tac _ _ _ = NONE; | 
| 14255 | 1331 | |
| 15570 | 1332 | val split_frees_tacs = List.mapPartial (split_free_tac P i) frees; | 
| 17261 | 1333 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1334 | val simprocs = if has_rec goal then [record_split_simproc P] else []; | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1335 | val thms' = K_comp_convs@thms | 
| 17261 | 1336 | in st |> ((EVERY split_frees_tacs) | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1337 | THEN (Simplifier.full_simp_tac (get_simpset thy addsimps thms' addsimprocs simprocs) i)) | 
| 15570 | 1338 | end handle Empty => Seq.empty; | 
| 14255 | 1339 | end; | 
| 1340 | ||
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1341 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1342 | (* record_split_tac *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1343 | (* splits all records in the goal, which are quantified by ! or !!. *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1344 | fun record_split_tac i st = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1345 | let | 
| 18858 | 1346 | val thy = Thm.theory_of_thm st; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1347 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1348 | val has_rec = exists_Const | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1349 | (fn (s, Type (_, [Type (_, [T, _]), _])) => | 
| 17261 | 1350 | (s = "all" orelse s = "All") andalso is_recT T | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1351 | | _ => false); | 
| 17261 | 1352 | |
| 18011 
685d95c793ff
cleaned up nth, nth_update, nth_map and nth_string functions
 haftmann parents: 
17960diff
changeset | 1353 | val goal = nth (Thm.prems_of st) (i - 1); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1354 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1355 | fun is_all t = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1356 | (case t of (Const (quantifier, _)$_) => | 
| 15273 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1357 | if quantifier = "All" orelse quantifier = "all" then ~1 else 0 | 
| 
771af451a062
* extended interface of record_split_simp_tac and record_split_simproc
 schirmer parents: 
15258diff
changeset | 1358 | | _ => 0); | 
| 17261 | 1359 | |
| 1360 | in if has_rec goal | |
| 1361 | then Simplifier.full_simp_tac | |
| 1362 | (HOL_basic_ss addsimprocs [record_split_simproc is_all]) i st | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1363 | else Seq.empty | 
| 15570 | 1364 | end handle Subscript => Seq.empty; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1365 | |
| 6358 | 1366 | (* wrapper *) | 
| 1367 | ||
| 5707 | 1368 | val record_split_name = "record_split_tac"; | 
| 1369 | val record_split_wrapper = (record_split_name, fn tac => record_split_tac ORELSE' tac); | |
| 5698 | 1370 | |
| 16330 | 1371 | |
| 1372 | ||
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1373 | (** theory extender interface **) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1374 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1375 | (* prepare arguments *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1376 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1377 | fun read_raw_parent ctxt raw_T = | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1378 | (case ProofContext.read_typ_abbrev ctxt raw_T of | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1379 | Type (name, Ts) => (Ts, name) | 
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1380 |   | T => error ("Bad parent record specification: " ^ Syntax.string_of_typ ctxt T));
 | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1381 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1382 | fun read_typ ctxt raw_T env = | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1383 | let | 
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1384 | val ctxt' = fold (Variable.declare_typ o TFree) env ctxt; | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1385 | val T = Syntax.read_typ ctxt' raw_T; | 
| 29270 
0eade173f77e
moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
 wenzelm parents: 
29265diff
changeset | 1386 | val env' = OldTerm.add_typ_tfrees (T, env); | 
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1387 | in (T, env') end; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1388 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1389 | fun cert_typ ctxt raw_T env = | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1390 | let | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1391 | val thy = ProofContext.theory_of ctxt; | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1392 | val T = Type.no_tvars (Sign.certify_typ thy raw_T) handle TYPE (msg, _, _) => error msg; | 
| 29270 
0eade173f77e
moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
 wenzelm parents: 
29265diff
changeset | 1393 | val env' = OldTerm.add_typ_tfrees (T, env); | 
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1394 | in (T, env') end; | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 1395 | |
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 1396 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1397 | (* attributes *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1398 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1399 | fun case_names_fields x = RuleCases.case_names ["fields"] x; | 
| 24830 
a7b3ab44d993
moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
 wenzelm parents: 
24712diff
changeset | 1400 | fun induct_type_global name = [case_names_fields, Induct.induct_type name]; | 
| 
a7b3ab44d993
moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
 wenzelm parents: 
24712diff
changeset | 1401 | fun cases_type_global name = [case_names_fields, Induct.cases_type name]; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1402 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1403 | (* tactics *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1404 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1405 | fun simp_all_tac ss simps = ALLGOALS (Simplifier.asm_full_simp_tac (ss addsimps simps)); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1406 | |
| 17261 | 1407 | (* do case analysis / induction according to rule on last parameter of ith subgoal | 
| 1408 | * (or on s if there are no parameters); | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1409 | * Instatiation of record variable (and predicate) in rule is calculated to | 
| 17261 | 1410 | * avoid problems with higher order unification. | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1411 | *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1412 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1413 | fun try_param_tac s rule i st = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1414 | let | 
| 17510 | 1415 | val cert = cterm_of (Thm.theory_of_thm st); | 
| 18011 
685d95c793ff
cleaned up nth, nth_update, nth_map and nth_string functions
 haftmann parents: 
17960diff
changeset | 1416 | val g = nth (prems_of st) (i - 1); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1417 | val params = Logic.strip_params g; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1418 | val concl = HOLogic.dest_Trueprop (Logic.strip_assums_concl g); | 
| 18145 | 1419 | val rule' = Thm.lift_rule (Thm.cprem_of st i) rule; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1420 | val (P, ys) = strip_comb (HOLogic.dest_Trueprop | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1421 | (Logic.strip_assums_concl (prop_of rule'))); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1422 | (* ca indicates if rule is a case analysis or induction rule *) | 
| 15570 | 1423 | val (x, ca) = (case rev (Library.drop (length params, ys)) of | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1424 | [] => (head_of (fst (HOLogic.dest_eq (HOLogic.dest_Trueprop | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1425 | (hd (rev (Logic.strip_assums_hyp (hd (prems_of rule')))))))), true) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1426 | | [x] => (head_of x, false)); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1427 | val rule'' = cterm_instantiate (map (pairself cert) (case (rev params) of | 
| 29265 
5b4247055bd7
moved old add_term_vars, add_term_frees etc. to structure OldTerm;
 wenzelm parents: 
29064diff
changeset | 1428 | [] => (case AList.lookup (op =) (map dest_Free (OldTerm.term_frees (prop_of st))) s of | 
| 15531 | 1429 | NONE => sys_error "try_param_tac: no such variable" | 
| 1430 | | SOME T => [(P, if ca then concl else lambda (Free (s, T)) concl), | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1431 | (x, Free (s, T))]) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1432 | | (_, T) :: _ => [(P, list_abs (params, if ca then concl | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1433 | else incr_boundvars 1 (Abs (s, T, concl)))), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1434 | (x, list_abs (params, Bound 0))])) rule' | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1435 | in compose_tac (false, rule'', nprems_of rule) i st end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1436 | |
| 15215 | 1437 | |
| 1438 | (* !!x1 ... xn. ... ==> EX x1 ... xn. P x1 ... xn; | |
| 1439 | instantiates x1 ... xn with parameters x1 ... xn *) | |
| 1440 | fun ex_inst_tac i st = | |
| 1441 | let | |
| 18858 | 1442 | val thy = Thm.theory_of_thm st; | 
| 18011 
685d95c793ff
cleaned up nth, nth_update, nth_map and nth_string functions
 haftmann parents: 
17960diff
changeset | 1443 | val g = nth (prems_of st) (i - 1); | 
| 15215 | 1444 | val params = Logic.strip_params g; | 
| 18145 | 1445 | val exI' = Thm.lift_rule (Thm.cprem_of st i) exI; | 
| 15215 | 1446 | val (_$(_$x)) = Logic.strip_assums_concl (hd (prems_of exI')); | 
| 18858 | 1447 | val cx = cterm_of thy (fst (strip_comb x)); | 
| 15215 | 1448 | |
| 17261 | 1449 | in Seq.single (Library.foldl (fn (st,v) => | 
| 1450 | Seq.hd | |
| 1451 | (compose_tac (false, cterm_instantiate | |
| 18858 | 1452 | [(cx,cterm_of thy (list_abs (params,Bound v)))] exI',1) | 
| 15215 | 1453 | i st)) (st,((length params) - 1) downto 0)) | 
| 1454 | end; | |
| 1455 | ||
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1456 | fun extension_typedef name repT alphas thy = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1457 | let | 
| 20484 | 1458 | fun get_thms thy name = | 
| 1459 | let | |
| 1460 |         val SOME { Abs_induct = abs_induct,
 | |
| 1461 | Abs_inject=abs_inject, Abs_inverse = abs_inverse, ...} = TypedefPackage.get_info thy name; | |
| 21708 | 1462 | val rewrite_rule = MetaSimplifier.rewrite_rule [rec_UNIV_I, rec_True_simp]; | 
| 20484 | 1463 | in map rewrite_rule [abs_inject, abs_inverse, abs_induct] end; | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 1464 | val tname = Binding.name (Long_Name.base_name name); | 
| 20484 | 1465 | in | 
| 1466 | thy | |
| 30345 | 1467 | |> TypecopyPackage.add_typecopy (Binding.suffix_name ext_typeN tname, alphas) repT NONE | 
| 20484 | 1468 | |-> (fn (name, _) => `(fn thy => get_thms thy name)) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1469 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1470 | |
| 17261 | 1471 | fun mixit convs refls = | 
| 15215 | 1472 | let fun f ((res,lhs,rhs),refl) = ((refl,List.revAppend (lhs,refl::tl rhs))::res,hd rhs::lhs,tl rhs); | 
| 15570 | 1473 | in #1 (Library.foldl f (([],[],convs),refls)) end; | 
| 15215 | 1474 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1475 | |
| 17261 | 1476 | fun extension_definition full name fields names alphas zeta moreT more vars thy = | 
| 1477 | let | |
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 1478 | val base = Long_Name.base_name; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1479 | val fieldTs = (map snd fields); | 
| 15215 | 1480 | val alphas_zeta = alphas@[zeta]; | 
| 1481 | val alphas_zetaTs = map (fn n => TFree (n, HOLogic.typeS)) alphas_zeta; | |
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1482 | val vT = TFree (Name.variant alphas_zeta "'v", HOLogic.typeS); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1483 | val extT_name = suffix ext_typeN name | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1484 | val extT = Type (extT_name, alphas_zetaTs); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1485 | val repT = foldr1 HOLogic.mk_prodT (fieldTs@[moreT]); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1486 | val fields_more = fields@[(full moreN,moreT)]; | 
| 15215 | 1487 | val fields_moreTs = fieldTs@[moreT]; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1488 | val bfields_more = map (apfst base) fields_more; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1489 | val r = Free (rN,extT) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1490 | val len = length fields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1491 | val idxms = 0 upto len; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1492 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1493 | (* prepare declarations and definitions *) | 
| 17261 | 1494 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1495 | (*fields constructor*) | 
| 15215 | 1496 | val ext_decl = (mk_extC (name,extT) fields_moreTs); | 
| 17261 | 1497 | (* | 
| 1498 | val ext_spec = Const ext_decl :== | |
| 1499 | (foldr (uncurry lambda) | |
| 1500 | (mk_Abs name repT extT $ (foldr1 HOLogic.mk_prod (vars@[more]))) (vars@[more])) | |
| 1501 | *) | |
| 1502 | val ext_spec = list_comb (Const ext_decl,vars@[more]) :== | |
| 15215 | 1503 | (mk_Abs name repT extT $ (foldr1 HOLogic.mk_prod (vars@[more]))); | 
| 1504 | ||
| 17261 | 1505 | fun mk_ext args = list_comb (Const ext_decl, args); | 
| 1506 | ||
| 1507 | (*destructors*) | |
| 16379 | 1508 | val _ = timing_msg "record extension preparing definitions"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1509 | val dest_decls = map (mk_selC extT o (apfst (suffix ext_dest))) bfields_more; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1510 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1511 | fun mk_dest_spec (i, (c,T)) = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1512 | let val snds = (funpow i HOLogic.mk_snd (mk_Rep name repT extT $ r)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1513 | in Const (mk_selC extT (suffix ext_dest c,T)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1514 | :== (lambda r (if i=len then snds else HOLogic.mk_fst snds)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1515 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1516 | val dest_specs = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1517 | ListPair.map mk_dest_spec (idxms, fields_more); | 
| 17261 | 1518 | |
| 16379 | 1519 | (*updates*) | 
| 15215 | 1520 | val upd_decls = map (mk_updC updN extT) bfields_more; | 
| 1521 | fun mk_upd_spec (c,T) = | |
| 1522 | let | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1523 | val args = map (fn (n,nT) => if n=c then Free (base c,T --> T)$ | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1524 | (mk_sel r (suffix ext_dest n,nT)) | 
| 17261 | 1525 | else (mk_sel r (suffix ext_dest n,nT))) | 
| 15215 | 1526 | fields_more; | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1527 | in Const (mk_updC updN extT (c,T))$(Free (base c,T --> T))$r | 
| 15215 | 1528 | :== mk_ext args | 
| 1529 | end; | |
| 1530 | val upd_specs = map mk_upd_spec fields_more; | |
| 17261 | 1531 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1532 | (* 1st stage: defs_thy *) | 
| 16379 | 1533 | fun mk_defs () = | 
| 17261 | 1534 | thy | 
| 30345 | 1535 | |> extension_typedef name repT (alphas @ [zeta]) | 
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1536 | ||> Sign.add_consts_i | 
| 30345 | 1537 | (map (Syntax.no_syn o apfst Binding.name) (apfst base ext_decl :: dest_decls @ upd_decls)) | 
| 29579 | 1538 | ||>> PureThy.add_defs false | 
| 1539 | (map (Thm.no_attributes o apfst Binding.name) (ext_spec :: dest_specs)) | |
| 1540 | ||>> PureThy.add_defs false | |
| 1541 | (map (Thm.no_attributes o apfst Binding.name) upd_specs) | |
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1542 | |-> (fn args as ((_, dest_defs), upd_defs) => | 
| 28370 | 1543 | fold Code.add_default_eqn dest_defs | 
| 1544 | #> fold Code.add_default_eqn upd_defs | |
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1545 | #> pair args); | 
| 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1546 | val ((([abs_inject, abs_inverse, abs_induct], ext_def :: dest_defs), upd_defs), defs_thy) = | 
| 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1547 | timeit_msg "record extension type/selector/update defs:" mk_defs; | 
| 17261 | 1548 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1549 | (* prepare propositions *) | 
| 16379 | 1550 | val _ = timing_msg "record extension preparing propositions"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1551 | val vars_more = vars@[more]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1552 | val named_vars_more = (names@[full moreN])~~vars_more; | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1553 | val variants = map (fn (Free (x,_))=>x) vars_more; | 
| 15215 | 1554 | val ext = mk_ext vars_more; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1555 | val s = Free (rN, extT); | 
| 15215 | 1556 | val w = Free (wN, extT); | 
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1557 | val P = Free (Name.variant variants "P", extT-->HOLogic.boolT); | 
| 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1558 | val C = Free (Name.variant variants "C", HOLogic.boolT); | 
| 17261 | 1559 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1560 | val inject_prop = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1561 | let val vars_more' = map (fn (Free (x,T)) => Free (x ^ "'",T)) vars_more; | 
| 17261 | 1562 | in All (map dest_Free (vars_more@vars_more')) | 
| 1563 | ((HOLogic.eq_const extT $ | |
| 1564 | mk_ext vars_more$mk_ext vars_more') | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1565 | === | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1566 | foldr1 HOLogic.mk_conj (map HOLogic.mk_eq (vars_more ~~ vars_more'))) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1567 | end; | 
| 17261 | 1568 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1569 | val induct_prop = | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1570 | (All (map dest_Free vars_more) (Trueprop (P $ ext)), Trueprop (P $ s)); | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1571 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1572 | val cases_prop = | 
| 17261 | 1573 | (All (map dest_Free vars_more) | 
| 1574 | (Trueprop (HOLogic.mk_eq (s,ext)) ==> Trueprop C)) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1575 | ==> Trueprop C; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1576 | |
| 17261 | 1577 | (*destructors*) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1578 | val dest_conv_props = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1579 | map (fn (c, x as Free (_,T)) => mk_sel ext (suffix ext_dest c,T) === x) named_vars_more; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1580 | |
| 15215 | 1581 | (*updates*) | 
| 1582 | fun mk_upd_prop (i,(c,T)) = | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1583 | let val x' = Free (Name.variant variants (base c ^ "'"),T --> T) | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1584 | val args' = nth_map i (K (x'$nth vars_more i)) vars_more | 
| 15215 | 1585 | in mk_upd updN c x' ext === mk_ext args' end; | 
| 1586 | val upd_conv_props = ListPair.map mk_upd_prop (idxms, fields_more); | |
| 1587 | ||
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1588 | val surjective_prop = | 
| 17261 | 1589 | let val args = | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1590 | map (fn (c, Free (_,T)) => mk_sel s (suffix ext_dest c,T)) named_vars_more; | 
| 15215 | 1591 | in s === mk_ext args end; | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1592 | |
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1593 | val split_meta_prop = | 
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1594 | let val P = Free (Name.variant variants "P", extT-->Term.propT) in | 
| 17261 | 1595 | Logic.mk_equals | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1596 | (All [dest_Free s] (P $ s), All (map dest_Free vars_more) (P $ ext)) | 
| 17261 | 1597 | end; | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1598 | |
| 17510 | 1599 | fun prove stndrd = quick_and_dirty_prove stndrd defs_thy; | 
| 1600 | val prove_standard = quick_and_dirty_prove true defs_thy; | |
| 15215 | 1601 | fun prove_simp stndrd simps = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1602 | let val tac = simp_all_tac HOL_ss simps | 
| 15215 | 1603 | in fn prop => prove stndrd [] prop (K tac) end; | 
| 17261 | 1604 | |
| 15215 | 1605 | fun inject_prf () = (prove_simp true [ext_def,abs_inject,Pair_eq] inject_prop); | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1606 | val inject = timeit_msg "record extension inject proof:" inject_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1607 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1608 | fun induct_prf () = | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1609 | let val (assm, concl) = induct_prop | 
| 20248 | 1610 |       in prove_standard [assm] concl (fn {prems, ...} =>
 | 
| 17261 | 1611 | EVERY [try_param_tac rN abs_induct 1, | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1612 | simp_tac (HOL_ss addsimps [split_paired_all]) 1, | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1613 | resolve_tac (map (rewrite_rule [ext_def]) prems) 1]) | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1614 | end; | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1615 | val induct = timeit_msg "record extension induct proof:" induct_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1616 | |
| 15215 | 1617 | fun cases_prf_opt () = | 
| 17261 | 1618 | let | 
| 15215 | 1619 | val (_$(Pvar$_)) = concl_of induct; | 
| 17261 | 1620 | val ind = cterm_instantiate | 
| 18858 | 1621 | [(cterm_of defs_thy Pvar, cterm_of defs_thy | 
| 15215 | 1622 | (lambda w (HOLogic.imp$HOLogic.mk_eq(r,w)$C)))] | 
| 1623 | induct; | |
| 1624 | in standard (ObjectLogic.rulify (mp OF [ind, refl])) end; | |
| 1625 | ||
| 1626 | fun cases_prf_noopt () = | |
| 27217 | 1627 | prove_standard [] cases_prop (fn _ => | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1628 | EVERY [asm_full_simp_tac (HOL_basic_ss addsimps [atomize_all, atomize_imp]) 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1629 | try_param_tac rN induct 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1630 | rtac impI 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1631 | REPEAT (etac allE 1), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1632 | etac mp 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1633 | rtac refl 1]) | 
| 15215 | 1634 | |
| 1635 | val cases_prf = quick_and_dirty_prf cases_prf_noopt cases_prf_opt; | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1636 | val cases = timeit_msg "record extension cases proof:" cases_prf; | 
| 17261 | 1637 | |
| 1638 | fun dest_convs_prf () = map (prove_simp false | |
| 15215 | 1639 | ([ext_def,abs_inverse]@Pair_sel_convs@dest_defs)) dest_conv_props; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1640 | val dest_convs = timeit_msg "record extension dest_convs proof:" dest_convs_prf; | 
| 15215 | 1641 | fun dest_convs_standard_prf () = map standard dest_convs; | 
| 1642 | ||
| 17261 | 1643 | val dest_convs_standard = | 
| 1644 | timeit_msg "record extension dest_convs_standard proof:" dest_convs_standard_prf; | |
| 1645 | ||
| 1646 | fun upd_convs_prf_noopt () = map (prove_simp true (dest_convs_standard@upd_defs)) | |
| 15215 | 1647 | upd_conv_props; | 
| 1648 | fun upd_convs_prf_opt () = | |
| 17261 | 1649 | let | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1650 | |
| 17261 | 1651 | fun mkrefl (c,T) = Thm.reflexive | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1652 | (cterm_of defs_thy (Free (Name.variant variants (base c ^ "'"),T-->T))); | 
| 15215 | 1653 | val refls = map mkrefl fields_more; | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1654 | val dest_convs' = map mk_meta_eq dest_convs; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1655 | val map_eqs = map (uncurry Thm.combination) (refls ~~ dest_convs'); | 
| 24867 | 1656 | |
| 18858 | 1657 | val constr_refl = Thm.reflexive (cterm_of defs_thy (head_of ext)); | 
| 17261 | 1658 | |
| 15215 | 1659 | fun mkthm (udef,(fld_refl,thms)) = | 
| 15570 | 1660 | let val bdyeq = Library.foldl (uncurry Thm.combination) (constr_refl,thms); | 
| 15215 | 1661 | (* (|N=N (|N=N,M=M,K=K,more=more|) | 
| 1662 | M=M (|N=N,M=M,K=K,more=more|) | |
| 1663 | K=K' | |
| 1664 | more = more (|N=N,M=M,K=K,more=more|) = | |
| 1665 | (|N=N,M=M,K=K',more=more|) | |
| 1666 | *) | |
| 1667 | val (_$(_$v$r)$_) = prop_of udef; | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1668 | val (_$(v'$_)$_) = prop_of fld_refl; | 
| 17261 | 1669 | val udef' = cterm_instantiate | 
| 18858 | 1670 | [(cterm_of defs_thy v,cterm_of defs_thy v'), | 
| 1671 | (cterm_of defs_thy r,cterm_of defs_thy ext)] udef; | |
| 17261 | 1672 | in standard (Thm.transitive udef' bdyeq) end; | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1673 | in map mkthm (rev upd_defs ~~ (mixit dest_convs' map_eqs)) end; | 
| 17261 | 1674 | |
| 15215 | 1675 | val upd_convs_prf = quick_and_dirty_prf upd_convs_prf_noopt upd_convs_prf_opt; | 
| 1676 | ||
| 17261 | 1677 | val upd_convs = | 
| 1678 | timeit_msg "record extension upd_convs proof:" upd_convs_prf; | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 1679 | |
| 17261 | 1680 | fun surjective_prf () = | 
| 27217 | 1681 | prove_standard [] surjective_prop (fn _ => | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1682 | (EVERY [try_param_tac rN induct 1, | 
| 15215 | 1683 | simp_tac (HOL_basic_ss addsimps dest_convs_standard) 1])); | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1684 | val surjective = timeit_msg "record extension surjective proof:" surjective_prf; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1685 | |
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1686 | fun split_meta_prf () = | 
| 27217 | 1687 | prove_standard [] split_meta_prop (fn _ => | 
| 21687 | 1688 | EVERY [rtac equal_intr_rule 1, Goal.norm_hhf_tac 1, | 
| 17960 | 1689 | etac meta_allE 1, atac 1, | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1690 | rtac (prop_subst OF [surjective]) 1, | 
| 17960 | 1691 | REPEAT (etac meta_allE 1), atac 1]); | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1692 | val split_meta = timeit_msg "record extension split_meta proof:" split_meta_prf; | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1693 | |
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1694 | |
| 24867 | 1695 | val (([inject',induct',cases',surjective',split_meta'], | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1696 | [dest_convs',upd_convs']), | 
| 18377 | 1697 | thm_thy) = | 
| 17261 | 1698 | defs_thy | 
| 29579 | 1699 | |> (PureThy.add_thms o map (Thm.no_attributes o apfst Binding.name)) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1700 |            [("ext_inject", inject),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1701 |             ("ext_induct", induct),
 | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1702 |             ("ext_cases", cases),
 | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1703 |             ("ext_surjective", surjective),
 | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 1704 |             ("ext_split", split_meta)]
 | 
| 29579 | 1705 | ||>> (PureThy.add_thmss o map (Thm.no_attributes o apfst Binding.name)) | 
| 1706 |             [("dest_convs", dest_convs_standard), ("upd_convs", upd_convs)]
 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1707 | |
| 15215 | 1708 | in (thm_thy,extT,induct',inject',dest_convs',split_meta',upd_convs') | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1709 | end; | 
| 17261 | 1710 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1711 | fun chunks [] [] = [] | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1712 | | chunks [] xs = [xs] | 
| 15570 | 1713 | | chunks (l::ls) xs = Library.take (l,xs)::chunks ls (Library.drop (l,xs)); | 
| 17261 | 1714 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1715 | fun chop_last [] = error "last: list should not be empty" | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1716 | | chop_last [x] = ([],x) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1717 | | chop_last (x::xs) = let val (tl,l) = chop_last xs in (x::tl,l) end; | 
| 17261 | 1718 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1719 | fun subst_last s [] = error "subst_last: list should not be empty" | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1720 | | subst_last s ([x]) = [s] | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1721 | | subst_last s (x::xs) = (x::subst_last s xs); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1722 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1723 | (* mk_recordT builds up the record type from the current extension tpye extT and a list | 
| 17261 | 1724 | * of parent extensions, starting with the root of the record hierarchy | 
| 1725 | *) | |
| 21078 | 1726 | fun mk_recordT extT = | 
| 1727 | fold_rev (fn (parent, Ts) => fn T => Type (parent, subst_last T Ts)) extT; | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1728 | |
| 15215 | 1729 | |
| 1730 | ||
| 1731 | fun obj_to_meta_all thm = | |
| 1732 | let | |
| 17261 | 1733 | fun E thm = case (SOME (spec OF [thm]) handle THM _ => NONE) of | 
| 15531 | 1734 | SOME thm' => E thm' | 
| 1735 | | NONE => thm; | |
| 15215 | 1736 | val th1 = E thm; | 
| 1737 | val th2 = Drule.forall_intr_vars th1; | |
| 1738 | in th2 end; | |
| 1739 | ||
| 1740 | fun meta_to_obj_all thm = | |
| 1741 | let | |
| 26626 
c6231d64d264
rep_cterm/rep_thm: no longer dereference theory_ref;
 wenzelm parents: 
26496diff
changeset | 1742 | val thy = Thm.theory_of_thm thm; | 
| 
c6231d64d264
rep_cterm/rep_thm: no longer dereference theory_ref;
 wenzelm parents: 
26496diff
changeset | 1743 | val prop = Thm.prop_of thm; | 
| 15215 | 1744 | val params = Logic.strip_params prop; | 
| 1745 | val concl = HOLogic.dest_Trueprop (Logic.strip_assums_concl prop); | |
| 22596 | 1746 | val ct = cterm_of thy | 
| 15215 | 1747 | (HOLogic.mk_Trueprop (HOLogic.list_all (params, concl))); | 
| 1748 | val thm' = Seq.hd (REPEAT (rtac allI 1) (Thm.trivial ct)); | |
| 1749 | in | |
| 1750 | Thm.implies_elim thm' thm | |
| 1751 | end; | |
| 1752 | ||
| 1753 | ||
| 1754 | ||
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1755 | (* record_definition *) | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1756 | |
| 17261 | 1757 | fun record_definition (args, bname) parent (parents: parent_info list) raw_fields thy = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1758 | let | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1759 | val external_names = NameSpace.external_names (Sign.naming_of thy); | 
| 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1760 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1761 | val alphas = map fst args; | 
| 28965 | 1762 | val name = Sign.full_bname thy bname; | 
| 1763 | val full = Sign.full_bname_path thy bname; | |
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 1764 | val base = Long_Name.base_name; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1765 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1766 | val (bfields, field_syntax) = split_list (map (fn (x, T, mx) => ((x, T), mx)) raw_fields); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1767 | |
| 15570 | 1768 | val parent_fields = List.concat (map #fields parents); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1769 | val parent_chunks = map (length o #fields) parents; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1770 | val parent_names = map fst parent_fields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1771 | val parent_types = map snd parent_fields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1772 | val parent_fields_len = length parent_fields; | 
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1773 | val parent_variants = Name.variant_list [moreN, rN, rN ^ "'", wN] (map base parent_names); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1774 | val parent_vars = ListPair.map Free (parent_variants, parent_types); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1775 | val parent_len = length parents; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1776 | val parents_idx = (map #name parents) ~~ (0 upto (parent_len - 1)); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1777 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1778 | val fields = map (apfst full) bfields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1779 | val names = map fst fields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1780 | val extN = full bname; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1781 | val types = map snd fields; | 
| 30190 | 1782 | val alphas_fields = List.foldr OldTerm.add_typ_tfree_names [] types; | 
| 17261 | 1783 | val alphas_ext = alphas inter alphas_fields; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1784 | val len = length fields; | 
| 30715 
e23e15f52d42
avoid mixing of left/right associative infixes, to make it work with experimental Poly/ML 5.3 branch;
 wenzelm parents: 
30364diff
changeset | 1785 | val variants = | 
| 
e23e15f52d42
avoid mixing of left/right associative infixes, to make it work with experimental Poly/ML 5.3 branch;
 wenzelm parents: 
30364diff
changeset | 1786 | Name.variant_list (moreN :: rN :: (rN ^ "'") :: wN :: parent_variants) (map fst bfields); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1787 | val vars = ListPair.map Free (variants, types); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1788 | val named_vars = names ~~ vars; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1789 | val idxs = 0 upto (len - 1); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1790 | val idxms = 0 upto len; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1791 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1792 | val all_fields = parent_fields @ fields; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1793 | val all_names = parent_names @ names; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1794 | val all_types = parent_types @ types; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1795 | val all_len = parent_fields_len + len; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1796 | val all_variants = parent_variants @ variants; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1797 | val all_vars = parent_vars @ vars; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1798 | val all_named_vars = (parent_names ~~ parent_vars) @ named_vars; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1799 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1800 | |
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1801 | val zeta = Name.variant alphas "'z"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1802 | val moreT = TFree (zeta, HOLogic.typeS); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1803 | val more = Free (moreN, moreT); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1804 | val full_moreN = full moreN; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1805 | val bfields_more = bfields @ [(moreN,moreT)]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1806 | val fields_more = fields @ [(full_moreN,moreT)]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1807 | val vars_more = vars @ [more]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1808 | val named_vars_more = named_vars @[(full_moreN,more)]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1809 | val all_vars_more = all_vars @ [more]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1810 | val all_named_vars_more = all_named_vars @ [(full_moreN,more)]; | 
| 17261 | 1811 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1812 | (* 1st stage: extension_thy *) | 
| 15215 | 1813 | val (extension_thy,extT,ext_induct,ext_inject,ext_dest_convs,ext_split,u_convs) = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1814 | thy | 
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1815 | |> Sign.add_path bname | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1816 | |> extension_definition full extN fields names alphas_ext zeta moreT more vars; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1817 | |
| 17261 | 1818 | val _ = timing_msg "record preparing definitions"; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1819 | val Type extension_scheme = extT; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1820 | val extension_name = unsuffix ext_typeN (fst extension_scheme); | 
| 17261 | 1821 | val extension = let val (n,Ts) = extension_scheme in (n,subst_last HOLogic.unitT Ts) end; | 
| 1822 | val extension_names = | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1823 | (map ((unsuffix ext_typeN) o fst o #extension) parents) @ [extN]; | 
| 15570 | 1824 |     val extension_id = Library.foldl (op ^) ("",extension_names);
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1825 | |
| 17261 | 1826 | |
| 21078 | 1827 | fun rec_schemeT n = mk_recordT (map #extension (prune n parents)) extT; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1828 | val rec_schemeT0 = rec_schemeT 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1829 | |
| 17261 | 1830 | fun recT n = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1831 | let val (c,Ts) = extension | 
| 21078 | 1832 | in mk_recordT (map #extension (prune n parents)) (Type (c,subst_last HOLogic.unitT Ts)) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1833 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1834 | val recT0 = recT 0; | 
| 17261 | 1835 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1836 | fun mk_rec args n = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1837 | let val (args',more) = chop_last args; | 
| 17261 | 1838 | fun mk_ext' (((name,T),args),more) = mk_ext (name,T) (args@[more]); | 
| 1839 | fun build Ts = | |
| 30190 | 1840 | List.foldr mk_ext' more (prune n (extension_names ~~ Ts ~~ (chunks parent_chunks args'))) | 
| 17261 | 1841 | in | 
| 1842 | if more = HOLogic.unit | |
| 1843 | then build (map recT (0 upto parent_len)) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1844 | else build (map rec_schemeT (0 upto parent_len)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1845 | end; | 
| 17261 | 1846 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1847 | val r_rec0 = mk_rec all_vars_more 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1848 | val r_rec_unit0 = mk_rec (all_vars@[HOLogic.unit]) 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1849 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1850 | fun r n = Free (rN, rec_schemeT n) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1851 | val r0 = r 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1852 | fun r_unit n = Free (rN, recT n) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1853 | val r_unit0 = r_unit 0; | 
| 15215 | 1854 | val w = Free (wN, rec_schemeT 0) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1855 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1856 | (* prepare print translation functions *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1857 | val field_tr's = | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1858 | print_translation (distinct (op =) (maps external_names (full_moreN :: names))); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1859 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1860 | val adv_ext_tr's = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1861 | let | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1862 | val trnames = external_names extN; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1863 | in map (gen_record_tr') trnames end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1864 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1865 | val adv_record_type_abbr_tr's = | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1866 | let val trnames = external_names (hd extension_names); | 
| 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1867 | val lastExt = unsuffix ext_typeN (fst extension); | 
| 17190 | 1868 | in map (gen_record_type_abbr_tr' name alphas zeta lastExt rec_schemeT0) trnames | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1869 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1870 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1871 | val adv_record_type_tr's = | 
| 25070 
e2a39b6526b0
replaced NameSpace.accesses' by NameSpace.external_names (depening on naming);
 wenzelm parents: 
24867diff
changeset | 1872 | let val trnames = if parent_len > 0 then external_names extN else []; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1873 | (* avoid conflict with adv_record_type_abbr_tr's *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1874 | in map (gen_record_type_tr') trnames | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1875 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1876 | |
| 17261 | 1877 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1878 | (* prepare declarations *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1879 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1880 | val sel_decls = map (mk_selC rec_schemeT0) bfields_more; | 
| 15215 | 1881 | val upd_decls = map (mk_updC updateN rec_schemeT0) bfields_more; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1882 | val make_decl = (makeN, all_types ---> recT0); | 
| 17261 | 1883 | val fields_decl = (fields_selN, types ---> Type extension); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1884 | val extend_decl = (extendN, recT0 --> moreT --> rec_schemeT0); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1885 | val truncate_decl = (truncateN, rec_schemeT0 --> recT0); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1886 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1887 | (* prepare definitions *) | 
| 17261 | 1888 | |
| 1889 | fun parent_more s = | |
| 1890 | if null parents then s | |
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 1891 | else mk_sel s (Long_Name.qualify (#name (List.last parents)) moreN, extT); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1892 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1893 | fun parent_more_upd v s = | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1894 | if null parents then v$s | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 1895 | else let val mp = Long_Name.qualify (#name (List.last parents)) moreN; | 
| 15215 | 1896 | in mk_upd updateN mp v s end; | 
| 17261 | 1897 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1898 | (*record (scheme) type abbreviation*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1899 | val recordT_specs = | 
| 30345 | 1900 | [(Binding.name (suffix schemeN bname), alphas @ [zeta], rec_schemeT0, Syntax.NoSyn), | 
| 1901 | (Binding.name bname, alphas, recT0, Syntax.NoSyn)]; | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1902 | |
| 17261 | 1903 | (*selectors*) | 
| 1904 | fun mk_sel_spec (c,T) = | |
| 1905 | Const (mk_selC rec_schemeT0 (c,T)) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1906 | :== (lambda r0 (Const (mk_selC extT (suffix ext_dest c,T))$parent_more r0)); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1907 | val sel_specs = map mk_sel_spec fields_more; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1908 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1909 | (*updates*) | 
| 15215 | 1910 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1911 | fun mk_upd_spec (c,T) = | 
| 17261 | 1912 | let | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1913 | val new = mk_upd' updN c (Free (base c,T-->T)) extT(*(parent_more r0)*); | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1914 | in Const (mk_updC updateN rec_schemeT0 (c,T))$(Free (base c,T-->T))$r0 | 
| 15215 | 1915 | :== (parent_more_upd new r0) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1916 | end; | 
| 17261 | 1917 | val upd_specs = map mk_upd_spec fields_more; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1918 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1919 | (*derived operations*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1920 | val make_spec = Const (full makeN, all_types ---> recT0) $$ all_vars :== | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1921 | mk_rec (all_vars @ [HOLogic.unit]) 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1922 | val fields_spec = Const (full fields_selN, types ---> Type extension) $$ vars :== | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1923 | mk_rec (all_vars @ [HOLogic.unit]) parent_len; | 
| 17261 | 1924 | val extend_spec = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1925 | Const (full extendN, recT0-->moreT-->rec_schemeT0) $ r_unit0 $ more :== | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1926 | mk_rec ((map (mk_sel r_unit0) all_fields) @ [more]) 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1927 | val truncate_spec = Const (full truncateN, rec_schemeT0 --> recT0) $ r0 :== | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1928 | mk_rec ((map (mk_sel r0) all_fields) @ [HOLogic.unit]) 0; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1929 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1930 | (* 2st stage: defs_thy *) | 
| 17261 | 1931 | |
| 16379 | 1932 | fun mk_defs () = | 
| 1933 | extension_thy | |
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1934 | |> Sign.add_trfuns | 
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1935 | ([],[],field_tr's, []) | 
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1936 | |> Sign.add_advanced_trfuns | 
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1937 | ([],[],adv_ext_tr's @ adv_record_type_tr's @ adv_record_type_abbr_tr's,[]) | 
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1938 | |> Sign.parent_path | 
| 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1939 | |> Sign.add_tyabbrs_i recordT_specs | 
| 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1940 | |> Sign.add_path bname | 
| 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 1941 | |> Sign.add_consts_i | 
| 30345 | 1942 | (map2 (fn (x, T) => fn mx => (Binding.name x, T, mx)) | 
| 1943 | sel_decls (field_syntax @ [Syntax.NoSyn])) | |
| 1944 | |> (Sign.add_consts_i o map (fn (x, T) => (Binding.name x, T, Syntax.NoSyn))) | |
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1945 | (upd_decls @ [make_decl, fields_decl, extend_decl, truncate_decl]) | 
| 29579 | 1946 | |> ((PureThy.add_defs false o map (Thm.no_attributes o apfst Binding.name)) sel_specs) | 
| 1947 | ||>> ((PureThy.add_defs false o map (Thm.no_attributes o apfst Binding.name)) upd_specs) | |
| 1948 | ||>> ((PureThy.add_defs false o map (Thm.no_attributes o apfst Binding.name)) | |
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1949 | [make_spec, fields_spec, extend_spec, truncate_spec]) | 
| 24867 | 1950 | |-> (fn defs as ((sel_defs, upd_defs), derived_defs) => | 
| 28370 | 1951 | fold Code.add_default_eqn sel_defs | 
| 1952 | #> fold Code.add_default_eqn upd_defs | |
| 1953 | #> fold Code.add_default_eqn derived_defs | |
| 22747 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1954 | #> pair defs) | 
| 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1955 | val (((sel_defs, upd_defs), derived_defs), defs_thy) = | 
| 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1956 | timeit_msg "record trfuns/tyabbrs/selectors/updates/make/fields/extend/truncate defs:" | 
| 
0c9c413b4678
add definitions explicitly to code generator table
 haftmann parents: 
22693diff
changeset | 1957 | mk_defs; | 
| 17261 | 1958 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1959 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1960 | (* prepare propositions *) | 
| 17261 | 1961 | val _ = timing_msg "record preparing propositions"; | 
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1962 | val P = Free (Name.variant all_variants "P", rec_schemeT0-->HOLogic.boolT); | 
| 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1963 | val C = Free (Name.variant all_variants "C", HOLogic.boolT); | 
| 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 1964 | val P_unit = Free (Name.variant all_variants "P", recT0-->HOLogic.boolT); | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1965 | |
| 17261 | 1966 | (*selectors*) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1967 | val sel_conv_props = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1968 | map (fn (c, x as Free (_,T)) => mk_sel r_rec0 (c,T) === x) named_vars_more; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1969 | |
| 17261 | 1970 | (*updates*) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1971 | fun mk_upd_prop (i,(c,T)) = | 
| 21226 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1972 | let val x' = Free (Name.variant all_variants (base c ^ "'"),T-->T); | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1973 | val n = parent_fields_len + i; | 
| 
a607ae87ee81
field-update in records is generalised to take a function on the field
 schirmer parents: 
21109diff
changeset | 1974 | val args' = nth_map n (K (x'$nth all_vars_more n)) all_vars_more | 
| 15215 | 1975 | in mk_upd updateN c x' r_rec0 === mk_rec args' 0 end; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1976 | val upd_conv_props = ListPair.map mk_upd_prop (idxms, fields_more); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1977 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1978 | (*induct*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1979 | val induct_scheme_prop = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1980 | All (map dest_Free all_vars_more) (Trueprop (P $ r_rec0)) ==> Trueprop (P $ r0); | 
| 17261 | 1981 | val induct_prop = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1982 | (All (map dest_Free all_vars) (Trueprop (P_unit $ r_rec_unit0)), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1983 | Trueprop (P_unit $ r_unit0)); | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1984 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1985 | (*surjective*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1986 | val surjective_prop = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1987 | let val args = map (fn (c,Free (_,T)) => mk_sel r0 (c,T)) all_named_vars_more | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1988 | in r0 === mk_rec args 0 end; | 
| 17261 | 1989 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1990 | (*cases*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1991 | val cases_scheme_prop = | 
| 17261 | 1992 | (All (map dest_Free all_vars_more) | 
| 1993 | (Trueprop (HOLogic.mk_eq (r0,r_rec0)) ==> Trueprop C)) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1994 | ==> Trueprop C; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1995 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1996 | val cases_prop = | 
| 17261 | 1997 | (All (map dest_Free all_vars) | 
| 1998 | (Trueprop (HOLogic.mk_eq (r_unit0,r_rec_unit0)) ==> Trueprop C)) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 1999 | ==> Trueprop C; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2000 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2001 | (*split*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2002 | val split_meta_prop = | 
| 20071 
8f3e1ddb50e6
replaced Term.variant(list) by Name.variant(_list);
 wenzelm parents: 
20049diff
changeset | 2003 | let val P = Free (Name.variant all_variants "P", rec_schemeT0-->Term.propT) in | 
| 17261 | 2004 | Logic.mk_equals | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2005 | (All [dest_Free r0] (P $ r0), All (map dest_Free all_vars_more) (P $ r_rec0)) | 
| 17261 | 2006 | end; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2007 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2008 | val split_object_prop = | 
| 30190 | 2009 | let fun ALL vs t = List.foldr (fn ((v,T),t) => HOLogic.mk_all (v,T,t)) t vs | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2010 | in (ALL [dest_Free r0] (P $ r0)) === (ALL (map dest_Free all_vars_more) (P $ r_rec0)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2011 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2012 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2013 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2014 | val split_ex_prop = | 
| 30190 | 2015 | let fun EX vs t = List.foldr (fn ((v,T),t) => HOLogic.mk_exists (v,T,t)) t vs | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2016 | in (EX [dest_Free r0] (P $ r0)) === (EX (map dest_Free all_vars_more) (P $ r_rec0)) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2017 | end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2018 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2019 | (*equality*) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2020 | val equality_prop = | 
| 17261 | 2021 | let | 
| 2022 | val s' = Free (rN ^ "'", rec_schemeT0) | |
| 2023 | fun mk_sel_eq (c,Free (_,T)) = mk_sel r0 (c,T) === mk_sel s' (c,T) | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2024 | val seleqs = map mk_sel_eq all_named_vars_more | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2025 | in All (map dest_Free [r0,s']) (Logic.list_implies (seleqs,r0 === s')) end; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2026 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2027 | (* 3rd stage: thms_thy *) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2028 | |
| 17510 | 2029 | fun prove stndrd = quick_and_dirty_prove stndrd defs_thy; | 
| 2030 | val prove_standard = quick_and_dirty_prove true defs_thy; | |
| 17261 | 2031 | |
| 15215 | 2032 | fun prove_simp stndrd ss simps = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2033 | let val tac = simp_all_tac ss simps | 
| 15215 | 2034 | in fn prop => prove stndrd [] prop (K tac) end; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2035 | |
| 17510 | 2036 | val ss = get_simpset defs_thy; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2037 | |
| 17261 | 2038 | fun sel_convs_prf () = map (prove_simp false ss | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2039 | (sel_defs@ext_dest_convs)) sel_conv_props; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2040 | val sel_convs = timeit_msg "record sel_convs proof:" sel_convs_prf; | 
| 15215 | 2041 | fun sel_convs_standard_prf () = map standard sel_convs | 
| 17261 | 2042 | val sel_convs_standard = | 
| 2043 | timeit_msg "record sel_convs_standard proof:" sel_convs_standard_prf; | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2044 | |
| 17261 | 2045 | fun upd_convs_prf () = | 
| 2046 | map (prove_simp true ss (upd_defs@u_convs)) upd_conv_props; | |
| 2047 | ||
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2048 | val upd_convs = timeit_msg "record upd_convs proof:" upd_convs_prf; | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2049 | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2050 | val parent_induct = if null parents then [] else [#induct (hd (rev parents))]; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2051 | |
| 27217 | 2052 | fun induct_scheme_prf () = prove_standard [] induct_scheme_prop (fn _ => | 
| 17261 | 2053 | (EVERY [if null parent_induct | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2054 | then all_tac else try_param_tac rN (hd parent_induct) 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2055 | try_param_tac rN ext_induct 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2056 | asm_simp_tac HOL_basic_ss 1])); | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2057 | val induct_scheme = timeit_msg "record induct_scheme proof:" induct_scheme_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2058 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2059 | fun induct_prf () = | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2060 | let val (assm, concl) = induct_prop; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2061 | in | 
| 20248 | 2062 |         prove_standard [assm] concl (fn {prems, ...} =>
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2063 | try_param_tac rN induct_scheme 1 | 
| 27104 
791607529f6d
rep_datatype command now takes list of constructors as input arguments
 haftmann parents: 
26957diff
changeset | 2064 |           THEN try_param_tac "more" @{thm unit.induct} 1
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2065 | THEN resolve_tac prems 1) | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2066 | end; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2067 | val induct = timeit_msg "record induct proof:" induct_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2068 | |
| 17261 | 2069 | fun surjective_prf () = | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 2070 | prove_standard [] surjective_prop (fn prems => | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2071 | (EVERY [try_param_tac rN induct_scheme 1, | 
| 15215 | 2072 | simp_tac (ss addsimps sel_convs_standard) 1])) | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2073 | val surjective = timeit_msg "record surjective proof:" surjective_prf; | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2074 | |
| 15215 | 2075 | fun cases_scheme_prf_opt () = | 
| 17261 | 2076 | let | 
| 15215 | 2077 | val (_$(Pvar$_)) = concl_of induct_scheme; | 
| 17261 | 2078 | val ind = cterm_instantiate | 
| 18858 | 2079 | [(cterm_of defs_thy Pvar, cterm_of defs_thy | 
| 15215 | 2080 | (lambda w (HOLogic.imp$HOLogic.mk_eq(r0,w)$C)))] | 
| 2081 | induct_scheme; | |
| 2082 | in standard (ObjectLogic.rulify (mp OF [ind, refl])) end; | |
| 2083 | ||
| 2084 | fun cases_scheme_prf_noopt () = | |
| 27217 | 2085 | prove_standard [] cases_scheme_prop (fn _ => | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2086 | EVERY [asm_full_simp_tac (HOL_basic_ss addsimps [atomize_all, atomize_imp]) 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2087 | try_param_tac rN induct_scheme 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2088 | rtac impI 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2089 | REPEAT (etac allE 1), | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2090 | etac mp 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2091 | rtac refl 1]) | 
| 15215 | 2092 | val cases_scheme_prf = quick_and_dirty_prf cases_scheme_prf_noopt cases_scheme_prf_opt; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2093 | val cases_scheme = timeit_msg "record cases_scheme proof:" cases_scheme_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2094 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2095 | fun cases_prf () = | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 2096 | prove_standard [] cases_prop (fn _ => | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2097 | try_param_tac rN cases_scheme 1 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2098 | THEN simp_all_tac HOL_basic_ss [unit_all_eq1]); | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2099 | val cases = timeit_msg "record cases proof:" cases_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2100 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2101 | fun split_meta_prf () = | 
| 27217 | 2102 | prove false [] split_meta_prop (fn _ => | 
| 21687 | 2103 | EVERY [rtac equal_intr_rule 1, Goal.norm_hhf_tac 1, | 
| 17960 | 2104 | etac meta_allE 1, atac 1, | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2105 | rtac (prop_subst OF [surjective]) 1, | 
| 17960 | 2106 | REPEAT (etac meta_allE 1), atac 1]); | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2107 | val split_meta = timeit_msg "record split_meta proof:" split_meta_prf; | 
| 15215 | 2108 | val split_meta_standard = standard split_meta; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2109 | |
| 15215 | 2110 | fun split_object_prf_opt () = | 
| 17261 | 2111 | let | 
| 18858 | 2112 | val cPI= cterm_of defs_thy (lambda r0 (Trueprop (P$r0))); | 
| 15215 | 2113 | val (_$Abs(_,_,P$_)) = fst (Logic.dest_equals (concl_of split_meta_standard)); | 
| 18858 | 2114 | val cP = cterm_of defs_thy P; | 
| 15215 | 2115 | val split_meta' = cterm_instantiate [(cP,cPI)] split_meta_standard; | 
| 2116 | val (l,r) = HOLogic.dest_eq (HOLogic.dest_Trueprop split_object_prop); | |
| 18858 | 2117 | val cl = cterm_of defs_thy (HOLogic.mk_Trueprop l); | 
| 2118 | val cr = cterm_of defs_thy (HOLogic.mk_Trueprop r); | |
| 15215 | 2119 | val thl = assume cl (*All r. P r*) (* 1 *) | 
| 2120 | |> obj_to_meta_all (*!!r. P r*) | |
| 17261 | 2121 | |> equal_elim split_meta' (*!!n m more. P (ext n m more)*) | 
| 2122 | |> meta_to_obj_all (*All n m more. P (ext n m more)*) (* 2*) | |
| 15215 | 2123 | |> implies_intr cl (* 1 ==> 2 *) | 
| 2124 | val thr = assume cr (*All n m more. P (ext n m more)*) | |
| 2125 | |> obj_to_meta_all (*!!n m more. P (ext n m more)*) | |
| 17261 | 2126 | |> equal_elim (symmetric split_meta') (*!!r. P r*) | 
| 15215 | 2127 | |> meta_to_obj_all (*All r. P r*) | 
| 2128 | |> implies_intr cr (* 2 ==> 1 *) | |
| 17261 | 2129 | in standard (thr COMP (thl COMP iffI)) end; | 
| 15215 | 2130 | |
| 2131 | fun split_object_prf_noopt () = | |
| 27217 | 2132 | prove_standard [] split_object_prop (fn _ => | 
| 17261 | 2133 | EVERY [rtac iffI 1, | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2134 | REPEAT (rtac allI 1), etac allE 1, atac 1, | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2135 | rtac allI 1, rtac induct_scheme 1,REPEAT (etac allE 1),atac 1]); | 
| 15215 | 2136 | |
| 17261 | 2137 | val split_object_prf = quick_and_dirty_prf split_object_prf_noopt split_object_prf_opt; | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2138 | val split_object = timeit_msg "record split_object proof:" split_object_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2139 | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2140 | |
| 17261 | 2141 | fun split_ex_prf () = | 
| 27217 | 2142 | prove_standard [] split_ex_prop (fn _ => | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2143 | EVERY [rtac iffI 1, | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2144 | etac exE 1, | 
| 15215 | 2145 | simp_tac (HOL_basic_ss addsimps [split_meta_standard]) 1, | 
| 2146 | ex_inst_tac 1, | |
| 2147 | (*REPEAT (rtac exI 1),*) | |
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2148 | atac 1, | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2149 | REPEAT (etac exE 1), | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2150 | rtac exI 1, | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2151 | atac 1]); | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2152 | val split_ex = timeit_msg "record split_ex proof:" split_ex_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2153 | |
| 17261 | 2154 | fun equality_tac thms = | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2155 | let val (s'::s::eqs) = rev thms; | 
| 15215 | 2156 | val ss' = ss addsimps (s'::s::sel_convs_standard); | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2157 | val eqs' = map (simplify ss') eqs; | 
| 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2158 | in simp_tac (HOL_basic_ss addsimps (s'::s::eqs')) 1 end; | 
| 17261 | 2159 | |
| 27217 | 2160 |    fun equality_prf () = prove_standard [] equality_prop (fn {context, ...} =>
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2161 | fn st => let val [s, s'] = map #1 (rev (Tactic.innermost_params 1 st)) in | 
| 27239 | 2162 | st |> (res_inst_tac context [((rN, 0), s)] cases_scheme 1 | 
| 2163 | THEN res_inst_tac context [((rN, 0), s')] cases_scheme 1 | |
| 17261 | 2164 | THEN (METAHYPS equality_tac 1)) | 
| 15012 
28fa57b57209
Added reference record_definition_quick_and_dirty_sensitive, to
 schirmer parents: 
14981diff
changeset | 2165 | (* simp_all_tac ss (sel_convs) would also work but is less efficient *) | 
| 17261 | 2166 | end); | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 2167 | val equality = timeit_msg "record equality proof:" equality_prf; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2168 | |
| 18377 | 2169 | val ((([sel_convs',upd_convs',sel_defs',upd_defs',[split_meta',split_object',split_ex'],derived_defs'], | 
| 2170 | [surjective',equality']),[induct_scheme',induct',cases_scheme',cases']), thms_thy) = | |
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2171 | defs_thy | 
| 29579 | 2172 | |> (PureThy.add_thmss o map (Thm.no_attributes o apfst Binding.name)) | 
| 15215 | 2173 |          [("select_convs", sel_convs_standard),
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2174 |           ("update_convs", upd_convs),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2175 |           ("select_defs", sel_defs),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2176 |           ("update_defs", upd_defs),
 | 
| 15215 | 2177 |           ("splits", [split_meta_standard,split_object,split_ex]),
 | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2178 |           ("defs", derived_defs)]
 | 
| 29579 | 2179 | ||>> (PureThy.add_thms o map (Thm.no_attributes o apfst Binding.name)) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2180 |           [("surjective", surjective),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2181 |            ("equality", equality)]
 | 
| 29579 | 2182 | ||>> (PureThy.add_thms o (map o apfst o apfst) Binding.name) | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2183 |         [(("induct_scheme", induct_scheme), induct_type_global (suffix schemeN name)),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2184 |          (("induct", induct), induct_type_global name),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2185 |          (("cases_scheme", cases_scheme), cases_type_global (suffix schemeN name)),
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2186 |          (("cases", cases), cases_type_global name)];
 | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2187 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2188 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2189 | val sel_upd_simps = sel_convs' @ upd_convs'; | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2190 | val iffs = [ext_inject] | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2191 | val final_thy = | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2192 | thms_thy | 
| 18377 | 2193 | |> (snd oo PureThy.add_thmss) | 
| 29871 
74366d50cf2b
Added nitpick_const_simp attribute to recdef and record packages.
 blanchet parents: 
29579diff
changeset | 2194 | [((Binding.name "simps", sel_upd_simps), | 
| 
74366d50cf2b
Added nitpick_const_simp attribute to recdef and record packages.
 blanchet parents: 
29579diff
changeset | 2195 | [Simplifier.simp_add, Nitpick_Const_Simp_Thms.add]), | 
| 29579 | 2196 | ((Binding.name "iffs", iffs), [iff_add])] | 
| 17261 | 2197 | |> put_record name (make_record_info args parent fields extension induct_scheme') | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2198 | |> put_sel_upd (names @ [full_moreN]) sel_upd_simps | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2199 | |> add_record_equalities extension_id equality' | 
| 15015 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 2200 | |> add_extinjects ext_inject | 
| 
c5768e8c4da4
* record_upd_simproc also simplifies trivial updates:
 schirmer parents: 
15012diff
changeset | 2201 | |> add_extsplit extension_name ext_split | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2202 | |> add_record_splits extension_id (split_meta',split_object',split_ex',induct_scheme') | 
| 17261 | 2203 | |> add_extfields extension_name (fields @ [(full_moreN,moreT)]) | 
| 2204 | |> add_fieldext (extension_name,snd extension) (names @ [full_moreN]) | |
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 2205 | |> Sign.parent_path; | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2206 | |
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2207 | in final_thy | 
| 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2208 | end; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2209 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2210 | |
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2211 | (* add_record *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2212 | |
| 4895 | 2213 | (*we do all preparations and error checks here, deferring the real | 
| 2214 | work to record_definition*) | |
| 26477 
ecf06644f6cb
eliminated quiete_mode ref (turned into proper argument);
 wenzelm parents: 
26423diff
changeset | 2215 | fun gen_add_record prep_typ prep_raw_parent quiet_mode (params, bname) raw_parent raw_fields thy = | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2216 | let | 
| 17261 | 2217 | val _ = Theory.requires thy "Record" "record definitions"; | 
| 26477 
ecf06644f6cb
eliminated quiete_mode ref (turned into proper argument);
 wenzelm parents: 
26423diff
changeset | 2218 |     val _ = if quiet_mode then () else writeln ("Defining record " ^ quote bname ^ " ...");
 | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2219 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2220 | val ctxt = ProofContext.init thy; | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2221 | |
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2222 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2223 | (* parents *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2224 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2225 | fun prep_inst T = fst (cert_typ ctxt T []); | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2226 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2227 | val parent = Option.map (apfst (map prep_inst) o prep_raw_parent ctxt) raw_parent | 
| 18678 | 2228 |       handle ERROR msg => cat_error msg ("The error(s) above in parent record specification");
 | 
| 12247 | 2229 | val parents = add_parents thy parent []; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2230 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2231 | val init_env = | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2232 | (case parent of | 
| 15531 | 2233 | NONE => [] | 
| 30190 | 2234 | | SOME (types, _) => List.foldr OldTerm.add_typ_tfrees [] types); | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2235 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2236 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2237 | (* fields *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2238 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2239 | fun prep_field (c, raw_T, mx) env = | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2240 | let val (T, env') = prep_typ ctxt raw_T env handle ERROR msg => | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2241 |         cat_error msg ("The error(s) above occured in record field " ^ quote c)
 | 
| 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2242 | in ((c, T, mx), env') end; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2243 | |
| 27278 
129574589734
export read_typ/cert_typ -- version with regular context operations;
 wenzelm parents: 
27239diff
changeset | 2244 | val (bfields, envir) = fold_map prep_field raw_fields init_env; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2245 | val envir_names = map fst envir; | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2246 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2247 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2248 | (* args *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2249 | |
| 22578 | 2250 | val defaultS = Sign.defaultS thy; | 
| 17485 | 2251 | val args = map (fn x => (x, AList.lookup (op =) envir x |> the_default defaultS)) params; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2252 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2253 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2254 | (* errors *) | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2255 | |
| 28965 | 2256 | val name = Sign.full_bname thy bname; | 
| 17261 | 2257 | val err_dup_record = | 
| 4890 | 2258 | if is_none (get_record thy name) then [] | 
| 2259 | else ["Duplicate definition of record " ^ quote name]; | |
| 2260 | ||
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2261 | val err_dup_parms = | 
| 18964 | 2262 | (case duplicates (op =) params of | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2263 | [] => [] | 
| 4890 | 2264 | | dups => ["Duplicate parameter(s) " ^ commas dups]); | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2265 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2266 | val err_extra_frees = | 
| 20951 
868120282837
gen_rem(s) abandoned in favour of remove / subtract
 haftmann parents: 
20484diff
changeset | 2267 | (case subtract (op =) params envir_names of | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2268 | [] => [] | 
| 4890 | 2269 | | extras => ["Extra free type variable(s) " ^ commas extras]); | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2270 | |
| 4890 | 2271 | val err_no_fields = if null bfields then ["No fields present"] else []; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2272 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2273 | val err_dup_fields = | 
| 18964 | 2274 | (case duplicates (op =) (map #1 bfields) of | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2275 | [] => [] | 
| 4890 | 2276 | | dups => ["Duplicate field(s) " ^ commas_quote dups]); | 
| 2277 | ||
| 2278 | val err_bad_fields = | |
| 12506 | 2279 | if forall (not_equal moreN o #1) bfields then [] | 
| 4890 | 2280 | else ["Illegal field name " ^ quote moreN]; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2281 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2282 | val err_dup_sorts = | 
| 18964 | 2283 | (case duplicates (op =) envir_names of | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2284 | [] => [] | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2285 | | dups => ["Inconsistent sort constraints for " ^ commas dups]); | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2286 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2287 | val errs = | 
| 4890 | 2288 | err_dup_record @ err_dup_parms @ err_extra_frees @ err_no_fields @ | 
| 2289 | err_dup_fields @ err_bad_fields @ err_dup_sorts; | |
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2290 | in | 
| 14700 
2f885b7e5ba7
reimplementation of HOL records; only one type is created for
 schirmer parents: 
14643diff
changeset | 2291 | if null errs then () else error (cat_lines errs) ; | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2292 | thy |> record_definition (args, bname) parent parents bfields | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2293 | end | 
| 18678 | 2294 |   handle ERROR msg => cat_error msg ("Failed to define record " ^ quote bname);
 | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2295 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2296 | val add_record = gen_add_record read_typ read_raw_parent; | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2297 | val add_record_i = gen_add_record cert_typ (K I); | 
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2298 | |
| 6358 | 2299 | (* setup theory *) | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2300 | |
| 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2301 | val setup = | 
| 24712 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 2302 | Sign.add_trfuns ([], parse_translation, [], []) #> | 
| 
64ed05609568
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24624diff
changeset | 2303 | Sign.add_advanced_trfuns ([], adv_parse_translation, [], []) #> | 
| 26496 
49ae9456eba9
purely functional setup of claset/simpset/clasimpset;
 wenzelm parents: 
26477diff
changeset | 2304 | Simplifier.map_simpset (fn ss => | 
| 
49ae9456eba9
purely functional setup of claset/simpset/clasimpset;
 wenzelm parents: 
26477diff
changeset | 2305 | ss addsimprocs [record_simproc, record_upd_simproc, record_eq_simproc]); | 
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2306 | |
| 6358 | 2307 | (* outer syntax *) | 
| 2308 | ||
| 17057 | 2309 | local structure P = OuterParse and K = OuterKeyword in | 
| 6358 | 2310 | |
| 2311 | val record_decl = | |
| 12876 
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
 wenzelm parents: 
12590diff
changeset | 2312 | P.type_args -- P.name -- | 
| 
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
 wenzelm parents: 
12590diff
changeset | 2313 | (P.$$$ "=" |-- Scan.option (P.typ --| P.$$$ "+") -- Scan.repeat1 P.const); | 
| 6358 | 2314 | |
| 24867 | 2315 | val _ = | 
| 17261 | 2316 | OuterSyntax.command "record" "define extensible record" K.thy_decl | 
| 26477 
ecf06644f6cb
eliminated quiete_mode ref (turned into proper argument);
 wenzelm parents: 
26423diff
changeset | 2317 | (record_decl >> (fn (x, (y, z)) => Toplevel.theory (add_record false x y z))); | 
| 6358 | 2318 | |
| 4867 
9be2bf0ce909
package extensible records with structural subtyping in HOL -- still
 wenzelm parents: diff
changeset | 2319 | end; | 
| 5698 | 2320 | |
| 6384 | 2321 | end; | 
| 2322 | ||
| 15215 | 2323 | |
| 5698 | 2324 | structure BasicRecordPackage: BASIC_RECORD_PACKAGE = RecordPackage; | 
| 17261 | 2325 | open BasicRecordPackage; |