author | wenzelm |
Tue, 22 Jul 2025 12:02:53 +0200 | |
changeset 82894 | a8e47bd31965 |
parent 75276 | 686a6d7d0991 |
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 |
|
57668 | 4 |
Author: Martin Desharnais, TU Muenchen |
62324 | 5 |
Author: Ondrej Kuncar, TU Muenchen |
6 |
Copyright 2012, 2013, 2014, 2015 |
|
49284 | 7 |
|
8 |
Tactics for definition of bounded natural functors. |
|
9 |
*) |
|
10 |
||
11 |
signature BNF_DEF_TACTICS = |
|
12 |
sig |
|
60728 | 13 |
val mk_collect_set_map_tac: Proof.context -> thm list -> tactic |
14 |
val mk_in_mono_tac: Proof.context -> int -> tactic |
|
57970 | 15 |
val mk_inj_map_strong_tac: Proof.context -> thm -> thm list -> thm -> tactic |
60728 | 16 |
val mk_inj_map_tac: Proof.context -> int -> thm -> thm -> thm -> thm -> tactic |
53285 | 17 |
val mk_map_id: thm -> thm |
56903 | 18 |
val mk_map_ident: Proof.context -> thm -> thm |
75276 | 19 |
val mk_map_ident_strong: Proof.context -> thm -> thm -> thm |
53288 | 20 |
val mk_map_comp: thm -> thm |
51798 | 21 |
val mk_map_cong_tac: Proof.context -> thm -> tactic |
53290 | 22 |
val mk_set_map: thm -> thm |
49284 | 23 |
|
55197 | 24 |
val mk_rel_Grp_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm -> thm list -> tactic |
60728 | 25 |
val mk_rel_eq_tac: Proof.context -> int -> thm -> thm -> thm -> tactic |
55197 | 26 |
val mk_rel_OO_le_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm list -> tactic |
60728 | 27 |
val mk_rel_conversep_tac: Proof.context -> thm -> thm -> tactic |
55197 | 28 |
val mk_rel_conversep_le_tac: Proof.context -> thm list -> thm -> thm -> thm -> thm list -> tactic |
57932 | 29 |
val mk_rel_map0_tac: Proof.context -> int -> thm -> thm -> thm -> thm -> tactic |
60728 | 30 |
val mk_rel_mono_tac: Proof.context -> thm list -> thm -> tactic |
57967 | 31 |
val mk_rel_mono_strong0_tac: Proof.context -> thm -> thm list -> tactic |
61242 | 32 |
val mk_rel_cong_tac: Proof.context -> thm list * thm list -> thm -> tactic |
62324 | 33 |
val mk_rel_eq_onp_tac: Proof.context -> thm -> thm -> thm -> tactic |
34 |
val mk_pred_mono_strong0_tac: Proof.context -> thm -> thm -> tactic |
|
63714 | 35 |
val mk_pred_mono_tac: Proof.context -> thm -> thm -> 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
|
36 |
|
55197 | 37 |
val mk_map_transfer_tac: Proof.context -> thm -> thm -> thm list -> thm -> thm -> tactic |
62329 | 38 |
val mk_pred_transfer_tac: Proof.context -> int -> thm -> thm -> thm -> tactic |
39 |
val mk_rel_transfer_tac: Proof.context -> thm -> thm list -> thm -> tactic |
|
40 |
val mk_set_transfer_tac: Proof.context -> thm -> thm list -> tactic |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
41 |
|
55197 | 42 |
val mk_in_bd_tac: Proof.context -> int -> thm -> thm -> thm -> thm -> thm list -> thm list -> |
43 |
thm -> thm -> thm -> thm -> tactic |
|
54189
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
44 |
|
55197 | 45 |
val mk_trivial_wit_tac: Proof.context -> thm list -> thm list -> tactic |
49284 | 46 |
end; |
47 |
||
48 |
structure BNF_Def_Tactics : BNF_DEF_TACTICS = |
|
49 |
struct |
|
50 |
||
51 |
open BNF_Util |
|
52 |
open BNF_Tactics |
|
53 |
||
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
54 |
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
|
55 |
val ord_le_eq_trans = @{thm ord_le_eq_trans}; |
52749 | 56 |
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
|
57 |
|
53285 | 58 |
fun mk_map_id id = mk_trans (fun_cong OF [id]) @{thm id_apply}; |
56903 | 59 |
fun mk_map_ident ctxt = unfold_thms ctxt @{thms id_def}; |
75276 | 60 |
fun mk_map_ident_strong ctxt map_cong0 map_id = |
61 |
(trans OF [map_cong0, map_id]) |
|
62 |
|> unfold_thms ctxt @{thms id_apply} |
|
55067 | 63 |
fun mk_map_comp comp = @{thm comp_eq_dest_lhs} OF [mk_sym comp]; |
51798 | 64 |
fun mk_map_cong_tac ctxt cong0 = |
60728 | 65 |
(hyp_subst_tac ctxt THEN' rtac ctxt cong0 THEN' |
60752 | 66 |
REPEAT_DETERM o (dtac ctxt meta_spec THEN' etac ctxt meta_mp THEN' assume_tac ctxt)) 1; |
53290 | 67 |
fun mk_set_map set_map0 = set_map0 RS @{thm comp_eq_dest}; |
60757 | 68 |
|
69 |
fun mk_in_mono_tac ctxt n = |
|
70 |
if n = 0 then rtac ctxt subset_UNIV 1 |
|
71 |
else |
|
63399 | 72 |
(rtac ctxt @{thm subsetI} THEN' rtac ctxt @{thm CollectI}) 1 THEN |
73 |
REPEAT_DETERM (eresolve_tac ctxt @{thms CollectE conjE} 1) THEN |
|
60757 | 74 |
REPEAT_DETERM_N (n - 1) |
63399 | 75 |
((rtac ctxt conjI THEN' etac ctxt @{thm subset_trans} THEN' assume_tac ctxt) 1) THEN |
76 |
(etac ctxt @{thm subset_trans} THEN' assume_tac ctxt) 1; |
|
49284 | 77 |
|
60728 | 78 |
fun mk_inj_map_tac ctxt n map_id map_comp map_cong0 map_cong = |
56635 | 79 |
let |
80 |
val map_cong' = map_cong OF (asm_rl :: replicate n refl); |
|
81 |
val map_cong0' = map_cong0 OF (replicate n @{thm the_inv_f_o_f_id}); |
|
82 |
in |
|
60728 | 83 |
HEADGOAL (rtac ctxt @{thm injI} THEN' etac ctxt (map_cong' RS box_equals) THEN' |
84 |
REPEAT_DETERM_N 2 o (rtac ctxt (box_equals OF [map_cong0', map_comp RS sym, map_id]) THEN' |
|
60752 | 85 |
REPEAT_DETERM_N n o assume_tac ctxt)) |
56635 | 86 |
end; |
87 |
||
57970 | 88 |
fun mk_inj_map_strong_tac ctxt rel_eq rel_maps rel_mono_strong = |
89 |
let |
|
90 |
val rel_eq' = rel_eq RS @{thm predicate2_eqD}; |
|
91 |
val rel_maps' = map (fn thm => thm RS iffD1) rel_maps; |
|
92 |
in |
|
60728 | 93 |
HEADGOAL (dtac ctxt (rel_eq' RS iffD2) THEN' rtac ctxt (rel_eq' RS iffD1)) THEN |
94 |
EVERY (map (HEADGOAL o dtac ctxt) rel_maps') THEN |
|
95 |
HEADGOAL (etac ctxt rel_mono_strong) THEN |
|
57970 | 96 |
TRYALL (Goal.assume_rule_tac ctxt) |
97 |
end; |
|
98 |
||
60728 | 99 |
fun mk_collect_set_map_tac ctxt set_map0s = |
100 |
(rtac ctxt (@{thm collect_comp} RS trans) THEN' rtac ctxt @{thm arg_cong[of _ _ collect]} THEN' |
|
53289 | 101 |
EVERY' (map (fn set_map0 => |
60728 | 102 |
rtac ctxt (mk_trans @{thm image_insert} @{thm arg_cong2[of _ _ _ _ insert]}) THEN' |
103 |
rtac ctxt set_map0) set_map0s) THEN' |
|
104 |
rtac ctxt @{thm image_empty}) 1; |
|
49284 | 105 |
|
55197 | 106 |
fun mk_rel_Grp_tac ctxt rel_OO_Grps map_id0 map_cong0 map_id map_comp set_maps = |
49284 | 107 |
let |
54792 | 108 |
val n = length set_maps; |
61760 | 109 |
val rel_OO_Grps_tac = |
110 |
if null rel_OO_Grps then K all_tac else rtac ctxt (hd rel_OO_Grps RS trans); |
|
49284 | 111 |
in |
54792 | 112 |
if null set_maps then |
53270 | 113 |
unfold_thms_tac ctxt ((map_id0 RS @{thm Grp_UNIV_id}) :: rel_OO_Grps) THEN |
62617 | 114 |
resolve_tac ctxt @{thms refl 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
|
115 |
else |
60728 | 116 |
EVERY' [rel_OO_Grps_tac, rtac ctxt @{thm antisym}, rtac ctxt @{thm predicate2I}, |
63399 | 117 |
REPEAT_DETERM o eresolve_tac ctxt @{thms CollectE exE conjE GrpE relcomppE conversepE}, |
61760 | 118 |
hyp_subst_tac ctxt, rtac ctxt @{thm GrpI}, rtac ctxt trans, rtac ctxt map_comp, |
119 |
rtac ctxt map_cong0, |
|
120 |
REPEAT_DETERM_N n o EVERY' [rtac ctxt @{thm Collect_case_prod_Grp_eqD}, |
|
121 |
etac ctxt @{thm set_mp}, assume_tac ctxt], |
|
63399 | 122 |
rtac ctxt @{thm CollectI}, |
60728 | 123 |
CONJ_WRAP' (fn thm => EVERY' [rtac ctxt (thm RS ord_eq_le_trans), |
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61242
diff
changeset
|
124 |
rtac ctxt @{thm image_subsetI}, rtac ctxt @{thm Collect_case_prod_Grp_in}, |
60752 | 125 |
etac ctxt @{thm set_mp}, assume_tac ctxt]) |
54792 | 126 |
set_maps, |
60728 | 127 |
rtac ctxt @{thm predicate2I}, REPEAT_DETERM o eresolve_tac ctxt [@{thm GrpE}, exE, conjE], |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
128 |
hyp_subst_tac ctxt, |
60728 | 129 |
rtac ctxt @{thm relcomppI}, rtac ctxt @{thm conversepI}, |
53270 | 130 |
EVERY' (map2 (fn convol => fn map_id0 => |
60728 | 131 |
EVERY' [rtac ctxt @{thm GrpI}, |
132 |
rtac ctxt (@{thm box_equals} OF [map_cong0, map_comp RS sym, map_id0]), |
|
133 |
REPEAT_DETERM_N n o rtac ctxt (convol RS fun_cong), |
|
63399 | 134 |
REPEAT_DETERM o eresolve_tac ctxt @{thms CollectE conjE}, |
135 |
rtac ctxt @{thm CollectI}, |
|
49495 | 136 |
CONJ_WRAP' (fn thm => |
60728 | 137 |
EVERY' [rtac ctxt ord_eq_le_trans, rtac ctxt thm, rtac ctxt @{thm image_subsetI}, |
60752 | 138 |
rtac ctxt @{thm convol_mem_GrpI}, etac ctxt set_mp, assume_tac ctxt]) |
54792 | 139 |
set_maps]) |
53285 | 140 |
@{thms fst_convol snd_convol} [map_id, refl])] 1 |
49284 | 141 |
end; |
142 |
||
60728 | 143 |
fun mk_rel_eq_tac ctxt n rel_Grp rel_cong map_id0 = |
144 |
(EVERY' (rtac ctxt (rel_cong RS trans) :: replicate n (rtac ctxt @{thm eq_alt})) THEN' |
|
145 |
rtac ctxt (rel_Grp RSN (2, @{thm box_equals[OF _ sym sym[OF eq_alt]]})) THEN' |
|
62617 | 146 |
(if n = 0 then SELECT_GOAL (unfold_thms_tac ctxt (no_refl [map_id0])) THEN' rtac ctxt refl |
60728 | 147 |
else EVERY' [rtac ctxt @{thm arg_cong2[of _ _ _ _ "Grp"]}, |
63399 | 148 |
rtac ctxt @{thm equalityI}, rtac ctxt subset_UNIV, |
149 |
rtac ctxt @{thm subsetI}, rtac ctxt @{thm CollectI}, |
|
60728 | 150 |
CONJ_WRAP' (K (rtac ctxt subset_UNIV)) (1 upto n), rtac ctxt map_id0])) 1; |
49284 | 151 |
|
57932 | 152 |
fun mk_rel_map0_tac ctxt live rel_compp rel_conversep rel_Grp map_id = |
153 |
if live = 0 then |
|
154 |
HEADGOAL (Goal.conjunction_tac) THEN |
|
155 |
unfold_thms_tac ctxt @{thms id_apply} THEN |
|
60728 | 156 |
ALLGOALS (rtac ctxt refl) |
57932 | 157 |
else |
158 |
let |
|
159 |
val ks = 1 upto live; |
|
160 |
in |
|
161 |
Goal.conjunction_tac 1 THEN |
|
162 |
unfold_thms_tac ctxt [rel_compp, rel_conversep, rel_Grp, @{thm vimage2p_Grp}] THEN |
|
60728 | 163 |
TRYALL (EVERY' [rtac ctxt iffI, rtac ctxt @{thm relcomppI}, rtac ctxt @{thm GrpI}, |
63399 | 164 |
resolve_tac ctxt [map_id, refl], rtac ctxt @{thm CollectI}, |
61760 | 165 |
CONJ_WRAP' (K (rtac ctxt @{thm subset_UNIV})) ks, rtac ctxt @{thm relcomppI}, |
166 |
assume_tac ctxt, rtac ctxt @{thm conversepI}, rtac ctxt @{thm GrpI}, |
|
63399 | 167 |
resolve_tac ctxt [map_id, refl], rtac ctxt @{thm CollectI}, |
60728 | 168 |
CONJ_WRAP' (K (rtac ctxt @{thm subset_UNIV})) ks, |
59498
50b60f501b05
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents:
58446
diff
changeset
|
169 |
REPEAT_DETERM o eresolve_tac ctxt @{thms relcomppE conversepE GrpE}, |
60752 | 170 |
dtac ctxt (trans OF [sym, map_id]), hyp_subst_tac ctxt, assume_tac ctxt]) |
57932 | 171 |
end; |
172 |
||
60728 | 173 |
fun mk_rel_mono_tac ctxt rel_OO_Grps in_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
|
174 |
let |
66fa0f602cc4
more robust tactics (don't use unfolding when RHS might contain schematics not contained on the LHS)
traytel
parents:
52813
diff
changeset
|
175 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
60728 | 176 |
else rtac ctxt (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
177 |
rtac ctxt (hd rel_OO_Grps RS sym RSN (2, ord_le_eq_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
|
178 |
in |
60728 | 179 |
EVERY' [rel_OO_Grps_tac, rtac ctxt @{thm relcompp_mono}, rtac ctxt @{thm iffD2[OF conversep_mono]}, |
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61242
diff
changeset
|
180 |
rtac ctxt @{thm Grp_mono}, rtac ctxt in_mono, REPEAT_DETERM o etac ctxt @{thm Collect_case_prod_mono}, |
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61242
diff
changeset
|
181 |
rtac ctxt @{thm Grp_mono}, rtac ctxt in_mono, REPEAT_DETERM o etac ctxt @{thm Collect_case_prod_mono}] 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
|
182 |
end; |
49284 | 183 |
|
55197 | 184 |
fun mk_rel_conversep_le_tac ctxt rel_OO_Grps rel_eq map_cong0 map_comp set_maps = |
49284 | 185 |
let |
54792 | 186 |
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
|
187 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
60728 | 188 |
else rtac ctxt (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
189 |
rtac ctxt (hd rel_OO_Grps RS sym RS @{thm arg_cong[of _ _ conversep]} RSN (2, ord_le_eq_trans)); |
|
49284 | 190 |
in |
60728 | 191 |
if null set_maps then rtac ctxt (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
|
192 |
else |
60728 | 193 |
EVERY' [rel_OO_Grps_tac, rtac ctxt @{thm predicate2I}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
194 |
REPEAT_DETERM o |
63399 | 195 |
eresolve_tac ctxt @{thms CollectE exE conjE GrpE relcomppE conversepE}, |
60728 | 196 |
hyp_subst_tac ctxt, rtac ctxt @{thm conversepI}, rtac ctxt @{thm relcomppI}, rtac ctxt @{thm conversepI}, |
197 |
EVERY' (map (fn thm => EVERY' [rtac ctxt @{thm GrpI}, rtac ctxt sym, rtac ctxt trans, |
|
198 |
rtac ctxt map_cong0, REPEAT_DETERM_N n o rtac ctxt thm, |
|
63399 | 199 |
rtac ctxt (map_comp RS sym), rtac ctxt @{thm CollectI}, |
60728 | 200 |
CONJ_WRAP' (fn thm => EVERY' [rtac ctxt (thm RS ord_eq_le_trans), |
201 |
etac ctxt @{thm flip_pred}]) set_maps]) [@{thm snd_fst_flip}, @{thm fst_snd_flip}])] 1 |
|
49284 | 202 |
end; |
203 |
||
60728 | 204 |
fun mk_rel_conversep_tac ctxt le_conversep rel_mono = |
205 |
EVERY' [rtac ctxt @{thm antisym}, rtac ctxt le_conversep, rtac ctxt @{thm xt1(6)}, rtac ctxt conversep_shift, |
|
206 |
rtac ctxt le_conversep, rtac ctxt @{thm iffD2[OF conversep_mono]}, rtac ctxt rel_mono, |
|
207 |
REPEAT_DETERM o rtac ctxt @{thm eq_refl[OF sym[OF conversep_conversep]]}] 1; |
|
49284 | 208 |
|
55197 | 209 |
fun mk_rel_OO_le_tac ctxt rel_OO_Grps rel_eq map_cong0 map_comp set_maps = |
49284 | 210 |
let |
54792 | 211 |
val n = length set_maps; |
63399 | 212 |
fun in_tac nthO_in = rtac ctxt @{thm CollectI} THEN' |
60728 | 213 |
CONJ_WRAP' (fn thm => EVERY' [rtac ctxt (thm RS ord_eq_le_trans), |
60752 | 214 |
rtac ctxt @{thm image_subsetI}, rtac ctxt nthO_in, etac ctxt set_mp, assume_tac ctxt]) 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
|
215 |
val rel_OO_Grps_tac = if null rel_OO_Grps then K all_tac |
60728 | 216 |
else rtac ctxt (hd rel_OO_Grps RS ord_eq_le_trans) THEN' |
67399 | 217 |
rtac ctxt (@{thm arg_cong2[of _ _ _ _ "(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
|
218 |
(2, ord_le_eq_trans)); |
49284 | 219 |
in |
60728 | 220 |
if null set_maps then rtac ctxt (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
|
221 |
else |
60728 | 222 |
EVERY' [rel_OO_Grps_tac, rtac ctxt @{thm predicate2I}, |
63399 | 223 |
REPEAT_DETERM o eresolve_tac ctxt @{thms CollectE exE conjE GrpE relcomppE conversepE}, |
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
224 |
hyp_subst_tac ctxt, |
60728 | 225 |
rtac ctxt @{thm relcomppI}, rtac ctxt @{thm relcomppI}, rtac ctxt @{thm conversepI}, rtac ctxt @{thm GrpI}, |
226 |
rtac ctxt trans, rtac ctxt map_comp, rtac ctxt sym, rtac ctxt map_cong0, |
|
227 |
REPEAT_DETERM_N n o rtac ctxt @{thm fst_fstOp}, |
|
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
228 |
in_tac @{thm fstOp_in}, |
60728 | 229 |
rtac ctxt @{thm GrpI}, rtac ctxt trans, rtac ctxt map_comp, rtac ctxt map_cong0, |
230 |
REPEAT_DETERM_N n o EVERY' [rtac ctxt trans, rtac ctxt o_apply, |
|
63399 | 231 |
rtac ctxt @{thm ballE}, rtac ctxt subst, |
60752 | 232 |
rtac ctxt @{thm csquare_def}, rtac ctxt @{thm csquare_fstOp_sndOp}, assume_tac ctxt, |
233 |
etac ctxt notE, etac ctxt set_mp, assume_tac ctxt], |
|
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
234 |
in_tac @{thm fstOp_in}, |
60728 | 235 |
rtac ctxt @{thm relcomppI}, rtac ctxt @{thm conversepI}, rtac ctxt @{thm GrpI}, |
236 |
rtac ctxt trans, rtac ctxt map_comp, rtac ctxt map_cong0, |
|
237 |
REPEAT_DETERM_N n o rtac ctxt o_apply, |
|
51893
596baae88a88
got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents:
51798
diff
changeset
|
238 |
in_tac @{thm sndOp_in}, |
60728 | 239 |
rtac ctxt @{thm GrpI}, rtac ctxt trans, rtac ctxt map_comp, rtac ctxt sym, rtac ctxt map_cong0, |
240 |
REPEAT_DETERM_N n o rtac ctxt @{thm snd_sndOp}, |
|
54841
af71b753c459
express weak pullback property of bnfs only in terms of the relator
traytel
parents:
54792
diff
changeset
|
241 |
in_tac @{thm sndOp_in}] 1 |
49284 | 242 |
end; |
243 |
||
57967 | 244 |
fun mk_rel_mono_strong0_tac ctxt in_rel set_maps = |
60752 | 245 |
if null set_maps then assume_tac ctxt 1 |
51916 | 246 |
else |
54998 | 247 |
unfold_tac ctxt [in_rel] THEN |
63399 | 248 |
REPEAT_DETERM (eresolve_tac ctxt @{thms exE CollectE conjE} 1) THEN |
51916 | 249 |
hyp_subst_tac ctxt 1 THEN |
60728 | 250 |
EVERY' [rtac ctxt exI, rtac ctxt @{thm conjI[OF CollectI conjI[OF refl refl]]}, |
55163 | 251 |
CONJ_WRAP' (fn thm => |
60752 | 252 |
(etac ctxt (@{thm Collect_split_mono_strong} OF [thm, thm]) THEN' assume_tac ctxt)) |
55163 | 253 |
set_maps] 1; |
51916 | 254 |
|
58104 | 255 |
fun mk_rel_transfer_tac ctxt in_rel rel_map rel_mono_strong = |
256 |
let |
|
257 |
fun last_tac iffD = |
|
60728 | 258 |
HEADGOAL (etac ctxt rel_mono_strong) THEN |
259 |
REPEAT_DETERM (HEADGOAL (etac ctxt (@{thm predicate2_transferD} RS iffD) THEN' |
|
60752 | 260 |
REPEAT_DETERM o assume_tac ctxt)); |
58104 | 261 |
in |
60728 | 262 |
REPEAT_DETERM (HEADGOAL (rtac ctxt rel_funI)) THEN |
263 |
(HEADGOAL (hyp_subst_tac ctxt THEN' rtac ctxt refl) ORELSE |
|
59498
50b60f501b05
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents:
58446
diff
changeset
|
264 |
REPEAT_DETERM (HEADGOAL (eresolve_tac ctxt (Tactic.make_elim (in_rel RS iffD1) :: |
58104 | 265 |
@{thms exE conjE CollectE}))) THEN |
67222 | 266 |
HEADGOAL (hyp_subst_tac ctxt) THEN |
267 |
REPEAT_DETERM (HEADGOAL (resolve_tac ctxt (maps (fn thm => |
|
268 |
[thm RS trans, thm RS @{thm trans[rotated, OF sym]}]) rel_map))) THEN |
|
269 |
HEADGOAL (rtac ctxt iffI) THEN |
|
67223 | 270 |
last_tac iffD1 THEN last_tac iffD2) |
58104 | 271 |
end; |
272 |
||
55197 | 273 |
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
|
274 |
let |
53290 | 275 |
val n = length set_maps; |
63399 | 276 |
val in_tac = |
277 |
if n = 0 then rtac ctxt @{thm UNIV_I} |
|
278 |
else |
|
279 |
rtac ctxt @{thm CollectI} THEN' CONJ_WRAP' (fn thm => |
|
280 |
etac ctxt (thm RS |
|
281 |
@{thm ord_eq_le_trans[OF _ subset_trans[OF image_mono convol_image_vimage2p]]})) |
|
282 |
set_maps; |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
283 |
in |
60728 | 284 |
REPEAT_DETERM_N n (HEADGOAL (rtac ctxt rel_funI)) THEN |
55945 | 285 |
unfold_thms_tac ctxt @{thms rel_fun_iff_leq_vimage2p} THEN |
60752 | 286 |
HEADGOAL (EVERY' [rtac ctxt @{thm order_trans}, rtac ctxt rel_mono, |
287 |
REPEAT_DETERM_N n o assume_tac ctxt, |
|
60728 | 288 |
rtac ctxt @{thm predicate2I}, dtac ctxt (in_rel RS iffD1), |
63399 | 289 |
REPEAT_DETERM o eresolve_tac ctxt @{thms exE CollectE conjE}, hyp_subst_tac ctxt, |
60728 | 290 |
rtac ctxt @{thm vimage2pI}, rtac ctxt (in_rel RS iffD2), rtac ctxt exI, rtac ctxt conjI, in_tac, |
291 |
rtac ctxt conjI, |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
292 |
EVERY' (map (fn convol => |
60728 | 293 |
rtac ctxt (@{thm box_equals} OF [map_cong0, map_comp RS sym, map_comp RS sym]) THEN' |
294 |
REPEAT_DETERM_N n o rtac ctxt (convol RS fun_cong)) @{thms fst_convol snd_convol})]) |
|
52719
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
295 |
end; |
480a3479fa47
transfer rule for map (not yet registered as a transfer rule)
traytel
parents:
52659
diff
changeset
|
296 |
|
55197 | 297 |
fun mk_in_bd_tac ctxt live surj_imp_ordLeq_inst map_comp map_id map_cong0 set_maps set_bds |
298 |
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
|
299 |
if live = 0 then |
60728 | 300 |
rtac ctxt @{thm ordLeq_transitive[OF ordLeq_csum2[OF card_of_Card_order] |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
301 |
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
|
302 |
else |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
303 |
let |
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
304 |
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
|
305 |
val inserts = |
57970 | 306 |
map (fn set_bd => |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
307 |
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
|
308 |
[set_bd, bd_Card_order RS @{thm card_of_Field_ordIso} RS @{thm ordIso_symmetric}]]) |
57970 | 309 |
set_bds; |
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
310 |
in |
60728 | 311 |
EVERY' [rtac ctxt (Drule.rotate_prems 1 ctrans), rtac ctxt @{thm cprod_cinfinite_bound}, |
312 |
rtac ctxt (ctrans OF @{thms ordLeq_csum2 ordLeq_cexp2}), rtac ctxt @{thm card_of_Card_order}, |
|
313 |
rtac ctxt @{thm ordLeq_csum2}, rtac ctxt @{thm Card_order_ctwo}, rtac ctxt @{thm Card_order_csum}, |
|
314 |
rtac ctxt @{thm ordIso_ordLeq_trans}, rtac ctxt @{thm cexp_cong1}, |
|
315 |
if live = 1 then rtac ctxt @{thm ordIso_refl[OF Card_order_csum]} |
|
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
316 |
else |
60728 | 317 |
REPEAT_DETERM_N (live - 2) o rtac ctxt @{thm ordIso_transitive[OF csum_cong2]} THEN' |
318 |
REPEAT_DETERM_N (live - 1) o rtac ctxt @{thm csum_csum}, |
|
319 |
rtac ctxt bd_Card_order, rtac ctxt (@{thm cexp_mono2_Cnotzero} RS ctrans), rtac ctxt @{thm ordLeq_csum1}, |
|
320 |
rtac ctxt bd_Card_order, rtac ctxt @{thm Card_order_csum}, rtac ctxt bd_Cnotzero, |
|
321 |
rtac ctxt @{thm csum_Cfinite_cexp_Cinfinite}, |
|
322 |
rtac ctxt (if live = 1 then @{thm card_of_Card_order} else @{thm Card_order_csum}), |
|
323 |
CONJ_WRAP_GEN' (rtac ctxt @{thm Cfinite_csum}) (K (rtac ctxt @{thm Cfinite_cone})) set_maps, |
|
324 |
rtac ctxt bd'_Cinfinite, rtac ctxt @{thm card_of_Card_order}, |
|
325 |
rtac ctxt @{thm Card_order_cexp}, rtac ctxt @{thm Cinfinite_cexp}, rtac ctxt @{thm ordLeq_csum2}, |
|
326 |
rtac ctxt @{thm Card_order_ctwo}, rtac ctxt bd'_Cinfinite, |
|
327 |
rtac ctxt (Drule.rotate_prems 1 (@{thm cprod_mono2} RSN (2, ctrans))), |
|
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
328 |
REPEAT_DETERM_N (live - 1) o |
60728 | 329 |
(rtac ctxt (bd_Cinfinite RS @{thm cprod_cexp_csum_cexp_Cinfinite} RSN (2, ctrans)) THEN' |
330 |
rtac ctxt @{thm ordLeq_ordIso_trans[OF cprod_mono2 ordIso_symmetric[OF cprod_cexp]]}), |
|
331 |
rtac ctxt @{thm ordLeq_refl[OF Card_order_cexp]}] 1 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
|
332 |
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
|
333 |
unfold_thms_tac ctxt @{thms cprod_def Field_card_of} THEN |
63399 | 334 |
EVERY' [rtac ctxt (Drule.rotate_prems 1 ctrans), rtac ctxt surj_imp_ordLeq_inst, |
335 |
rtac ctxt @{thm subsetI}, |
|
61841
4d3527b94f2a
more general types Proof.method / context_tactic;
wenzelm
parents:
61760
diff
changeset
|
336 |
Method.insert_tac ctxt inserts, REPEAT_DETERM o dtac ctxt meta_spec, |
63399 | 337 |
REPEAT_DETERM o eresolve_tac ctxt [exE, Tactic.make_elim conjunct1], |
338 |
etac ctxt @{thm CollectE}, |
|
52635
4f84b730c489
got rid of in_bd BNF property (derivable from set_bd+map_cong+map_comp+map_id)
traytel
parents:
51916
diff
changeset
|
339 |
if live = 1 then K all_tac |
60728 | 340 |
else REPEAT_DETERM_N (live - 2) o (etac ctxt conjE THEN' rotate_tac ~1) THEN' etac ctxt conjE, |
341 |
rtac ctxt (Drule.rotate_prems 1 @{thm image_eqI}), rtac ctxt @{thm SigmaI}, rtac ctxt @{thm UNIV_I}, |
|
342 |
CONJ_WRAP_GEN' (rtac ctxt @{thm SigmaI}) |
|
60752 | 343 |
(K (etac ctxt @{thm If_the_inv_into_in_Func} THEN' assume_tac ctxt)) set_maps, |
60728 | 344 |
rtac ctxt sym, |
345 |
rtac ctxt (Drule.rotate_prems 1 |
|
55990 | 346 |
((@{thm box_equals} OF [map_cong0 OF replicate live @{thm If_the_inv_into_f_f}, |
53288 | 347 |
map_comp RS sym, map_id]) RSN (2, trans))), |
60752 | 348 |
REPEAT_DETERM_N (2 * live) o assume_tac ctxt, |
60728 | 349 |
REPEAT_DETERM_N live o rtac ctxt (@{thm prod.case} RS trans), |
350 |
rtac ctxt refl, |
|
63399 | 351 |
rtac ctxt @{thm surj_imp_ordLeq}, |
352 |
rtac ctxt @{thm subsetI}, |
|
353 |
rtac ctxt (Drule.rotate_prems 1 @{thm image_eqI}), |
|
354 |
REPEAT_DETERM o eresolve_tac ctxt @{thms CollectE conjE}, rtac ctxt @{thm 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
|
355 |
CONJ_WRAP' (fn thm => |
60728 | 356 |
rtac ctxt (thm RS ord_eq_le_trans) THEN' etac ctxt @{thm subset_trans[OF image_mono Un_upper1]}) |
53290 | 357 |
set_maps, |
60728 | 358 |
rtac ctxt sym, |
359 |
rtac ctxt (@{thm box_equals} OF [map_cong0 OF replicate live @{thm fun_cong[OF case_sum_o_inj(1)]}, |
|
53288 | 360 |
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
|
361 |
end; |
51916 | 362 |
|
55197 | 363 |
fun mk_trivial_wit_tac ctxt wit_defs set_maps = |
60752 | 364 |
unfold_thms_tac ctxt wit_defs THEN |
365 |
HEADGOAL (EVERY' (map (fn thm => |
|
63399 | 366 |
dtac ctxt (thm RS @{thm equalityD1} RS set_mp) THEN' |
367 |
etac ctxt @{thm imageE} THEN' assume_tac ctxt) set_maps)) THEN |
|
60752 | 368 |
ALLGOALS (assume_tac ctxt); |
54189
c0186a0d8cb3
define a trivial nonemptiness witness if none is provided
traytel
parents:
53562
diff
changeset
|
369 |
|
58106 | 370 |
fun mk_set_transfer_tac ctxt in_rel set_maps = |
371 |
Goal.conjunction_tac 1 THEN |
|
60728 | 372 |
EVERY (map (fn set_map => HEADGOAL (rtac ctxt rel_funI) THEN |
59498
50b60f501b05
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents:
58446
diff
changeset
|
373 |
REPEAT_DETERM (HEADGOAL (eresolve_tac ctxt (Tactic.make_elim (in_rel RS iffD1) :: |
58106 | 374 |
@{thms exE conjE CollectE}))) THEN |
60728 | 375 |
HEADGOAL (hyp_subst_tac ctxt THEN' rtac ctxt (@{thm iffD2[OF arg_cong2]} OF [set_map, set_map]) THEN' |
376 |
rtac ctxt @{thm rel_setI}) THEN |
|
63399 | 377 |
REPEAT (HEADGOAL (etac ctxt @{thm imageE} THEN' dtac ctxt @{thm set_mp} THEN' assume_tac ctxt THEN' |
59498
50b60f501b05
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents:
58446
diff
changeset
|
378 |
REPEAT_DETERM o (eresolve_tac ctxt @{thms CollectE case_prodE}) THEN' hyp_subst_tac ctxt THEN' |
63399 | 379 |
rtac ctxt @{thm bexI} THEN' etac ctxt @{thm subst_Pair[OF _ refl]} THEN' etac ctxt @{thm imageI}))) |
380 |
set_maps); |
|
58106 | 381 |
|
61242 | 382 |
fun mk_rel_cong_tac ctxt (eqs, prems) mono = |
383 |
let |
|
384 |
fun mk_tac thm = etac ctxt thm THEN_ALL_NEW assume_tac ctxt; |
|
62324 | 385 |
fun mk_tacs iffD = etac ctxt mono :: |
61242 | 386 |
map (fn thm => (unfold_thms ctxt @{thms simp_implies_def} thm RS iffD) |
387 |
|> Drule.rotate_prems ~1 |> mk_tac) prems; |
|
388 |
in |
|
389 |
unfold_thms_tac ctxt eqs THEN |
|
390 |
HEADGOAL (EVERY' (rtac ctxt iffI :: mk_tacs iffD1 @ mk_tacs iffD2)) |
|
391 |
end; |
|
392 |
||
62324 | 393 |
fun subst_conv ctxt thm = |
74545 | 394 |
(Conv.arg_conv o Conv.arg_conv) |
395 |
(Conv.top_sweep_rewrs_conv [safe_mk_meta_eq thm] ctxt); |
|
62324 | 396 |
|
397 |
fun mk_rel_eq_onp_tac ctxt pred_def map_id0 rel_Grp = |
|
398 |
HEADGOAL (EVERY' |
|
399 |
[SELECT_GOAL (unfold_thms_tac ctxt (pred_def :: @{thms UNIV_def eq_onp_Grp Ball_Collect})), |
|
400 |
CONVERSION (subst_conv ctxt (map_id0 RS sym)), |
|
401 |
rtac ctxt (unfold_thms ctxt @{thms UNIV_def} rel_Grp)]); |
|
402 |
||
403 |
fun mk_pred_mono_strong0_tac ctxt pred_rel rel_mono_strong0 = |
|
404 |
unfold_thms_tac ctxt [pred_rel] THEN |
|
405 |
HEADGOAL (etac ctxt rel_mono_strong0 THEN_ALL_NEW etac ctxt @{thm eq_onp_mono0}); |
|
406 |
||
63714 | 407 |
fun mk_pred_mono_tac ctxt rel_eq_onp rel_mono = |
408 |
unfold_thms_tac ctxt (map mk_sym [@{thm eq_onp_mono_iff}, rel_eq_onp]) THEN |
|
409 |
HEADGOAL (rtac ctxt rel_mono THEN_ALL_NEW assume_tac ctxt); |
|
410 |
||
62329 | 411 |
fun mk_pred_transfer_tac ctxt n in_rel pred_map pred_cong = |
412 |
HEADGOAL (EVERY' [REPEAT_DETERM_N (n + 1) o rtac ctxt rel_funI, dtac ctxt (in_rel RS iffD1), |
|
63399 | 413 |
REPEAT_DETERM o eresolve_tac ctxt @{thms exE conjE CollectE}, hyp_subst_tac ctxt, |
62329 | 414 |
rtac ctxt (box_equals OF [@{thm _}, pred_map RS sym, pred_map RS sym]), |
415 |
rtac ctxt (refl RS pred_cong), REPEAT_DETERM_N n o |
|
67399 | 416 |
(etac ctxt @{thm rel_fun_Collect_case_prodD[where B="(=)"]} THEN_ALL_NEW assume_tac ctxt)]); |
62329 | 417 |
|
49284 | 418 |
end; |