author | desharna |
Wed, 30 Jul 2014 10:50:28 +0200 | |
changeset 57700 | a2c4adb839a9 |
parent 57633 | 4ff8c090d580 |
child 57882 | 38bf4de248a6 |
permissions | -rw-r--r-- |
54701 | 1 |
(* Title: HOL/Tools/Ctr_Sugar/ctr_sugar.ML |
49017 | 2 |
Author: Jasmin Blanchette, TU Muenchen |
54397 | 3 |
Copyright 2012, 2013 |
49017 | 4 |
|
51797 | 5 |
Wrapping existing freely generated type's constructors. |
49017 | 6 |
*) |
7 |
||
54006 | 8 |
signature CTR_SUGAR = |
49017 | 9 |
sig |
51840 | 10 |
type ctr_sugar = |
51839 | 11 |
{ctrs: term list, |
52375 | 12 |
casex: term, |
51839 | 13 |
discs: term list, |
51819 | 14 |
selss: term list list, |
15 |
exhaust: thm, |
|
52375 | 16 |
nchotomy: thm, |
51819 | 17 |
injects: thm list, |
18 |
distincts: thm list, |
|
19 |
case_thms: thm list, |
|
52375 | 20 |
case_cong: thm, |
21 |
weak_case_cong: thm, |
|
22 |
split: thm, |
|
23 |
split_asm: thm, |
|
56858 | 24 |
disc_defs: thm list, |
51819 | 25 |
disc_thmss: thm list list, |
26 |
discIs: thm list, |
|
56858 | 27 |
sel_defs: thm list, |
53475 | 28 |
sel_thmss: thm list list, |
54900 | 29 |
disc_excludesss: thm list list list, |
53475 | 30 |
disc_exhausts: thm list, |
53916 | 31 |
sel_exhausts: thm list, |
53475 | 32 |
collapses: thm list, |
33 |
expands: thm list, |
|
53917 | 34 |
sel_splits: thm list, |
35 |
sel_split_asms: thm list, |
|
54491 | 36 |
case_eq_ifs: thm list}; |
51809 | 37 |
|
51840 | 38 |
val morph_ctr_sugar: morphism -> ctr_sugar -> ctr_sugar |
54256 | 39 |
val transfer_ctr_sugar: Proof.context -> ctr_sugar -> ctr_sugar |
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
40 |
val ctr_sugar_of: Proof.context -> string -> ctr_sugar option |
53906 | 41 |
val ctr_sugars_of: Proof.context -> ctr_sugar list |
54403 | 42 |
val ctr_sugar_of_case: Proof.context -> string -> ctr_sugar option |
56345 | 43 |
val ctr_sugar_interpretation: (ctr_sugar -> theory -> theory) -> theory -> theory |
54399 | 44 |
val register_ctr_sugar: string -> ctr_sugar -> local_theory -> local_theory |
55444
ec73f81e49e7
iteration n in the 'default' vs. 'update_new' vs. 'update' saga -- 'update' makes sense now that we honor the canonical order on 'merge' (as opposed to raising 'DUP')
blanchet
parents:
55410
diff
changeset
|
45 |
val default_register_ctr_sugar_global: string -> ctr_sugar -> theory -> theory |
51823
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
46 |
|
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
47 |
val mk_half_pairss: 'a list * 'a list -> ('a * 'a) list list |
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
48 |
val join_halves: int -> 'a list list -> 'a list list -> 'a list * 'a list list list |
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
49 |
|
49203 | 50 |
val mk_ctr: typ list -> term -> term |
53864
a48d4bd3faaa
use case rather than sequence of ifs in expansion
blanchet
parents:
53857
diff
changeset
|
51 |
val mk_case: typ list -> typ -> term -> term |
49484 | 52 |
val mk_disc_or_sel: typ list -> term -> term |
49622 | 53 |
val name_of_ctr: term -> string |
51777
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
54 |
val name_of_disc: term -> string |
53888 | 55 |
val dest_ctr: Proof.context -> string -> term -> term * term list |
54970
891141de5672
only destruct cases equipped with the right stuff (in particular, 'sel_split')
blanchet
parents:
54900
diff
changeset
|
56 |
val dest_case: Proof.context -> string -> typ list -> term -> |
891141de5672
only destruct cases equipped with the right stuff (in particular, 'sel_split')
blanchet
parents:
54900
diff
changeset
|
57 |
(ctr_sugar * term list * term list) option |
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
58 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
59 |
type ('c, 'a) ctr_spec = (binding * 'c) * 'a list |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
60 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
61 |
val disc_of_ctr_spec: ('c, 'a) ctr_spec -> binding |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
62 |
val ctr_of_ctr_spec: ('c, 'a) ctr_spec -> 'c |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
63 |
val args_of_ctr_spec: ('c, 'a) ctr_spec -> 'a list |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
64 |
|
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
65 |
val free_constructors: ({prems: thm list, context: Proof.context} -> tactic) list list -> |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
66 |
(((bool * bool) * binding) * (term, binding) ctr_spec list) * term list -> local_theory -> |
51840 | 67 |
ctr_sugar * local_theory |
49286 | 68 |
val parse_bound_term: (binding * string) parser |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
69 |
val parse_ctr_options: (bool * bool) parser |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
70 |
val parse_ctr_spec: 'c parser -> 'a parser -> ('c, 'a) ctr_spec parser |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
71 |
val parse_sel_default_eqs: string list parser |
49017 | 72 |
end; |
73 |
||
54006 | 74 |
structure Ctr_Sugar : CTR_SUGAR = |
49017 | 75 |
struct |
76 |
||
54008
b15cfc2864de
refactoring -- splitting between constructor sugar dependencies and true BNF dependencies
blanchet
parents:
54007
diff
changeset
|
77 |
open Ctr_Sugar_Util |
54006 | 78 |
open Ctr_Sugar_Tactics |
54615
62fb5af93fe2
generalized datatype code generation code so that it works with old-style and new-style (co)datatypes (as long as they are not local)
blanchet
parents:
54493
diff
changeset
|
79 |
open Ctr_Sugar_Code |
49017 | 80 |
|
51840 | 81 |
type ctr_sugar = |
51839 | 82 |
{ctrs: term list, |
52375 | 83 |
casex: term, |
51839 | 84 |
discs: term list, |
51819 | 85 |
selss: term list list, |
86 |
exhaust: thm, |
|
52375 | 87 |
nchotomy: thm, |
51819 | 88 |
injects: thm list, |
89 |
distincts: thm list, |
|
90 |
case_thms: thm list, |
|
52375 | 91 |
case_cong: thm, |
92 |
weak_case_cong: thm, |
|
93 |
split: thm, |
|
94 |
split_asm: thm, |
|
56858 | 95 |
disc_defs: thm list, |
51819 | 96 |
disc_thmss: thm list list, |
97 |
discIs: thm list, |
|
56858 | 98 |
sel_defs: thm list, |
53475 | 99 |
sel_thmss: thm list list, |
54900 | 100 |
disc_excludesss: thm list list list, |
53475 | 101 |
disc_exhausts: thm list, |
53916 | 102 |
sel_exhausts: thm list, |
53475 | 103 |
collapses: thm list, |
104 |
expands: thm list, |
|
53917 | 105 |
sel_splits: thm list, |
106 |
sel_split_asms: thm list, |
|
54491 | 107 |
case_eq_ifs: thm list}; |
51809 | 108 |
|
52375 | 109 |
fun morph_ctr_sugar phi {ctrs, casex, discs, selss, exhaust, nchotomy, injects, distincts, |
56858 | 110 |
case_thms, case_cong, weak_case_cong, split, split_asm, disc_defs, disc_thmss, discIs, sel_defs, |
111 |
sel_thmss, disc_excludesss, disc_exhausts, sel_exhausts, collapses, expands, sel_splits, |
|
112 |
sel_split_asms, case_eq_ifs} = |
|
51839 | 113 |
{ctrs = map (Morphism.term phi) ctrs, |
52375 | 114 |
casex = Morphism.term phi casex, |
51839 | 115 |
discs = map (Morphism.term phi) discs, |
51823
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
116 |
selss = map (map (Morphism.term phi)) selss, |
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
117 |
exhaust = Morphism.thm phi exhaust, |
52375 | 118 |
nchotomy = Morphism.thm phi nchotomy, |
51823
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
119 |
injects = map (Morphism.thm phi) injects, |
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
120 |
distincts = map (Morphism.thm phi) distincts, |
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
121 |
case_thms = map (Morphism.thm phi) case_thms, |
52375 | 122 |
case_cong = Morphism.thm phi case_cong, |
123 |
weak_case_cong = Morphism.thm phi weak_case_cong, |
|
124 |
split = Morphism.thm phi split, |
|
125 |
split_asm = Morphism.thm phi split_asm, |
|
56858 | 126 |
disc_defs = map (Morphism.thm phi) disc_defs, |
51823
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
127 |
disc_thmss = map (map (Morphism.thm phi)) disc_thmss, |
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
128 |
discIs = map (Morphism.thm phi) discIs, |
56858 | 129 |
sel_defs = map (Morphism.thm phi) sel_defs, |
53475 | 130 |
sel_thmss = map (map (Morphism.thm phi)) sel_thmss, |
54900 | 131 |
disc_excludesss = map (map (map (Morphism.thm phi))) disc_excludesss, |
53475 | 132 |
disc_exhausts = map (Morphism.thm phi) disc_exhausts, |
53916 | 133 |
sel_exhausts = map (Morphism.thm phi) sel_exhausts, |
53475 | 134 |
collapses = map (Morphism.thm phi) collapses, |
135 |
expands = map (Morphism.thm phi) expands, |
|
53917 | 136 |
sel_splits = map (Morphism.thm phi) sel_splits, |
137 |
sel_split_asms = map (Morphism.thm phi) sel_split_asms, |
|
54491 | 138 |
case_eq_ifs = map (Morphism.thm phi) case_eq_ifs}; |
51823
38996458bc5c
create data structure for storing (co)datatype information
blanchet
parents:
51819
diff
changeset
|
139 |
|
53906 | 140 |
val transfer_ctr_sugar = |
54740 | 141 |
morph_ctr_sugar o Morphism.transfer_morphism o Proof_Context.theory_of; |
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
142 |
|
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
143 |
structure Data = Generic_Data |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
144 |
( |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
145 |
type T = ctr_sugar Symtab.table; |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
146 |
val empty = Symtab.empty; |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
147 |
val extend = I; |
55394
d5ebe055b599
more liberal merging of BNFs and constructor sugar
blanchet
parents:
55356
diff
changeset
|
148 |
fun merge data : T = Symtab.merge (K true) data; |
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
149 |
); |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
150 |
|
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
151 |
fun ctr_sugar_of ctxt = |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
152 |
Symtab.lookup (Data.get (Context.Proof ctxt)) |
53906 | 153 |
#> Option.map (transfer_ctr_sugar ctxt); |
154 |
||
155 |
fun ctr_sugars_of ctxt = |
|
156 |
Symtab.fold (cons o transfer_ctr_sugar ctxt o snd) (Data.get (Context.Proof ctxt)) []; |
|
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
157 |
|
54403 | 158 |
fun ctr_sugar_of_case ctxt s = |
159 |
find_first (fn {casex = Const (s', _), ...} => s' = s | _ => false) (ctr_sugars_of ctxt); |
|
160 |
||
56345 | 161 |
structure Ctr_Sugar_Interpretation = Interpretation |
162 |
( |
|
163 |
type T = ctr_sugar; |
|
164 |
val eq: T * T -> bool = op = o pairself #ctrs; |
|
165 |
); |
|
166 |
||
56376
5a93b8f928a2
added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
blanchet
parents:
56345
diff
changeset
|
167 |
fun with_repaired_path f (ctr_sugar as {ctrs = ctr1 :: _, ...} : ctr_sugar) thy = |
5a93b8f928a2
added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
blanchet
parents:
56345
diff
changeset
|
168 |
thy |
56767 | 169 |
|> Sign.root_path |
56376
5a93b8f928a2
added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
blanchet
parents:
56345
diff
changeset
|
170 |
|> Sign.add_path (Long_Name.qualifier (fst (dest_Type (body_type (fastype_of ctr1))))) |
56767 | 171 |
|> (fn thy => f (morph_ctr_sugar (Morphism.transfer_morphism thy) ctr_sugar) thy) |
172 |
|> Sign.restore_naming thy; |
|
56376
5a93b8f928a2
added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
blanchet
parents:
56345
diff
changeset
|
173 |
|
56657 | 174 |
fun ctr_sugar_interpretation f = Ctr_Sugar_Interpretation.interpretation (with_repaired_path f); |
56345 | 175 |
|
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
176 |
fun register_ctr_sugar key ctr_sugar = |
54285
578371ba74cc
reverted 3e1d230f1c00 -- pervasiveness is useful, cf. Coinductive_Nat in the AFP
blanchet
parents:
54265
diff
changeset
|
177 |
Local_Theory.declaration {syntax = false, pervasive = true} |
56345 | 178 |
(fn phi => Data.map (Symtab.update (key, morph_ctr_sugar phi ctr_sugar))) |
179 |
#> Local_Theory.background_theory (Ctr_Sugar_Interpretation.data ctr_sugar); |
|
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
180 |
|
56345 | 181 |
fun default_register_ctr_sugar_global key ctr_sugar thy = |
182 |
let val tab = Data.get (Context.Theory thy) in |
|
183 |
if Symtab.defined tab key then |
|
184 |
thy |
|
185 |
else |
|
186 |
thy |
|
187 |
|> Context.theory_map (Data.put (Symtab.update_new (key, ctr_sugar) tab)) |
|
188 |
|> Ctr_Sugar_Interpretation.data ctr_sugar |
|
189 |
end; |
|
54400 | 190 |
|
49223 | 191 |
val isN = "is_"; |
192 |
val unN = "un_"; |
|
57629
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
193 |
val notN = "not_"; |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
194 |
|
49223 | 195 |
fun mk_unN 1 1 suf = unN ^ suf |
196 |
| mk_unN _ l suf = unN ^ suf ^ string_of_int l; |
|
49046
3c5eba97d93a
allow default names for selectors via wildcard (_) + fix wrong index (k)
blanchet
parents:
49045
diff
changeset
|
197 |
|
49594
55e798614c45
tweaked theorem names (in particular, dropped s's)
blanchet
parents:
49591
diff
changeset
|
198 |
val caseN = "case"; |
49054 | 199 |
val case_congN = "case_cong"; |
54491 | 200 |
val case_eq_ifN = "case_eq_if"; |
49118 | 201 |
val collapseN = "collapse"; |
49122 | 202 |
val disc_excludeN = "disc_exclude"; |
49054 | 203 |
val disc_exhaustN = "disc_exhaust"; |
53694 | 204 |
val discN = "disc"; |
53700 | 205 |
val discIN = "discI"; |
49054 | 206 |
val distinctN = "distinct"; |
49075 | 207 |
val exhaustN = "exhaust"; |
49486 | 208 |
val expandN = "expand"; |
49075 | 209 |
val injectN = "inject"; |
210 |
val nchotomyN = "nchotomy"; |
|
53694 | 211 |
val selN = "sel"; |
53916 | 212 |
val sel_exhaustN = "sel_exhaust"; |
53917 | 213 |
val sel_splitN = "sel_split"; |
214 |
val sel_split_asmN = "sel_split_asm"; |
|
49054 | 215 |
val splitN = "split"; |
49633 | 216 |
val splitsN = "splits"; |
49054 | 217 |
val split_asmN = "split_asm"; |
218 |
val weak_case_cong_thmsN = "weak_case_cong"; |
|
49019 | 219 |
|
53700 | 220 |
val cong_attrs = @{attributes [cong]}; |
53836 | 221 |
val dest_attrs = @{attributes [dest]}; |
53700 | 222 |
val safe_elim_attrs = @{attributes [elim!]}; |
223 |
val iff_attrs = @{attributes [iff]}; |
|
54145
297d1c603999
make sure that registered code equations are actually equations
blanchet
parents:
54008
diff
changeset
|
224 |
val inductsimp_attrs = @{attributes [induct_simp]}; |
297d1c603999
make sure that registered code equations are actually equations
blanchet
parents:
54008
diff
changeset
|
225 |
val nitpicksimp_attrs = @{attributes [nitpick_simp]}; |
49300 | 226 |
val simp_attrs = @{attributes [simp]}; |
54151 | 227 |
val code_nitpicksimp_attrs = Code.add_default_eqn_attrib :: nitpicksimp_attrs; |
228 |
val code_nitpicksimp_simp_attrs = code_nitpicksimp_attrs @ simp_attrs; |
|
49046
3c5eba97d93a
allow default names for selectors via wildcard (_) + fix wrong index (k)
blanchet
parents:
49045
diff
changeset
|
229 |
|
55480
59cc4a8bc28a
allow different functions to recurse on the same type, like in the old package
blanchet
parents:
55471
diff
changeset
|
230 |
fun unflat_lookup eq xs ys = map (fn xs' => permute_like_unique eq xs xs' ys); |
49258
84f13469d7f0
allow same selector name for several constructors
blanchet
parents:
49257
diff
changeset
|
231 |
|
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
232 |
fun mk_half_pairss' _ ([], []) = [] |
49591
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
233 |
| mk_half_pairss' indent (x :: xs, _ :: ys) = |
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
234 |
indent @ fold_rev (cons o single o pair x) ys (mk_half_pairss' ([] :: indent) (xs, ys)); |
49486 | 235 |
|
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
236 |
fun mk_half_pairss p = mk_half_pairss' [[]] p; |
49027 | 237 |
|
49486 | 238 |
fun join_halves n half_xss other_half_xss = |
55342 | 239 |
(splice (flat half_xss) (flat other_half_xss), |
240 |
map2 (map2 append) (Library.chop_groups n half_xss) |
|
241 |
(transpose (Library.chop_groups n other_half_xss))); |
|
49027 | 242 |
|
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
243 |
fun mk_undefined T = Const (@{const_name undefined}, T); |
49055 | 244 |
|
49500 | 245 |
fun mk_ctr Ts t = |
246 |
let val Type (_, Ts0) = body_type (fastype_of t) in |
|
54435
4a655e62ad34
fixed type variable confusion in 'datatype_new_compat'
blanchet
parents:
54422
diff
changeset
|
247 |
subst_nonatomic_types (Ts0 ~~ Ts) t |
49203 | 248 |
end; |
249 |
||
49536 | 250 |
fun mk_case Ts T t = |
251 |
let val (Type (_, Ts0), body) = strip_type (fastype_of t) |>> List.last in |
|
54435
4a655e62ad34
fixed type variable confusion in 'datatype_new_compat'
blanchet
parents:
54422
diff
changeset
|
252 |
subst_nonatomic_types ((body, T) :: (Ts0 ~~ Ts)) t |
49536 | 253 |
end; |
254 |
||
53864
a48d4bd3faaa
use case rather than sequence of ifs in expansion
blanchet
parents:
53857
diff
changeset
|
255 |
fun mk_disc_or_sel Ts t = |
54435
4a655e62ad34
fixed type variable confusion in 'datatype_new_compat'
blanchet
parents:
54422
diff
changeset
|
256 |
subst_nonatomic_types (snd (Term.dest_Type (domain_type (fastype_of t))) ~~ Ts) t; |
53864
a48d4bd3faaa
use case rather than sequence of ifs in expansion
blanchet
parents:
53857
diff
changeset
|
257 |
|
51777
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
258 |
val name_of_ctr = name_of_const "constructor"; |
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
259 |
|
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
260 |
fun name_of_disc t = |
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
261 |
(case head_of t of |
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
262 |
Abs (_, _, @{const Not} $ (t' $ Bound 0)) => |
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
263 |
Long_Name.map_base_name (prefix notN) (name_of_disc t') |
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
264 |
| Abs (_, _, Const (@{const_name HOL.eq}, _) $ Bound 0 $ t') => |
57260
8747af0d1012
fixed postprocessing of 'coinduct' formula to obtain right property format (without needless hypotheses)
blanchet
parents:
57200
diff
changeset
|
265 |
Long_Name.map_base_name (prefix isN) (name_of_disc t') |
51777
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
266 |
| Abs (_, _, @{const Not} $ (Const (@{const_name HOL.eq}, _) $ Bound 0 $ t')) => |
57260
8747af0d1012
fixed postprocessing of 'coinduct' formula to obtain right property format (without needless hypotheses)
blanchet
parents:
57200
diff
changeset
|
267 |
Long_Name.map_base_name (prefix (notN ^ isN)) (name_of_disc t') |
51777
48a0ae342ea0
generate proper attributes for coinduction rules
blanchet
parents:
51771
diff
changeset
|
268 |
| t' => name_of_const "destructor" t'); |
49622 | 269 |
|
270 |
val base_name_of_ctr = Long_Name.base_name o name_of_ctr; |
|
49046
3c5eba97d93a
allow default names for selectors via wildcard (_) + fix wrong index (k)
blanchet
parents:
49045
diff
changeset
|
271 |
|
53888 | 272 |
fun dest_ctr ctxt s t = |
55342 | 273 |
let val (f, args) = Term.strip_comb t in |
53888 | 274 |
(case ctr_sugar_of ctxt s of |
275 |
SOME {ctrs, ...} => |
|
276 |
(case find_first (can (fo_match ctxt f)) ctrs of |
|
277 |
SOME f' => (f', args) |
|
278 |
| NONE => raise Fail "dest_ctr") |
|
279 |
| NONE => raise Fail "dest_ctr") |
|
280 |
end; |
|
281 |
||
53870 | 282 |
fun dest_case ctxt s Ts t = |
283 |
(case Term.strip_comb t of |
|
284 |
(Const (c, _), args as _ :: _) => |
|
285 |
(case ctr_sugar_of ctxt s of |
|
54970
891141de5672
only destruct cases equipped with the right stuff (in particular, 'sel_split')
blanchet
parents:
54900
diff
changeset
|
286 |
SOME (ctr_sugar as {casex = Const (case_name, _), discs = discs0, selss = selss0, ...}) => |
53870 | 287 |
if case_name = c then |
53924 | 288 |
let val n = length discs0 in |
289 |
if n < length args then |
|
290 |
let |
|
291 |
val (branches, obj :: leftovers) = chop n args; |
|
292 |
val discs = map (mk_disc_or_sel Ts) discs0; |
|
293 |
val selss = map (map (mk_disc_or_sel Ts)) selss0; |
|
294 |
val conds = map (rapp obj) discs; |
|
295 |
val branch_argss = map (fn sels => map (rapp obj) sels @ leftovers) selss; |
|
296 |
val branches' = map2 (curry Term.betapplys) branches branch_argss; |
|
297 |
in |
|
54970
891141de5672
only destruct cases equipped with the right stuff (in particular, 'sel_split')
blanchet
parents:
54900
diff
changeset
|
298 |
SOME (ctr_sugar, conds, branches') |
53924 | 299 |
end |
300 |
else |
|
301 |
NONE |
|
53870 | 302 |
end |
303 |
else |
|
304 |
NONE |
|
305 |
| _ => NONE) |
|
306 |
| _ => NONE); |
|
307 |
||
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
308 |
fun const_or_free_name (Const (s, _)) = Long_Name.base_name s |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
309 |
| const_or_free_name (Free (s, _)) = s |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
310 |
| const_or_free_name t = raise TERM ("const_or_free_name", [t]) |
49437 | 311 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
312 |
fun extract_sel_default ctxt t = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
313 |
let |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
314 |
fun malformed () = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
315 |
error ("Malformed selector default value equation: " ^ Syntax.string_of_term ctxt t); |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
316 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
317 |
val ((sel, (ctr, vars)), rhs) = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
318 |
fst (Term.replace_dummy_patterns (Syntax.check_term ctxt t) 0) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
319 |
|> HOLogic.dest_eq |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
320 |
|>> (Term.dest_comb |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
321 |
#>> const_or_free_name |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
322 |
##> (Term.strip_comb #>> (Term.dest_Const #> fst))) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
323 |
handle TERM _ => malformed (); |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
324 |
in |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
325 |
if forall (is_Free orf is_Var) vars andalso not (has_duplicates (op aconv) vars) then |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
326 |
((ctr, sel), fold_rev Term.lambda vars rhs) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
327 |
else |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
328 |
malformed () |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
329 |
end; |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
330 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
331 |
type ('c, 'a) ctr_spec = (binding * 'c) * 'a list; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
332 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
333 |
fun disc_of_ctr_spec ((disc, _), _) = disc; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
334 |
fun ctr_of_ctr_spec ((_, ctr), _) = ctr; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
335 |
fun args_of_ctr_spec (_, args) = args; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
336 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
337 |
fun prepare_free_constructors prep_term |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
338 |
((((discs_sels, no_code), raw_case_binding), ctr_specs), sel_default_eqs) no_defs_lthy = |
49017 | 339 |
let |
49019 | 340 |
(* TODO: sanity checks on arguments *) |
49025 | 341 |
|
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
342 |
val raw_ctrs = map ctr_of_ctr_spec ctr_specs; |
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
343 |
val raw_disc_bindings = map disc_of_ctr_spec ctr_specs; |
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
344 |
val raw_sel_bindingss = map args_of_ctr_spec ctr_specs; |
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
345 |
|
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
346 |
val n = length raw_ctrs; |
49054 | 347 |
val ks = 1 upto n; |
348 |
||
49121 | 349 |
val _ = if n > 0 then () else error "No constructors specified"; |
350 |
||
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
351 |
val ctrs0 = map (prep_term no_defs_lthy) raw_ctrs; |
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
352 |
|
53908 | 353 |
val Type (fcT_name, As0) = body_type (fastype_of (hd ctrs0)); |
354 |
val fc_b_name = Long_Name.base_name fcT_name; |
|
355 |
val fc_b = Binding.name fc_b_name; |
|
49055 | 356 |
|
55410 | 357 |
fun qualify mandatory = Binding.qualify mandatory fc_b_name; |
49633 | 358 |
|
54386 | 359 |
fun dest_TFree_or_TVar (TFree sS) = sS |
53268
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
360 |
| dest_TFree_or_TVar (TVar ((s, _), S)) = (s, S) |
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
361 |
| dest_TFree_or_TVar _ = error "Invalid type argument"; |
52965
0cd62cb233e0
handle both TVars and TFrees -- necessary for 'wrap_free_constructors'
blanchet
parents:
52963
diff
changeset
|
362 |
|
53268
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
363 |
val (unsorted_As, B) = |
49055 | 364 |
no_defs_lthy |
53268
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
365 |
|> variant_tfrees (map (fst o dest_TFree_or_TVar) As0) |
49055 | 366 |
||> the_single o fst o mk_TFrees 1; |
367 |
||
53268
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
368 |
val As = map2 (resort_tfree o snd o dest_TFree_or_TVar) As0 unsorted_As; |
de1dc709f9d4
handle type class annotations on (co)datatype parameters gracefully
blanchet
parents:
53210
diff
changeset
|
369 |
|
53908 | 370 |
val fcT = Type (fcT_name, As); |
49055 | 371 |
val ctrs = map (mk_ctr As) ctrs0; |
372 |
val ctr_Tss = map (binder_types o fastype_of) ctrs; |
|
373 |
||
374 |
val ms = map length ctr_Tss; |
|
375 |
||
57091 | 376 |
fun can_definitely_rely_on_disc k = |
377 |
not (Binding.is_empty (nth raw_disc_bindings (k - 1))) orelse nth ms (k - 1) = 0; |
|
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
378 |
fun can_rely_on_disc k = |
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
379 |
can_definitely_rely_on_disc k orelse (k = 1 andalso not (can_definitely_rely_on_disc 2)); |
53925 | 380 |
fun should_omit_disc_binding k = n = 1 orelse (n = 2 andalso can_rely_on_disc (3 - k)); |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
381 |
|
57090
0224caba67ca
use '%x. x = C' as default discriminator for nullary constructor C, instead of relying on odd '=:' syntax
blanchet
parents:
57038
diff
changeset
|
382 |
val equal_binding = @{binding "="}; |
0224caba67ca
use '%x. x = C' as default discriminator for nullary constructor C, instead of relying on odd '=:' syntax
blanchet
parents:
57038
diff
changeset
|
383 |
|
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
384 |
fun is_disc_binding_valid b = |
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
385 |
not (Binding.is_empty b orelse Binding.eq_name (b, equal_binding)); |
51787
1267c28c7bdd
changed discriminator default: avoid mixing ctor and dtor views
blanchet
parents:
51781
diff
changeset
|
386 |
|
52322 | 387 |
val standard_disc_binding = Binding.name o prefix isN o base_name_of_ctr; |
49120
7f8e69fc6ac9
smarter "*" syntax -- fallback on "_" if "*" is impossible
blanchet
parents:
49119
diff
changeset
|
388 |
|
49336 | 389 |
val disc_bindings = |
55470
46e6e1d91056
removed needless robustness (no longer needed thanks to new syntax)
blanchet
parents:
55469
diff
changeset
|
390 |
raw_disc_bindings |
49120
7f8e69fc6ac9
smarter "*" syntax -- fallback on "_" if "*" is impossible
blanchet
parents:
49119
diff
changeset
|
391 |
|> map4 (fn k => fn m => fn ctr => fn disc => |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
392 |
qualify false |
51787
1267c28c7bdd
changed discriminator default: avoid mixing ctor and dtor views
blanchet
parents:
51781
diff
changeset
|
393 |
(if Binding.is_empty disc then |
57091 | 394 |
if m = 0 then equal_binding |
395 |
else if should_omit_disc_binding k then disc |
|
57090
0224caba67ca
use '%x. x = C' as default discriminator for nullary constructor C, instead of relying on odd '=:' syntax
blanchet
parents:
57038
diff
changeset
|
396 |
else standard_disc_binding ctr |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
397 |
else if Binding.eq_name (disc, standard_binding) then |
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
398 |
standard_disc_binding ctr |
49302
f5bd87aac224
added optional qualifiers for constructors and destructors, similarly to the old package
blanchet
parents:
49300
diff
changeset
|
399 |
else |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
400 |
disc)) ks ms ctrs0; |
49056 | 401 |
|
51787
1267c28c7bdd
changed discriminator default: avoid mixing ctor and dtor views
blanchet
parents:
51781
diff
changeset
|
402 |
fun standard_sel_binding m l = Binding.name o mk_unN m l o base_name_of_ctr; |
49120
7f8e69fc6ac9
smarter "*" syntax -- fallback on "_" if "*" is impossible
blanchet
parents:
49119
diff
changeset
|
403 |
|
49336 | 404 |
val sel_bindingss = |
55470
46e6e1d91056
removed needless robustness (no longer needed thanks to new syntax)
blanchet
parents:
55469
diff
changeset
|
405 |
map3 (fn ctr => fn m => map2 (fn l => fn sel => |
49633 | 406 |
qualify false |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
407 |
(if Binding.is_empty sel orelse Binding.eq_name (sel, standard_binding) then |
51787
1267c28c7bdd
changed discriminator default: avoid mixing ctor and dtor views
blanchet
parents:
51781
diff
changeset
|
408 |
standard_sel_binding m l ctr |
49302
f5bd87aac224
added optional qualifiers for constructors and destructors, similarly to the old package
blanchet
parents:
49300
diff
changeset
|
409 |
else |
55470
46e6e1d91056
removed needless robustness (no longer needed thanks to new syntax)
blanchet
parents:
55469
diff
changeset
|
410 |
sel)) (1 upto m) o pad_list Binding.empty m) ctrs0 ms raw_sel_bindingss; |
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
411 |
|
49201 | 412 |
val case_Ts = map (fn Ts => Ts ---> B) ctr_Tss; |
49043 | 413 |
|
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
414 |
val (((((((([exh_y], (xss, xss')), yss), fs), gs), [u', v']), [w]), (p, p')), names_lthy) = |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
415 |
no_defs_lthy |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
416 |
|> mk_Frees "y" [fcT] (* for compatibility with "datatype_realizer.ML" *) |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
417 |
||>> mk_Freess' "x" ctr_Tss |
49025 | 418 |
||>> mk_Freess "y" ctr_Tss |
49201 | 419 |
||>> mk_Frees "f" case_Ts |
420 |
||>> mk_Frees "g" case_Ts |
|
53908 | 421 |
||>> (apfst (map (rpair fcT)) oo Variable.variant_fixes) [fc_b_name, fc_b_name ^ "'"] |
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
422 |
||>> mk_Frees "z" [B] |
49043 | 423 |
||>> yield_singleton (apfst (op ~~) oo mk_Frees' "P") HOLogic.boolT; |
424 |
||
49498 | 425 |
val u = Free u'; |
426 |
val v = Free v'; |
|
49463 | 427 |
val q = Free (fst p', mk_pred1T B); |
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
428 |
|
49025 | 429 |
val xctrs = map2 (curry Term.list_comb) ctrs xss; |
430 |
val yctrs = map2 (curry Term.list_comb) ctrs yss; |
|
49032 | 431 |
|
49043 | 432 |
val xfs = map2 (curry Term.list_comb) fs xss; |
433 |
val xgs = map2 (curry Term.list_comb) gs xss; |
|
434 |
||
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
435 |
(* TODO: Eta-expension is for compatibility with the old datatype package (but it also provides |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
436 |
nicer names). Consider removing. *) |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
437 |
val eta_fs = map2 (fold_rev Term.lambda) xss xfs; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
438 |
val eta_gs = map2 (fold_rev Term.lambda) xss xgs; |
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
439 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
440 |
val case_binding = |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
441 |
qualify false |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
442 |
(if Binding.is_empty raw_case_binding orelse |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
443 |
Binding.eq_name (raw_case_binding, standard_binding) then |
54493
5b34a5b93ec2
use type suffixes instead of prefixes for 'case', '(un)fold', '(co)rec'
blanchet
parents:
54491
diff
changeset
|
444 |
Binding.prefix_name (caseN ^ "_") fc_b |
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
445 |
else |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
446 |
raw_case_binding); |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
447 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
448 |
fun mk_case_disj xctr xf xs = |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
449 |
list_exists_free xs (HOLogic.mk_conj (HOLogic.mk_eq (u, xctr), HOLogic.mk_eq (w, xf))); |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
450 |
|
53925 | 451 |
val case_rhs = fold_rev (fold_rev Term.lambda) [fs, [u]] |
452 |
(Const (@{const_name The}, (B --> HOLogic.boolT) --> B) $ |
|
453 |
Term.lambda w (Library.foldr1 HOLogic.mk_disj (map3 mk_case_disj xctrs xfs xss))); |
|
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
454 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
455 |
val ((raw_case, (_, raw_case_def)), (lthy', lthy)) = no_defs_lthy |
54155 | 456 |
|> Local_Theory.define ((case_binding, NoSyn), |
457 |
((Binding.conceal (Thm.def_binding case_binding), []), case_rhs)) |
|
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
458 |
||> `Local_Theory.restore; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
459 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
460 |
val phi = Proof_Context.export_morphism lthy lthy'; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
461 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
462 |
val case_def = Morphism.thm phi raw_case_def; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
463 |
|
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
464 |
val case0 = Morphism.term phi raw_case; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
465 |
val casex = mk_case As B case0; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
466 |
|
51759
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
467 |
val fcase = Term.list_comb (casex, fs); |
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
468 |
|
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
469 |
val ufcase = fcase $ u; |
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
470 |
val vfcase = fcase $ v; |
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
471 |
|
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
472 |
val eta_fcase = Term.list_comb (casex, eta_fs); |
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
473 |
val eta_gcase = Term.list_comb (casex, eta_gs); |
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
474 |
|
51759
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
475 |
val eta_ufcase = eta_fcase $ u; |
587bba425430
eta-contracted weak congruence rules (like in the old package)
blanchet
parents:
51757
diff
changeset
|
476 |
val eta_vgcase = eta_gcase $ v; |
49486 | 477 |
|
49591
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
478 |
fun mk_uu_eq () = HOLogic.mk_eq (u, u); |
49486 | 479 |
|
49591
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
480 |
val uv_eq = mk_Trueprop_eq (u, v); |
49486 | 481 |
|
482 |
val exist_xs_u_eq_ctrs = |
|
483 |
map2 (fn xctr => fn xs => list_exists_free xs (HOLogic.mk_eq (u, xctr))) xctrs xss; |
|
49022 | 484 |
|
51743 | 485 |
val unique_disc_no_def = TrueI; (*arbitrary marker*) |
486 |
val alternate_disc_no_def = FalseE; (*arbitrary marker*) |
|
487 |
||
49486 | 488 |
fun alternate_disc_lhs get_udisc k = |
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
489 |
HOLogic.mk_not |
51790
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
490 |
(let val b = nth disc_bindings (k - 1) in |
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
491 |
if is_disc_binding_valid b then get_udisc b (k - 1) else nth exist_xs_u_eq_ctrs (k - 1) |
22517d04d20b
more intuitive syntax for equality-style discriminators of nullary constructors
blanchet
parents:
51787
diff
changeset
|
492 |
end); |
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
493 |
|
57094
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57091
diff
changeset
|
494 |
val no_discs_sels = |
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57091
diff
changeset
|
495 |
not discs_sels andalso |
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57091
diff
changeset
|
496 |
forall (forall Binding.is_empty) (raw_disc_bindings :: raw_sel_bindingss) andalso |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
497 |
null sel_default_eqs; |
57094
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57091
diff
changeset
|
498 |
|
53917 | 499 |
val (all_sels_distinct, discs, selss, disc_defs, sel_defs, sel_defss, lthy') = |
52969
f2df0730f8ac
clarified option name (since case/fold/rec are also destructors)
blanchet
parents:
52968
diff
changeset
|
500 |
if no_discs_sels then |
55407
81f7e60755c3
use right local theory -- shows up when 'no_discs_sels' is set
blanchet
parents:
55394
diff
changeset
|
501 |
(true, [], [], [], [], [], lthy') |
49278 | 502 |
else |
503 |
let |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
504 |
val sel_bindings = flat sel_bindingss; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
505 |
val uniq_sel_bindings = distinct Binding.eq_name sel_bindings; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
506 |
val all_sels_distinct = (length uniq_sel_bindings = length sel_bindings); |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
507 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
508 |
val sel_binding_index = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
509 |
if all_sels_distinct then 1 upto length sel_bindings |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
510 |
else map (fn b => find_index (curry Binding.eq_name b) uniq_sel_bindings) sel_bindings; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
511 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
512 |
val all_proto_sels = flat (map3 (fn k => fn xs => map (fn x => (k, (xs, x)))) ks xss xss); |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
513 |
val sel_infos = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
514 |
AList.group (op =) (sel_binding_index ~~ all_proto_sels) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
515 |
|> sort (int_ord o pairself fst) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
516 |
|> map snd |> curry (op ~~) uniq_sel_bindings; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
517 |
val sel_bindings = map fst sel_infos; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
518 |
val sel_Ts = map (curry (op -->) fcT o fastype_of o snd o snd o hd o snd) sel_infos; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
519 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
520 |
val sel_default_lthy = no_defs_lthy |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
521 |
|> Proof_Context.allow_dummies |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
522 |
|> Proof_Context.add_fixes |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
523 |
(map2 (fn b => fn T => (b, SOME T, NoSyn)) sel_bindings sel_Ts) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
524 |
|> snd; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
525 |
|
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
526 |
val sel_defaults = |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
527 |
map (extract_sel_default sel_default_lthy o prep_term sel_default_lthy) sel_default_eqs; |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
528 |
|
53908 | 529 |
fun disc_free b = Free (Binding.name_of b, mk_pred1T fcT); |
49025 | 530 |
|
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
531 |
fun disc_spec b exist_xs_u_eq_ctr = mk_Trueprop_eq (disc_free b $ u, exist_xs_u_eq_ctr); |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
532 |
|
49500 | 533 |
fun alternate_disc k = |
534 |
Term.lambda u (alternate_disc_lhs (K o rapp u o disc_free) (3 - k)); |
|
49278 | 535 |
|
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
536 |
fun mk_sel_case_args b proto_sels T = |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
537 |
map3 (fn Const (c, _) => fn Ts => fn k => |
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
538 |
(case AList.lookup (op =) proto_sels k of |
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
539 |
NONE => |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
540 |
(case filter (curry (op =) (c, Binding.name_of b) o fst) sel_defaults of |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
541 |
[] => fold_rev (Term.lambda o curry Free Name.uu) Ts (mk_undefined T) |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
542 |
| [(_, t)] => t |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
543 |
| _ => error "Multiple default values for selector/constructor pair") |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
544 |
| SOME (xs, x) => fold_rev Term.lambda xs x)) ctrs ctr_Tss ks; |
49258
84f13469d7f0
allow same selector name for several constructors
blanchet
parents:
49257
diff
changeset
|
545 |
|
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
546 |
fun sel_spec b proto_sels = |
49278 | 547 |
let |
548 |
val _ = |
|
549 |
(case duplicates (op =) (map fst proto_sels) of |
|
550 |
k :: _ => error ("Duplicate selector name " ^ quote (Binding.name_of b) ^ |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
551 |
" for constructor " ^ quote (Syntax.string_of_term lthy (nth ctrs (k - 1)))) |
49278 | 552 |
| [] => ()) |
553 |
val T = |
|
554 |
(case distinct (op =) (map (fastype_of o snd o snd) proto_sels) of |
|
555 |
[T] => T |
|
556 |
| T :: T' :: _ => error ("Inconsistent range type for selector " ^ |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
557 |
quote (Binding.name_of b) ^ ": " ^ quote (Syntax.string_of_typ lthy T) ^ |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
558 |
" vs. " ^ quote (Syntax.string_of_typ lthy T'))); |
49278 | 559 |
in |
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
560 |
mk_Trueprop_eq (Free (Binding.name_of b, fcT --> T) $ u, |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
561 |
Term.list_comb (mk_case As T case0, mk_sel_case_args b proto_sels T) $ u) |
49278 | 562 |
end; |
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
563 |
|
49336 | 564 |
fun unflat_selss xs = unflat_lookup Binding.eq_name sel_bindings xs sel_bindingss; |
49258
84f13469d7f0
allow same selector name for several constructors
blanchet
parents:
49257
diff
changeset
|
565 |
|
49278 | 566 |
val (((raw_discs, raw_disc_defs), (raw_sels, raw_sel_defs)), (lthy', lthy)) = |
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
567 |
lthy |
51809 | 568 |
|> apfst split_list o fold_map3 (fn k => fn exist_xs_u_eq_ctr => fn b => |
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
569 |
if Binding.is_empty b then |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
570 |
if n = 1 then pair (Term.lambda u (mk_uu_eq ()), unique_disc_no_def) |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
571 |
else pair (alternate_disc k, alternate_disc_no_def) |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
572 |
else if Binding.eq_name (b, equal_binding) then |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
573 |
pair (Term.lambda u exist_xs_u_eq_ctr, refl) |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
574 |
else |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
575 |
Specification.definition (SOME (b, NONE, NoSyn), |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
576 |
((Thm.def_binding b, []), disc_spec b exist_xs_u_eq_ctr)) #>> apsnd snd) |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
577 |
ks exist_xs_u_eq_ctrs disc_bindings |
49278 | 578 |
||>> apfst split_list o fold_map (fn (b, proto_sels) => |
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
579 |
Specification.definition (SOME (b, NONE, NoSyn), |
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
580 |
((Thm.def_binding b, []), sel_spec b proto_sels)) #>> apsnd snd) sel_infos |
49278 | 581 |
||> `Local_Theory.restore; |
49022 | 582 |
|
49278 | 583 |
val phi = Proof_Context.export_morphism lthy lthy'; |
49025 | 584 |
|
49278 | 585 |
val disc_defs = map (Morphism.thm phi) raw_disc_defs; |
49281 | 586 |
val sel_defs = map (Morphism.thm phi) raw_sel_defs; |
587 |
val sel_defss = unflat_selss sel_defs; |
|
49278 | 588 |
|
589 |
val discs0 = map (Morphism.term phi) raw_discs; |
|
590 |
val selss0 = unflat_selss (map (Morphism.term phi) raw_sels); |
|
49028 | 591 |
|
49278 | 592 |
val discs = map (mk_disc_or_sel As) discs0; |
593 |
val selss = map (map (mk_disc_or_sel As)) selss0; |
|
594 |
in |
|
53917 | 595 |
(all_sels_distinct, discs, selss, disc_defs, sel_defs, sel_defss, lthy') |
49278 | 596 |
end; |
49025 | 597 |
|
49032 | 598 |
fun mk_imp_p Qs = Logic.list_implies (Qs, HOLogic.mk_Trueprop p); |
49029 | 599 |
|
49458 | 600 |
val exhaust_goal = |
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
601 |
let fun mk_prem xctr xs = fold_rev Logic.all xs (mk_imp_p [mk_Trueprop_eq (exh_y, xctr)]) in |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
602 |
fold_rev Logic.all [p, exh_y] (mk_imp_p (map2 mk_prem xctrs xss)) |
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
603 |
end; |
49019 | 604 |
|
49484 | 605 |
val inject_goalss = |
49017 | 606 |
let |
49034
b77e1910af8a
make parallel list indexing possible for inject theorems
blanchet
parents:
49033
diff
changeset
|
607 |
fun mk_goal _ _ [] [] = [] |
49025 | 608 |
| mk_goal xctr yctr xs ys = |
49121 | 609 |
[fold_rev Logic.all (xs @ ys) (mk_Trueprop_eq (HOLogic.mk_eq (xctr, yctr), |
610 |
Library.foldr1 HOLogic.mk_conj (map2 (curry HOLogic.mk_eq) xs ys)))]; |
|
49017 | 611 |
in |
49034
b77e1910af8a
make parallel list indexing possible for inject theorems
blanchet
parents:
49033
diff
changeset
|
612 |
map4 mk_goal xctrs yctrs xss yss |
49017 | 613 |
end; |
614 |
||
49484 | 615 |
val half_distinct_goalss = |
49121 | 616 |
let |
49203 | 617 |
fun mk_goal ((xs, xc), (xs', xc')) = |
49121 | 618 |
fold_rev Logic.all (xs @ xs') |
49203 | 619 |
(HOLogic.mk_Trueprop (HOLogic.mk_not (HOLogic.mk_eq (xc, xc')))); |
49121 | 620 |
in |
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
621 |
map (map mk_goal) (mk_half_pairss (`I (xss ~~ xctrs))) |
49121 | 622 |
end; |
49019 | 623 |
|
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
624 |
val goalss = [exhaust_goal] :: inject_goalss @ half_distinct_goalss; |
49019 | 625 |
|
57633 | 626 |
fun after_qed ([exhaust_thm] :: thmss) lthy = |
49019 | 627 |
let |
57633 | 628 |
val ((inject_thms, inject_thmss), half_distinct_thmss) = chop n thmss |>> `flat; |
49438 | 629 |
|
53210
7219c61796c0
simplify code (now that ctr_sugar uses the same type variables as fp_sugar)
blanchet
parents:
53040
diff
changeset
|
630 |
val rho_As = map (pairself (certifyT lthy)) (map Logic.varifyT_global As ~~ As); |
49486 | 631 |
|
632 |
fun inst_thm t thm = |
|
633 |
Drule.instantiate' [] [SOME (certify lthy t)] |
|
53210
7219c61796c0
simplify code (now that ctr_sugar uses the same type variables as fp_sugar)
blanchet
parents:
53040
diff
changeset
|
634 |
(Thm.instantiate (rho_As, []) (Drule.zero_var_indexes thm)); |
49486 | 635 |
|
636 |
val uexhaust_thm = inst_thm u exhaust_thm; |
|
49032 | 637 |
|
49300 | 638 |
val exhaust_cases = map base_name_of_ctr ctrs; |
639 |
||
49048
4e0f0f98be02
rationalized data structure for distinctness theorems
blanchet
parents:
49046
diff
changeset
|
640 |
val other_half_distinct_thmss = map (map (fn thm => thm RS not_sym)) half_distinct_thmss; |
4e0f0f98be02
rationalized data structure for distinctness theorems
blanchet
parents:
49046
diff
changeset
|
641 |
|
49486 | 642 |
val (distinct_thms, (distinct_thmsss', distinct_thmsss)) = |
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
643 |
join_halves n half_distinct_thmss other_half_distinct_thmss ||> `transpose; |
49019 | 644 |
|
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
645 |
val nchotomy_thm = |
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
646 |
let |
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
647 |
val goal = |
49486 | 648 |
HOLogic.mk_Trueprop (HOLogic.mk_all (fst u', snd u', |
649 |
Library.foldr1 HOLogic.mk_disj exist_xs_u_eq_ctrs)); |
|
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
650 |
in |
51551 | 651 |
Goal.prove_sorry lthy [] [] goal (fn _ => mk_nchotomy_tac n exhaust_thm) |
49667
44d85dc8ca08
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel
parents:
49633
diff
changeset
|
652 |
|> Thm.close_derivation |
49020
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
653 |
end; |
f379cf5d71bd
more work on BNF sugar -- up to derivation of nchotomy
blanchet
parents:
49019
diff
changeset
|
654 |
|
52968
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
655 |
val case_thms = |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
656 |
let |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
657 |
val goals = |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
658 |
map3 (fn xctr => fn xf => fn xs => |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
659 |
fold_rev Logic.all (fs @ xs) (mk_Trueprop_eq (fcase $ xctr, xf))) xctrs xfs xss; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
660 |
in |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
661 |
map4 (fn k => fn goal => fn injects => fn distinctss => |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
662 |
Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, ...} => |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
663 |
mk_case_tac ctxt n k case_def injects distinctss) |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
664 |
|> Thm.close_derivation) |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
665 |
ks goals inject_thmss distinct_thmsss |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
666 |
end; |
2b430bbb5a1a
define case constant from other 'free constructor' axioms
blanchet
parents:
52965
diff
changeset
|
667 |
|
53917 | 668 |
val (case_cong_thm, weak_case_cong_thm) = |
669 |
let |
|
670 |
fun mk_prem xctr xs xf xg = |
|
671 |
fold_rev Logic.all xs (Logic.mk_implies (mk_Trueprop_eq (v, xctr), |
|
672 |
mk_Trueprop_eq (xf, xg))); |
|
673 |
||
674 |
val goal = |
|
675 |
Logic.list_implies (uv_eq :: map4 mk_prem xctrs xss xfs xgs, |
|
676 |
mk_Trueprop_eq (eta_ufcase, eta_vgcase)); |
|
677 |
val weak_goal = Logic.mk_implies (uv_eq, mk_Trueprop_eq (ufcase, vfcase)); |
|
678 |
in |
|
679 |
(Goal.prove_sorry lthy [] [] goal (fn _ => mk_case_cong_tac lthy uexhaust_thm case_thms), |
|
680 |
Goal.prove_sorry lthy [] [] weak_goal (K (etac arg_cong 1))) |
|
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
681 |
|> pairself (singleton (Proof_Context.export names_lthy lthy) #> |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
682 |
Thm.close_derivation) |
53917 | 683 |
end; |
684 |
||
685 |
val split_lhs = q $ ufcase; |
|
686 |
||
687 |
fun mk_split_conjunct xctr xs f_xs = |
|
688 |
list_all_free xs (HOLogic.mk_imp (HOLogic.mk_eq (u, xctr), q $ f_xs)); |
|
689 |
fun mk_split_disjunct xctr xs f_xs = |
|
690 |
list_exists_free xs (HOLogic.mk_conj (HOLogic.mk_eq (u, xctr), |
|
691 |
HOLogic.mk_not (q $ f_xs))); |
|
692 |
||
693 |
fun mk_split_goal xctrs xss xfs = |
|
694 |
mk_Trueprop_eq (split_lhs, Library.foldr1 HOLogic.mk_conj |
|
695 |
(map3 mk_split_conjunct xctrs xss xfs)); |
|
696 |
fun mk_split_asm_goal xctrs xss xfs = |
|
697 |
mk_Trueprop_eq (split_lhs, HOLogic.mk_not (Library.foldr1 HOLogic.mk_disj |
|
698 |
(map3 mk_split_disjunct xctrs xss xfs))); |
|
699 |
||
700 |
fun prove_split selss goal = |
|
701 |
Goal.prove_sorry lthy [] [] goal (fn _ => |
|
702 |
mk_split_tac lthy uexhaust_thm case_thms selss inject_thmss distinct_thmsss) |
|
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
703 |
|> singleton (Proof_Context.export names_lthy lthy) |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
704 |
|> Thm.close_derivation; |
53917 | 705 |
|
706 |
fun prove_split_asm asm_goal split_thm = |
|
707 |
Goal.prove_sorry lthy [] [] asm_goal (fn {context = ctxt, ...} => |
|
708 |
mk_split_asm_tac ctxt split_thm) |
|
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
709 |
|> singleton (Proof_Context.export names_lthy lthy) |
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
710 |
|> Thm.close_derivation; |
53917 | 711 |
|
712 |
val (split_thm, split_asm_thm) = |
|
713 |
let |
|
714 |
val goal = mk_split_goal xctrs xss xfs; |
|
715 |
val asm_goal = mk_split_asm_goal xctrs xss xfs; |
|
716 |
||
717 |
val thm = prove_split (replicate n []) goal; |
|
718 |
val asm_thm = prove_split_asm asm_goal thm; |
|
719 |
in |
|
720 |
(thm, asm_thm) |
|
721 |
end; |
|
722 |
||
56858 | 723 |
val (sel_defs, all_sel_thms, sel_thmss, disc_defs, disc_thmss, nontriv_disc_thmss, |
724 |
discI_thms, nontriv_discI_thms, disc_exclude_thms, disc_exclude_thmsss, |
|
725 |
disc_exhaust_thms, sel_exhaust_thms, all_collapse_thms, safe_collapse_thms, |
|
726 |
expand_thms, sel_split_thms, sel_split_asm_thms, case_eq_if_thms) = |
|
52969
f2df0730f8ac
clarified option name (since case/fold/rec are also destructors)
blanchet
parents:
52968
diff
changeset
|
727 |
if no_discs_sels then |
56858 | 728 |
([], [], [], [], [], [], [], [], [], [], [], [], [], [], [], [], [], []) |
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
729 |
else |
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
730 |
let |
53917 | 731 |
val udiscs = map (rapp u) discs; |
732 |
val uselss = map (map (rapp u)) selss; |
|
733 |
val usel_ctrs = map2 (curry Term.list_comb) ctrs uselss; |
|
734 |
val usel_fs = map2 (curry Term.list_comb) fs uselss; |
|
735 |
||
736 |
val vdiscs = map (rapp v) discs; |
|
737 |
val vselss = map (map (rapp v)) selss; |
|
738 |
||
49364
838b5e8ede73
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
blanchet
parents:
49336
diff
changeset
|
739 |
fun make_sel_thm xs' case_thm sel_def = |
838b5e8ede73
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
blanchet
parents:
49336
diff
changeset
|
740 |
zero_var_indexes (Drule.gen_all (Drule.rename_bvars' (map (SOME o fst) xs') |
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
741 |
(Drule.forall_intr_vars (case_thm RS (sel_def RS trans))))); |
49281 | 742 |
|
53704 | 743 |
val sel_thmss = map3 (map oo make_sel_thm) xss' case_thms sel_defss; |
744 |
||
49281 | 745 |
fun has_undefined_rhs thm = |
746 |
(case snd (HOLogic.dest_eq (HOLogic.dest_Trueprop (prop_of thm))) of |
|
747 |
Const (@{const_name undefined}, _) => true |
|
748 |
| _ => false); |
|
749 |
||
750 |
val all_sel_thms = |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
751 |
(if all_sels_distinct andalso null sel_default_eqs then |
49285
036b833b99aa
removed wrong "transpose" and ensure "sel" theorems are put in the right order (grouped per selector, in the order in which the selectors appear)
blanchet
parents:
49281
diff
changeset
|
752 |
flat sel_thmss |
036b833b99aa
removed wrong "transpose" and ensure "sel" theorems are put in the right order (grouped per selector, in the order in which the selectors appear)
blanchet
parents:
49281
diff
changeset
|
753 |
else |
49364
838b5e8ede73
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
blanchet
parents:
49336
diff
changeset
|
754 |
map_product (fn s => fn (xs', c) => make_sel_thm xs' c s) sel_defs |
838b5e8ede73
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
blanchet
parents:
49336
diff
changeset
|
755 |
(xss' ~~ case_thms)) |
49285
036b833b99aa
removed wrong "transpose" and ensure "sel" theorems are put in the right order (grouped per selector, in the order in which the selectors appear)
blanchet
parents:
49281
diff
changeset
|
756 |
|> filter_out has_undefined_rhs; |
49278 | 757 |
|
758 |
fun mk_unique_disc_def () = |
|
759 |
let |
|
760 |
val m = the_single ms; |
|
49591
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
761 |
val goal = mk_Trueprop_eq (mk_uu_eq (), the_single exist_xs_u_eq_ctrs); |
49278 | 762 |
in |
51551 | 763 |
Goal.prove_sorry lthy [] [] goal (fn _ => mk_unique_disc_def_tac m uexhaust_thm) |
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
764 |
|> singleton (Proof_Context.export names_lthy lthy) |
49692 | 765 |
|> Thm.close_derivation |
49278 | 766 |
end; |
767 |
||
768 |
fun mk_alternate_disc_def k = |
|
769 |
let |
|
770 |
val goal = |
|
49486 | 771 |
mk_Trueprop_eq (alternate_disc_lhs (K (nth udiscs)) (3 - k), |
772 |
nth exist_xs_u_eq_ctrs (k - 1)); |
|
49278 | 773 |
in |
51551 | 774 |
Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, ...} => |
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
775 |
mk_alternate_disc_def_tac ctxt k (nth disc_defs (2 - k)) |
49486 | 776 |
(nth distinct_thms (2 - k)) uexhaust_thm) |
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
777 |
|> singleton (Proof_Context.export names_lthy lthy) |
49692 | 778 |
|> Thm.close_derivation |
49278 | 779 |
end; |
49028 | 780 |
|
49278 | 781 |
val has_alternate_disc_def = |
782 |
exists (fn def => Thm.eq_thm_prop (def, alternate_disc_no_def)) disc_defs; |
|
783 |
||
784 |
val disc_defs' = |
|
785 |
map2 (fn k => fn def => |
|
786 |
if Thm.eq_thm_prop (def, unique_disc_no_def) then mk_unique_disc_def () |
|
787 |
else if Thm.eq_thm_prop (def, alternate_disc_no_def) then mk_alternate_disc_def k |
|
54634
366297517091
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
blanchet
parents:
54626
diff
changeset
|
788 |
else def) ks disc_defs; |
49278 | 789 |
|
790 |
val discD_thms = map (fn def => def RS iffD1) disc_defs'; |
|
791 |
val discI_thms = |
|
792 |
map2 (fn m => fn def => funpow m (fn thm => exI RS thm) (def RS iffD2)) ms |
|
793 |
disc_defs'; |
|
794 |
val not_discI_thms = |
|
795 |
map2 (fn m => fn def => funpow m (fn thm => allI RS thm) |
|
49504
df9b897fb254
renamed "iter"/"coiter" to "fold"/"unfold" (cf. Wadler)
blanchet
parents:
49500
diff
changeset
|
796 |
(unfold_thms lthy @{thms not_ex} (def RS @{thm ssubst[of _ _ Not]}))) |
49278 | 797 |
ms disc_defs'; |
798 |
||
799 |
val (disc_thmss', disc_thmss) = |
|
800 |
let |
|
801 |
fun mk_thm discI _ [] = refl RS discI |
|
802 |
| mk_thm _ not_discI [distinct] = distinct RS not_discI; |
|
803 |
fun mk_thms discI not_discI distinctss = map (mk_thm discI not_discI) distinctss; |
|
804 |
in |
|
805 |
map3 mk_thms discI_thms not_discI_thms distinct_thmsss' |> `transpose |
|
806 |
end; |
|
807 |
||
55464 | 808 |
val nontriv_disc_thmss = |
809 |
map2 (fn b => if is_disc_binding_valid b then I else K []) disc_bindings disc_thmss; |
|
53704 | 810 |
|
811 |
fun is_discI_boring b = |
|
812 |
(n = 1 andalso Binding.is_empty b) orelse Binding.eq_name (b, equal_binding); |
|
813 |
||
814 |
val nontriv_discI_thms = |
|
815 |
flat (map2 (fn b => if is_discI_boring b then K [] else single) disc_bindings |
|
816 |
discI_thms); |
|
49028 | 817 |
|
49486 | 818 |
val (disc_exclude_thms, (disc_exclude_thmsss', disc_exclude_thmsss)) = |
819 |
let |
|
820 |
fun mk_goal [] = [] |
|
821 |
| mk_goal [((_, udisc), (_, udisc'))] = |
|
822 |
[Logic.all u (Logic.mk_implies (HOLogic.mk_Trueprop udisc, |
|
823 |
HOLogic.mk_Trueprop (HOLogic.mk_not udisc')))]; |
|
824 |
||
49667
44d85dc8ca08
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel
parents:
49633
diff
changeset
|
825 |
fun prove tac goal = |
51551 | 826 |
Goal.prove_sorry lthy [] [] goal (K tac) |
49667
44d85dc8ca08
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel
parents:
49633
diff
changeset
|
827 |
|> Thm.close_derivation; |
49486 | 828 |
|
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
829 |
val half_pairss = mk_half_pairss (`I (ms ~~ discD_thms ~~ udiscs)); |
49486 | 830 |
|
831 |
val half_goalss = map mk_goal half_pairss; |
|
832 |
val half_thmss = |
|
833 |
map3 (fn [] => K (K []) | [goal] => fn [(((m, discD), _), _)] => |
|
51798 | 834 |
fn disc_thm => [prove (mk_half_disc_exclude_tac lthy m discD disc_thm) goal]) |
49486 | 835 |
half_goalss half_pairss (flat disc_thmss'); |
49278 | 836 |
|
49486 | 837 |
val other_half_goalss = map (mk_goal o map swap) half_pairss; |
838 |
val other_half_thmss = |
|
839 |
map2 (map2 (prove o mk_other_half_disc_exclude_tac)) half_thmss |
|
840 |
other_half_goalss; |
|
841 |
in |
|
49585
5c4a12550491
generate high-level "maps", "sets", and "rels" properties
blanchet
parents:
49536
diff
changeset
|
842 |
join_halves n half_thmss other_half_thmss ||> `transpose |
49486 | 843 |
|>> has_alternate_disc_def ? K [] |
844 |
end; |
|
49278 | 845 |
|
49486 | 846 |
val disc_exhaust_thm = |
847 |
let |
|
848 |
fun mk_prem udisc = mk_imp_p [HOLogic.mk_Trueprop udisc]; |
|
849 |
val goal = fold_rev Logic.all [p, u] (mk_imp_p (map mk_prem udiscs)); |
|
850 |
in |
|
51551 | 851 |
Goal.prove_sorry lthy [] [] goal (fn _ => |
49486 | 852 |
mk_disc_exhaust_tac n exhaust_thm discI_thms) |
49667
44d85dc8ca08
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel
parents:
49633
diff
changeset
|
853 |
|> Thm.close_derivation |
49486 | 854 |
end; |
49028 | 855 |
|
53740 | 856 |
val (safe_collapse_thms, all_collapse_thms) = |
49486 | 857 |
let |
54008
b15cfc2864de
refactoring -- splitting between constructor sugar dependencies and true BNF dependencies
blanchet
parents:
54007
diff
changeset
|
858 |
fun mk_goal m udisc usel_ctr = |
49486 | 859 |
let |
860 |
val prem = HOLogic.mk_Trueprop udisc; |
|
53916 | 861 |
val concl = mk_Trueprop_eq ((usel_ctr, u) |> m = 0 ? swap); |
49486 | 862 |
in |
53740 | 863 |
(prem aconv concl, Logic.all u (Logic.mk_implies (prem, concl))) |
49486 | 864 |
end; |
54008
b15cfc2864de
refactoring -- splitting between constructor sugar dependencies and true BNF dependencies
blanchet
parents:
54007
diff
changeset
|
865 |
val (trivs, goals) = map3 mk_goal ms udiscs usel_ctrs |> split_list; |
53740 | 866 |
val thms = |
867 |
map5 (fn m => fn discD => fn sel_thms => fn triv => fn goal => |
|
868 |
Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, ...} => |
|
869 |
mk_collapse_tac ctxt m discD sel_thms ORELSE HEADGOAL atac) |
|
870 |
|> Thm.close_derivation |
|
871 |
|> not triv ? perhaps (try (fn thm => refl RS thm))) |
|
872 |
ms discD_thms sel_thmss trivs goals; |
|
49486 | 873 |
in |
53740 | 874 |
(map_filter (fn (true, _) => NONE | (false, thm) => SOME thm) (trivs ~~ thms), |
875 |
thms) |
|
49486 | 876 |
end; |
49025 | 877 |
|
53916 | 878 |
val swapped_all_collapse_thms = |
879 |
map2 (fn m => fn thm => if m = 0 then thm else thm RS sym) ms all_collapse_thms; |
|
880 |
||
881 |
val sel_exhaust_thm = |
|
882 |
let |
|
883 |
fun mk_prem usel_ctr = mk_imp_p [mk_Trueprop_eq (u, usel_ctr)]; |
|
884 |
val goal = fold_rev Logic.all [p, u] (mk_imp_p (map mk_prem usel_ctrs)); |
|
885 |
in |
|
886 |
Goal.prove_sorry lthy [] [] goal (fn _ => |
|
887 |
mk_sel_exhaust_tac n disc_exhaust_thm swapped_all_collapse_thms) |
|
888 |
|> Thm.close_derivation |
|
889 |
end; |
|
890 |
||
53919 | 891 |
val expand_thm = |
49486 | 892 |
let |
893 |
fun mk_prems k udisc usels vdisc vsels = |
|
894 |
(if k = n then [] else [mk_Trueprop_eq (udisc, vdisc)]) @ |
|
895 |
(if null usels then |
|
896 |
[] |
|
897 |
else |
|
898 |
[Logic.list_implies |
|
899 |
(if n = 1 then [] else map HOLogic.mk_Trueprop [udisc, vdisc], |
|
900 |
HOLogic.mk_Trueprop (Library.foldr1 HOLogic.mk_conj |
|
901 |
(map2 (curry HOLogic.mk_eq) usels vsels)))]); |
|
902 |
||
49591
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
903 |
val goal = |
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
904 |
Library.foldr Logic.list_implies |
91b228e26348
generate high-level "coinduct" and "strong_coinduct" properties
blanchet
parents:
49586
diff
changeset
|
905 |
(map5 mk_prems ks udiscs uselss vdiscs vselss, uv_eq); |
49486 | 906 |
val uncollapse_thms = |
53740 | 907 |
map2 (fn thm => fn [] => thm | _ => thm RS sym) all_collapse_thms uselss; |
49486 | 908 |
in |
53919 | 909 |
Goal.prove_sorry lthy [] [] goal (fn _ => |
910 |
mk_expand_tac lthy n ms (inst_thm u disc_exhaust_thm) |
|
911 |
(inst_thm v disc_exhaust_thm) uncollapse_thms disc_exclude_thmsss |
|
912 |
disc_exclude_thmsss') |
|
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
913 |
|> singleton (Proof_Context.export names_lthy lthy) |
53919 | 914 |
|> Thm.close_derivation |
49486 | 915 |
end; |
49278 | 916 |
|
53917 | 917 |
val (sel_split_thm, sel_split_asm_thm) = |
918 |
let |
|
919 |
val zss = map (K []) xss; |
|
920 |
val goal = mk_split_goal usel_ctrs zss usel_fs; |
|
921 |
val asm_goal = mk_split_asm_goal usel_ctrs zss usel_fs; |
|
922 |
||
923 |
val thm = prove_split sel_thmss goal; |
|
924 |
val asm_thm = prove_split_asm asm_goal thm; |
|
925 |
in |
|
926 |
(thm, asm_thm) |
|
927 |
end; |
|
928 |
||
54491 | 929 |
val case_eq_if_thm = |
49486 | 930 |
let |
53917 | 931 |
val goal = mk_Trueprop_eq (ufcase, mk_IfN B udiscs usel_fs); |
49486 | 932 |
in |
53919 | 933 |
Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, ...} => |
54491 | 934 |
mk_case_eq_if_tac ctxt n uexhaust_thm case_thms disc_thmss' sel_thmss) |
55409
b74248961819
made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet
parents:
55407
diff
changeset
|
935 |
|> singleton (Proof_Context.export names_lthy lthy) |
53919 | 936 |
|> Thm.close_derivation |
49486 | 937 |
end; |
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
938 |
in |
56858 | 939 |
(sel_defs, all_sel_thms, sel_thmss, disc_defs, disc_thmss, nontriv_disc_thmss, |
940 |
discI_thms, nontriv_discI_thms, disc_exclude_thms, disc_exclude_thmsss, |
|
941 |
[disc_exhaust_thm], [sel_exhaust_thm], all_collapse_thms, safe_collapse_thms, |
|
942 |
[expand_thm], [sel_split_thm], [sel_split_asm_thm], [case_eq_if_thm]) |
|
49116
3d520eec2746
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
blanchet
parents:
49114
diff
changeset
|
943 |
end; |
49025 | 944 |
|
49437 | 945 |
val exhaust_case_names_attr = Attrib.internal (K (Rule_Cases.case_names exhaust_cases)); |
53908 | 946 |
val cases_type_attr = Attrib.internal (K (Induct.cases_type fcT_name)); |
49300 | 947 |
|
55464 | 948 |
val nontriv_disc_eq_thmss = |
949 |
map (map (fn th => th RS @{thm eq_False[THEN iffD2]} |
|
950 |
handle THM _ => th RS @{thm eq_True[THEN iffD2]})) nontriv_disc_thmss; |
|
951 |
||
54151 | 952 |
val anonymous_notes = |
953 |
[(map (fn th => th RS notE) distinct_thms, safe_elim_attrs), |
|
55464 | 954 |
(flat nontriv_disc_eq_thmss, code_nitpicksimp_attrs)] |
54151 | 955 |
|> map (fn (thms, attrs) => ((Binding.empty, attrs), [(thms, [])])); |
956 |
||
57038 | 957 |
(* "exhaust" is deliberately put first to avoid apparent circular dependencies in the proof |
958 |
objects, which would confuse MaSh. *) |
|
49052 | 959 |
val notes = |
57038 | 960 |
[(exhaustN, [exhaust_thm], [exhaust_case_names_attr, cases_type_attr]), |
961 |
(caseN, case_thms, code_nitpicksimp_simp_attrs), |
|
49594
55e798614c45
tweaked theorem names (in particular, dropped s's)
blanchet
parents:
49591
diff
changeset
|
962 |
(case_congN, [case_cong_thm], []), |
54491 | 963 |
(case_eq_ifN, case_eq_if_thms, []), |
53740 | 964 |
(collapseN, safe_collapse_thms, simp_attrs), |
55464 | 965 |
(discN, flat nontriv_disc_thmss, simp_attrs), |
53700 | 966 |
(discIN, nontriv_discI_thms, []), |
53836 | 967 |
(disc_excludeN, disc_exclude_thms, dest_attrs), |
49300 | 968 |
(disc_exhaustN, disc_exhaust_thms, [exhaust_case_names_attr]), |
54145
297d1c603999
make sure that registered code equations are actually equations
blanchet
parents:
54008
diff
changeset
|
969 |
(distinctN, distinct_thms, simp_attrs @ inductsimp_attrs), |
49486 | 970 |
(expandN, expand_thms, []), |
54145
297d1c603999
make sure that registered code equations are actually equations
blanchet
parents:
54008
diff
changeset
|
971 |
(injectN, inject_thms, iff_attrs @ inductsimp_attrs), |
49300 | 972 |
(nchotomyN, [nchotomy_thm], []), |
54145
297d1c603999
make sure that registered code equations are actually equations
blanchet
parents:
54008
diff
changeset
|
973 |
(selN, all_sel_thms, code_nitpicksimp_simp_attrs), |
53916 | 974 |
(sel_exhaustN, sel_exhaust_thms, [exhaust_case_names_attr]), |
53917 | 975 |
(sel_splitN, sel_split_thms, []), |
976 |
(sel_split_asmN, sel_split_asm_thms, []), |
|
49300 | 977 |
(splitN, [split_thm], []), |
978 |
(split_asmN, [split_asm_thm], []), |
|
49633 | 979 |
(splitsN, [split_thm, split_asm_thm], []), |
49300 | 980 |
(weak_case_cong_thmsN, [weak_case_cong_thm], cong_attrs)] |
981 |
|> filter_out (null o #2) |
|
982 |
|> map (fn (thmN, thms, attrs) => |
|
49633 | 983 |
((qualify true (Binding.name thmN), attrs), [(thms, [])])); |
49300 | 984 |
|
57629
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
985 |
val (noted, lthy') = |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
986 |
lthy |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
987 |
|> Spec_Rules.add Spec_Rules.Equational ([casex], case_thms) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
988 |
|> fold (Spec_Rules.add Spec_Rules.Equational) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
989 |
(AList.group (eq_list (op aconv)) (map (`(single o lhs_head_of)) all_sel_thms)) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
990 |
|> fold (Spec_Rules.add Spec_Rules.Equational) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
991 |
(filter_out (null o snd) (map single discs ~~ nontriv_disc_eq_thmss)) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
992 |
|> Local_Theory.declaration {syntax = false, pervasive = true} |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
993 |
(fn phi => Case_Translation.register |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
994 |
(Morphism.term phi casex) (map (Morphism.term phi) ctrs)) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
995 |
|> Local_Theory.background_theory (fold (fold Code.del_eqn) [disc_defs, sel_defs]) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
996 |
|> not no_code ? |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
997 |
Local_Theory.declaration {syntax = false, pervasive = false} |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
998 |
(fn phi => Context.mapping |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
999 |
(add_ctr_code fcT_name (map (Morphism.typ phi) As) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1000 |
(map (dest_Const o Morphism.term phi) ctrs) (Morphism.fact phi inject_thms) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1001 |
(Morphism.fact phi distinct_thms) (Morphism.fact phi case_thms)) |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1002 |
I) |
57633 | 1003 |
|> Local_Theory.notes (anonymous_notes @ notes) |
1004 |
(* for "datatype_realizer.ML": *) |
|
1005 |
|>> name_noted_thms fcT_name exhaustN; |
|
57629
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1006 |
|
53867
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
1007 |
val ctr_sugar = |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
1008 |
{ctrs = ctrs, casex = casex, discs = discs, selss = selss, exhaust = exhaust_thm, |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
1009 |
nchotomy = nchotomy_thm, injects = inject_thms, distincts = distinct_thms, |
8ad44ecc0d15
keep a database of free constructor type information
blanchet
parents:
53864
diff
changeset
|
1010 |
case_thms = case_thms, case_cong = case_cong_thm, weak_case_cong = weak_case_cong_thm, |
56858 | 1011 |
split = split_thm, split_asm = split_asm_thm, disc_defs = disc_defs, |
1012 |
disc_thmss = disc_thmss, discIs = discI_thms, sel_defs = sel_defs, sel_thmss = sel_thmss, |
|
1013 |
disc_excludesss = disc_exclude_thmsss, disc_exhausts = disc_exhaust_thms, |
|
1014 |
sel_exhausts = sel_exhaust_thms, collapses = all_collapse_thms, expands = expand_thms, |
|
1015 |
sel_splits = sel_split_thms, sel_split_asms = sel_split_asm_thms, |
|
57629
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1016 |
case_eq_ifs = case_eq_if_thms} |
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1017 |
|> morph_ctr_sugar (substitute_noted_thm noted); |
49019 | 1018 |
in |
57629
e88b5f59cade
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
blanchet
parents:
57260
diff
changeset
|
1019 |
(ctr_sugar, lthy' |> register_ctr_sugar fcT_name ctr_sugar) |
49019 | 1020 |
end; |
49017 | 1021 |
in |
49121 | 1022 |
(goalss, after_qed, lthy') |
49017 | 1023 |
end; |
1024 |
||
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1025 |
fun free_constructors tacss = (fn (goalss, after_qed, lthy) => |
51551 | 1026 |
map2 (map2 (Thm.close_derivation oo Goal.prove_sorry lthy [] [])) goalss tacss |
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1027 |
|> (fn thms => after_qed thms lthy)) oo prepare_free_constructors (K I); |
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
1028 |
|
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1029 |
val free_constructors_cmd = (fn (goalss, after_qed, lthy) => |
49297 | 1030 |
Proof.theorem NONE (snd oo after_qed) (map (map (rpair [])) goalss) lthy) oo |
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1031 |
prepare_free_constructors Syntax.read_term; |
49297 | 1032 |
|
57091 | 1033 |
val parse_bound_term = Parse.binding --| @{keyword ":"} -- Parse.term; |
49280
52413dc96326
allow default values for selectors in low-level "wrap_data" command
blanchet
parents:
49278
diff
changeset
|
1034 |
|
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
1035 |
val parse_ctr_options = |
54626 | 1036 |
Scan.optional (@{keyword "("} |-- Parse.list1 |
57094
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57091
diff
changeset
|
1037 |
(Parse.reserved "discs_sels" >> K 0 || Parse.reserved "no_code" >> K 1) --| |
55410 | 1038 |
@{keyword ")"} |
1039 |
>> (fn js => (member (op =) js 0, member (op =) js 1))) |
|
1040 |
(false, false); |
|
49278 | 1041 |
|
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
1042 |
fun parse_ctr_spec parse_ctr parse_arg = |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
1043 |
parse_opt_binding_colon -- parse_ctr -- Scan.repeat parse_arg; |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
1044 |
|
57091 | 1045 |
val parse_ctr_specs = Parse.enum1 "|" (parse_ctr_spec Parse.term Parse.binding); |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
1046 |
val parse_sel_default_eqs = Scan.optional (@{keyword "where"} |-- Parse.enum1 "|" Parse.prop) []; |
55469
b19dd108f0c2
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet
parents:
55468
diff
changeset
|
1047 |
|
49017 | 1048 |
val _ = |
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1049 |
Outer_Syntax.local_theory_to_proof @{command_spec "free_constructors"} |
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1050 |
"register an existing freely generated type's constructors" |
57091 | 1051 |
(parse_ctr_options -- Parse.binding --| @{keyword "for"} -- parse_ctr_specs |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57094
diff
changeset
|
1052 |
-- parse_sel_default_eqs |
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55464
diff
changeset
|
1053 |
>> free_constructors_cmd); |
49017 | 1054 |
|
56522
f54003750e7d
don't forget to init Interpretation and transfer theorems in the interpretation hook
kuncar
parents:
56376
diff
changeset
|
1055 |
val _ = Context.>> (Context.map_theory Ctr_Sugar_Interpretation.init); |
f54003750e7d
don't forget to init Interpretation and transfer theorems in the interpretation hook
kuncar
parents:
56376
diff
changeset
|
1056 |
|
49017 | 1057 |
end; |