author | wenzelm |
Wed, 23 Jul 2014 15:11:42 +0200 | |
changeset 57618 | d762318438c3 |
parent 56903 | 69b6369a98fa |
child 57668 | 09d2b853b20c |
permissions | -rw-r--r-- |
55061 | 1 |
(* Title: HOL/Tools/BNF/bnf_def_tactics.ML |
49284 | 2 |
Author: Dmitriy Traytel, TU Muenchen |
3 |
Author: Jasmin Blanchette, TU Muenchen |
|
4 |
Copyright 2012 |
|
5 |
||
6 |
Tactics for definition of bounded natural functors. |
|
7 |
*) |
|
8 |
||
9 |
signature BNF_DEF_TACTICS = |
|
10 |
sig |
|
51766
f19a4d0ab1bf
renamed "set_natural" to "set_map", reflecting {Bl,Po,Tr} concensus
blanchet
parents:
51762
diff
changeset
|
11 |
val mk_collect_set_map_tac: thm list -> tactic |
56635 | 12 |
val mk_in_mono_tac: int -> tactic |
13 |
val mk_inj_map_tac: int -> thm -> thm -> thm -> thm -> tactic |
|
53285 | 14 |
val mk_map_id: thm -> thm |
56903 | 15 |
val mk_map_ident: Proof.context -> thm -> thm |
53288 | 16 |
val mk_map_comp: thm -> thm |
51798 | 17 |
val mk_map_cong_tac: Proof.context -> thm -> tactic |
53290 | 18 |
val mk_set_map: thm -> thm |
49284 | 19 |
|
55197 | 20 |
val mk_rel_Grp_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm -> thm list -> tactic |
51894 | 21 |
val mk_rel_eq_tac: int -> thm -> thm -> thm -> tactic |
55197 | 22 |
val mk_rel_OO_le_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm list -> tactic |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
23 |
val mk_rel_conversep_tac: thm -> thm -> tactic |
55197 | 24 |
val mk_rel_conversep_le_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm list -> tactic |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
25 |
val mk_rel_mono_tac: thm list -> thm -> tactic |
55197 | 26 |
val mk_rel_mono_strong_tac: Proof.context -> thm -> thm list -> tactic |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
27 |
|
55197 | 28 |
val mk_map_transfer_tac: Proof.context -> thm -> thm -> thm list -> thm -> thm -> tactic |
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
29 |
|
55197 | 30 |
val mk_in_bd_tac: Proof.context -> int -> thm -> thm -> thm -> thm -> thm list -> thm list -> |
31 |
thm -> thm -> thm -> thm -> tactic |
|
54189
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
32 |
|
55197 | 33 |
val mk_trivial_wit_tac: Proof.context -> thm list -> thm list -> tactic |
49284 | 34 |
end; |
35 |
||
36 |
structure BNF_Def_Tactics : BNF_DEF_TACTICS = |
|
37 |
struct |
|
38 |
||
39 |
open BNF_Util |
|
40 |
open BNF_Tactics |
|
41 |
||
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
42 |
val ord_eq_le_trans = @{thm ord_eq_le_trans}; |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
43 |
val ord_le_eq_trans = @{thm ord_le_eq_trans}; |
52749 | 44 |
val conversep_shift = @{thm conversep_le_swap} RS iffD1; |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
45 |
|
53285 | 46 |
fun mk_map_id id = mk_trans (fun_cong OF [id]) @{thm id_apply}; |
56903 | 47 |
fun mk_map_ident ctxt = unfold_thms ctxt @{thms id_def}; |
55067 | 48 |
fun mk_map_comp comp = @{thm comp_eq_dest_lhs} OF [mk_sym comp]; |
51798 | 49 |
fun mk_map_cong_tac ctxt cong0 = |
50 |
(hyp_subst_tac ctxt THEN' rtac cong0 THEN' |
|
51762 | 51 |
REPEAT_DETERM o (dtac meta_spec THEN' etac meta_mp THEN' atac)) 1; |
53290 | 52 |
fun mk_set_map set_map0 = set_map0 RS @{thm comp_eq_dest}; |
49490 | 53 |
fun mk_in_mono_tac n = if n = 0 then rtac subset_UNIV 1 |
49284 | 54 |
else (rtac subsetI THEN' |
55 |
rtac CollectI) 1 THEN |
|
56 |
REPEAT_DETERM (eresolve_tac [CollectE, conjE] 1) THEN |
|
57 |
REPEAT_DETERM_N (n - 1) |
|
58 |
((rtac conjI THEN' etac subset_trans THEN' atac) 1) THEN |
|
59 |
(etac subset_trans THEN' atac) 1; |
|
60 |
||
56635 | 61 |
fun mk_inj_map_tac n map_id map_comp map_cong0 map_cong = |
62 |
let |
|
63 |
val map_cong' = map_cong OF (asm_rl :: replicate n refl); |
|
64 |
val map_cong0' = map_cong0 OF (replicate n @{thm the_inv_f_o_f_id}); |
|
65 |
in |
|
66 |
HEADGOAL (rtac @{thm injI} THEN' etac (map_cong' RS box_equals) THEN' |
|
67 |
REPEAT_DETERM_N 2 o (rtac (box_equals OF [map_cong0', map_comp RS sym, map_id]) THEN' |
|
68 |
REPEAT_DETERM_N n o atac)) |
|
69 |
end; |
|
70 |
||
53289 | 71 |
fun mk_collect_set_map_tac set_map0s = |
55067 | 72 |
(rtac (@{thm collect_comp} RS trans) THEN' rtac @{thm arg_cong[of _ _ collect]} THEN' |
53289 | 73 |
EVERY' (map (fn set_map0 => |
49623 | 74 |
rtac (mk_trans @{thm image_insert} @{thm arg_cong2[of _ _ _ _ insert]}) THEN' |
53289 | 75 |
rtac set_map0) set_map0s) THEN' |
49623 | 76 |
rtac @{thm image_empty}) 1; |
49284 | 77 |
|
55197 | 78 |
fun mk_rel_Grp_tac ctxt rel_OO_Grps map_id0 map_cong0 map_id map_comp set_maps = |
49284 | 79 |
let |
54792 | 80 |
val n = length set_maps; |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
81 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac else rtac (hd rel_OO_Grps RS trans); |
49284 | 82 |
in |
54792 | 83 |
if null set_maps then |
53270 | 84 |
unfold_thms_tac ctxt ((map_id0 RS @{thm Grp_UNIV_id}) :: rel_OO_Grps) THEN |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
85 |
rtac @{thm Grp_UNIV_idI[OF refl]} 1 |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
86 |
else |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
87 |
EVERY' [rel_OO_Grps_tac, rtac @{thm antisym}, rtac @{thm predicate2I}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
88 |
REPEAT_DETERM o |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
89 |
eresolve_tac [CollectE, exE, conjE, @{thm GrpE}, @{thm relcomppE}, @{thm conversepE}], |
54792 | 90 |
hyp_subst_tac ctxt, rtac @{thm GrpI}, rtac trans, rtac map_comp, rtac map_cong0, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
91 |
REPEAT_DETERM_N n o EVERY' [rtac @{thm Collect_split_Grp_eqD}, etac @{thm set_mp}, atac], |
49284 | 92 |
rtac CollectI, |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
93 |
CONJ_WRAP' (fn thm => EVERY' [rtac (thm RS ord_eq_le_trans), |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
94 |
rtac @{thm image_subsetI}, rtac @{thm Collect_split_Grp_inD}, etac @{thm set_mp}, atac]) |
54792 | 95 |
set_maps, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
96 |
rtac @{thm predicate2I}, REPEAT_DETERM o eresolve_tac [@{thm GrpE}, exE, conjE], |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
97 |
hyp_subst_tac ctxt, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
98 |
rtac @{thm relcomppI}, rtac @{thm conversepI}, |
53270 | 99 |
EVERY' (map2 (fn convol => fn map_id0 => |
55990 | 100 |
EVERY' [rtac @{thm GrpI}, |
101 |
rtac (@{thm box_equals} OF [map_cong0, map_comp RS sym, map_id0]), |
|
49495 | 102 |
REPEAT_DETERM_N n o rtac (convol RS fun_cong), |
103 |
REPEAT_DETERM o eresolve_tac [CollectE, conjE], |
|
104 |
rtac CollectI, |
|
105 |
CONJ_WRAP' (fn thm => |
|
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
106 |
EVERY' [rtac ord_eq_le_trans, rtac thm, rtac @{thm image_subsetI}, |
52986
7f7bbeb16538
eliminated bogus assumption from theorem (that was instantiated with refl and resulted in flexflex pairs)
traytel
parents:
52844
diff
changeset
|
107 |
rtac @{thm convol_mem_GrpI}, etac set_mp, atac]) |
54792 | 108 |
set_maps]) |
53285 | 109 |
@{thms fst_convol snd_convol} [map_id, refl])] 1 |
49284 | 110 |
end; |
111 |
||
53270 | 112 |
fun mk_rel_eq_tac n rel_Grp rel_cong map_id0 = |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
113 |
(EVERY' (rtac (rel_cong RS trans) :: replicate n (rtac @{thm eq_alt})) THEN' |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
114 |
rtac (rel_Grp RSN (2, @{thm box_equals[OF _ sym sym[OF eq_alt]]})) THEN' |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
115 |
(if n = 0 then rtac refl |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
116 |
else EVERY' [rtac @{thm arg_cong2[of _ _ _ _ "Grp"]}, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
117 |
rtac @{thm equalityI}, rtac subset_UNIV, rtac subsetI, rtac CollectI, |
53270 | 118 |
CONJ_WRAP' (K (rtac subset_UNIV)) (1 upto n), rtac map_id0])) 1; |
49284 | 119 |
|
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
120 |
fun mk_rel_mono_tac rel_OO_Grps in_mono = |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
121 |
let |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
122 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
123 |
else rtac (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
124 |
rtac (hd rel_OO_Grps RS sym RSN (2, ord_le_eq_trans)); |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
125 |
in |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
126 |
EVERY' [rel_OO_Grps_tac, rtac @{thm relcompp_mono}, rtac @{thm iffD2[OF conversep_mono]}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
127 |
rtac @{thm Grp_mono}, rtac in_mono, REPEAT_DETERM o etac @{thm Collect_split_mono}, |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
128 |
rtac @{thm Grp_mono}, rtac in_mono, REPEAT_DETERM o etac @{thm Collect_split_mono}] 1 |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
129 |
end; |
49284 | 130 |
|
55197 | 131 |
fun mk_rel_conversep_le_tac ctxt rel_OO_Grps rel_eq map_cong0 map_comp set_maps = |
49284 | 132 |
let |
54792 | 133 |
val n = length set_maps; |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
134 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
135 |
else rtac (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
136 |
rtac (hd rel_OO_Grps RS sym RS @{thm arg_cong[of _ _ conversep]} RSN (2, ord_le_eq_trans)); |
49284 | 137 |
in |
54792 | 138 |
if null set_maps then rtac (rel_eq RS @{thm leq_conversepI}) 1 |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
139 |
else |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
140 |
EVERY' [rel_OO_Grps_tac, rtac @{thm predicate2I}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
141 |
REPEAT_DETERM o |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
142 |
eresolve_tac [CollectE, exE, conjE, @{thm GrpE}, @{thm relcomppE}, @{thm conversepE}], |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
143 |
hyp_subst_tac ctxt, rtac @{thm conversepI}, rtac @{thm relcomppI}, rtac @{thm conversepI}, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
144 |
EVERY' (map (fn thm => EVERY' [rtac @{thm GrpI}, rtac sym, rtac trans, |
51761
4c9f08836d87
renamed "map_cong" axiom to "map_cong0" in preparation for real "map_cong"
blanchet
parents:
49623
diff
changeset
|
145 |
rtac map_cong0, REPEAT_DETERM_N n o rtac thm, |
54792 | 146 |
rtac (map_comp RS sym), rtac CollectI, |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
147 |
CONJ_WRAP' (fn thm => EVERY' [rtac (thm RS ord_eq_le_trans), |
54792 | 148 |
etac @{thm flip_pred}]) set_maps]) [@{thm snd_fst_flip}, @{thm fst_snd_flip}])] 1 |
49284 | 149 |
end; |
150 |
||
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
151 |
fun mk_rel_conversep_tac le_conversep rel_mono = |
52749 | 152 |
EVERY' [rtac @{thm antisym}, rtac le_conversep, rtac @{thm xt1(6)}, rtac conversep_shift, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
153 |
rtac le_conversep, rtac @{thm iffD2[OF conversep_mono]}, rtac rel_mono, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
154 |
REPEAT_DETERM o rtac @{thm eq_refl[OF sym[OF conversep_conversep]]}] 1; |
49284 | 155 |
|
55197 | 156 |
fun mk_rel_OO_le_tac ctxt rel_OO_Grps rel_eq map_cong0 map_comp set_maps = |
49284 | 157 |
let |
54792 | 158 |
val n = length set_maps; |
49284 | 159 |
fun in_tac nthO_in = rtac CollectI THEN' |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
160 |
CONJ_WRAP' (fn thm => EVERY' [rtac (thm RS ord_eq_le_trans), |
54792 | 161 |
rtac @{thm image_subsetI}, rtac nthO_in, etac set_mp, atac]) set_maps; |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
162 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
163 |
else rtac (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
164 |
rtac (@{thm arg_cong2[of _ _ _ _ "op OO"]} OF (replicate 2 (hd rel_OO_Grps RS sym)) RSN |
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
165 |
(2, ord_le_eq_trans)); |
49284 | 166 |
in |
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
167 |
if null set_maps then rtac (rel_eq RS @{thm leq_OOI}) 1 |
52844
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
168 |
else |
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
169 |
EVERY' [rel_OO_Grps_tac, rtac @{thm predicate2I}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
170 |
REPEAT_DETERM o |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
171 |
eresolve_tac [CollectE, exE, conjE, @{thm GrpE}, @{thm relcomppE}, @{thm conversepE}], |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
172 |
hyp_subst_tac ctxt, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
173 |
rtac @{thm relcomppI}, rtac @{thm relcomppI}, rtac @{thm conversepI}, rtac @{thm GrpI}, |
54792 | 174 |
rtac trans, rtac map_comp, rtac sym, rtac map_cong0, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
175 |
REPEAT_DETERM_N n o rtac @{thm fst_fstOp}, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
176 |
in_tac @{thm fstOp_in}, |
54792 | 177 |
rtac @{thm GrpI}, rtac trans, rtac map_comp, rtac map_cong0, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
178 |
REPEAT_DETERM_N n o EVERY' [rtac trans, rtac o_apply, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
179 |
rtac ballE, rtac subst, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
180 |
rtac @{thm csquare_def}, rtac @{thm csquare_fstOp_sndOp}, atac, etac notE, |
49284 | 181 |
etac set_mp, atac], |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
182 |
in_tac @{thm fstOp_in}, |
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
183 |
rtac @{thm relcomppI}, rtac @{thm conversepI}, rtac @{thm GrpI}, |
54792 | 184 |
rtac trans, rtac map_comp, rtac map_cong0, |
49284 | 185 |
REPEAT_DETERM_N n o rtac o_apply, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
186 |
in_tac @{thm sndOp_in}, |
54792 | 187 |
rtac @{thm GrpI}, rtac trans, rtac map_comp, rtac sym, rtac map_cong0, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
188 |
REPEAT_DETERM_N n o rtac @{thm snd_sndOp}, |
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
189 |
in_tac @{thm sndOp_in}] 1 |
49284 | 190 |
end; |
191 |
||
55197 | 192 |
fun mk_rel_mono_strong_tac ctxt in_rel set_maps = |
54792 | 193 |
if null set_maps then atac 1 |
51916 | 194 |
else |
54998 | 195 |
unfold_tac ctxt [in_rel] THEN |
51916 | 196 |
REPEAT_DETERM (eresolve_tac [exE, CollectE, conjE] 1) THEN |
197 |
hyp_subst_tac ctxt 1 THEN |
|
198 |
EVERY' [rtac exI, rtac @{thm conjI[OF CollectI conjI[OF refl refl]]}, |
|
55163 | 199 |
CONJ_WRAP' (fn thm => |
200 |
(etac (@{thm Collect_split_mono_strong} OF [thm, thm]) THEN' atac)) |
|
201 |
set_maps] 1; |
|
51916 | 202 |
|
55197 | 203 |
fun mk_map_transfer_tac ctxt rel_mono in_rel set_maps map_cong0 map_comp = |
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
204 |
let |
53290 | 205 |
val n = length set_maps; |
53562 | 206 |
val in_tac = if n = 0 then rtac UNIV_I else |
207 |
rtac CollectI THEN' CONJ_WRAP' (fn thm => |
|
208 |
etac (thm RS |
|
209 |
@{thm ord_eq_le_trans[OF _ subset_trans[OF image_mono convol_image_vimage2p]]})) |
|
210 |
set_maps; |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
211 |
in |
55945 | 212 |
REPEAT_DETERM_N n (HEADGOAL (rtac @{thm rel_funI})) THEN |
213 |
unfold_thms_tac ctxt @{thms rel_fun_iff_leq_vimage2p} THEN |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
214 |
HEADGOAL (EVERY' [rtac @{thm order_trans}, rtac rel_mono, REPEAT_DETERM_N n o atac, |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
215 |
rtac @{thm predicate2I}, dtac (in_rel RS iffD1), |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
216 |
REPEAT_DETERM o eresolve_tac [exE, CollectE, conjE], hyp_subst_tac ctxt, |
53562 | 217 |
rtac @{thm vimage2pI}, rtac (in_rel RS iffD2), rtac exI, rtac conjI, in_tac, |
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
218 |
rtac conjI, |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
219 |
EVERY' (map (fn convol => |
55990 | 220 |
rtac (@{thm box_equals} OF [map_cong0, map_comp RS sym, map_comp RS sym]) THEN' |
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
221 |
REPEAT_DETERM_N n o rtac (convol RS fun_cong)) @{thms fst_convol snd_convol})]) |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
222 |
end; |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
223 |
|
55197 | 224 |
fun mk_in_bd_tac ctxt live surj_imp_ordLeq_inst map_comp map_id map_cong0 set_maps set_bds |
225 |
bd_card_order bd_Card_order bd_Cinfinite bd_Cnotzero = |
|
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
226 |
if live = 0 then |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
227 |
rtac @{thm ordLeq_transitive[OF ordLeq_csum2[OF card_of_Card_order] |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
228 |
ordLeq_cexp2[OF ordLeq_refl[OF Card_order_ctwo] Card_order_csum]]} 1 |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
229 |
else |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
230 |
let |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
231 |
val bd'_Cinfinite = bd_Cinfinite RS @{thm Cinfinite_csum1}; |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
232 |
val inserts = |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
233 |
map (fn set_bd => |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
234 |
iffD2 OF [@{thm card_of_ordLeq}, @{thm ordLeq_ordIso_trans} OF |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
235 |
[set_bd, bd_Card_order RS @{thm card_of_Field_ordIso} RS @{thm ordIso_symmetric}]]) |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
236 |
set_bds; |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
237 |
in |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
238 |
EVERY' [rtac (Drule.rotate_prems 1 ctrans), rtac @{thm cprod_cinfinite_bound}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
239 |
rtac (ctrans OF @{thms ordLeq_csum2 ordLeq_cexp2}), rtac @{thm card_of_Card_order}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
240 |
rtac @{thm ordLeq_csum2}, rtac @{thm Card_order_ctwo}, rtac @{thm Card_order_csum}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
241 |
rtac @{thm ordIso_ordLeq_trans}, rtac @{thm cexp_cong1}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
242 |
if live = 1 then rtac @{thm ordIso_refl[OF Card_order_csum]} |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
243 |
else |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
244 |
REPEAT_DETERM_N (live - 2) o rtac @{thm ordIso_transitive[OF csum_cong2]} THEN' |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
245 |
REPEAT_DETERM_N (live - 1) o rtac @{thm csum_csum}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
246 |
rtac bd_Card_order, rtac (@{thm cexp_mono2_Cnotzero} RS ctrans), rtac @{thm ordLeq_csum1}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
247 |
rtac bd_Card_order, rtac @{thm Card_order_csum}, rtac bd_Cnotzero, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
248 |
rtac @{thm csum_Cfinite_cexp_Cinfinite}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
249 |
rtac (if live = 1 then @{thm card_of_Card_order} else @{thm Card_order_csum}), |
53290 | 250 |
CONJ_WRAP_GEN' (rtac @{thm Cfinite_csum}) (K (rtac @{thm Cfinite_cone})) set_maps, |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
251 |
rtac bd'_Cinfinite, rtac @{thm card_of_Card_order}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
252 |
rtac @{thm Card_order_cexp}, rtac @{thm Cinfinite_cexp}, rtac @{thm ordLeq_csum2}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
253 |
rtac @{thm Card_order_ctwo}, rtac bd'_Cinfinite, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
254 |
rtac (Drule.rotate_prems 1 (@{thm cprod_mono2} RSN (2, ctrans))), |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
255 |
REPEAT_DETERM_N (live - 1) o |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
256 |
(rtac (bd_Cinfinite RS @{thm cprod_cexp_csum_cexp_Cinfinite} RSN (2, ctrans)) THEN' |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
257 |
rtac @{thm ordLeq_ordIso_trans[OF cprod_mono2 ordIso_symmetric[OF cprod_cexp]]}), |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
258 |
rtac @{thm ordLeq_refl[OF Card_order_cexp]}] 1 THEN |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
259 |
unfold_thms_tac ctxt [bd_card_order RS @{thm card_order_csum_cone_cexp_def}] THEN |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
260 |
unfold_thms_tac ctxt @{thms cprod_def Field_card_of} THEN |
52813 | 261 |
EVERY' [rtac (Drule.rotate_prems 1 ctrans), rtac surj_imp_ordLeq_inst, rtac subsetI, |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
262 |
Method.insert_tac inserts, REPEAT_DETERM o dtac meta_spec, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
263 |
REPEAT_DETERM o eresolve_tac [exE, Tactic.make_elim conjunct1], etac CollectE, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
264 |
if live = 1 then K all_tac |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
265 |
else REPEAT_DETERM_N (live - 2) o (etac conjE THEN' rotate_tac ~1) THEN' etac conjE, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
266 |
rtac (Drule.rotate_prems 1 @{thm image_eqI}), rtac @{thm SigmaI}, rtac @{thm UNIV_I}, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
267 |
CONJ_WRAP_GEN' (rtac @{thm SigmaI}) |
53290 | 268 |
(K (etac @{thm If_the_inv_into_in_Func} THEN' atac)) set_maps, |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
269 |
rtac sym, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
270 |
rtac (Drule.rotate_prems 1 |
55990 | 271 |
((@{thm box_equals} OF [map_cong0 OF replicate live @{thm If_the_inv_into_f_f}, |
53288 | 272 |
map_comp RS sym, map_id]) RSN (2, trans))), |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
273 |
REPEAT_DETERM_N (2 * live) o atac, |
55642
63beb38e9258
adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
blanchet
parents:
55414
diff
changeset
|
274 |
REPEAT_DETERM_N live o rtac (@{thm prod.case} RS trans), |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
275 |
rtac refl, |
52813 | 276 |
rtac @{thm surj_imp_ordLeq}, rtac subsetI, rtac (Drule.rotate_prems 1 @{thm image_eqI}), |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
277 |
REPEAT_DETERM o eresolve_tac [CollectE, conjE], rtac CollectI, |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
278 |
CONJ_WRAP' (fn thm => |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
279 |
rtac (thm RS ord_eq_le_trans) THEN' etac @{thm subset_trans[OF image_mono Un_upper1]}) |
53290 | 280 |
set_maps, |
52813 | 281 |
rtac sym, |
55990 | 282 |
rtac (@{thm box_equals} OF [map_cong0 OF replicate live @{thm fun_cong[OF case_sum_o_inj(1)]}, |
53288 | 283 |
map_comp RS sym, map_id])] 1 |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
284 |
end; |
51916 | 285 |
|
55197 | 286 |
fun mk_trivial_wit_tac ctxt wit_defs set_maps = |
54189
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
287 |
unfold_thms_tac ctxt wit_defs THEN HEADGOAL (EVERY' (map (fn thm => |
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
288 |
dtac (thm RS equalityD1 RS set_mp) THEN' etac imageE THEN' atac) set_maps)) THEN ALLGOALS atac; |
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
289 |
|
49284 | 290 |
end; |