author | haftmann |
Thu, 06 Aug 2015 23:56:48 +0200 | |
changeset 60867 | 86e7560e07d0 |
parent 60801 | 7664e0916eec |
child 61144 | 5e94dfead1c2 |
permissions | -rw-r--r-- |
19494 | 1 |
(* Title: HOL/Nominal/nominal_permeq.ML |
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
2 |
Author: Christian Urban, TU Muenchen |
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
3 |
Author: Julien Narboux, TU Muenchen |
17870 | 4 |
|
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
5 |
Methods for simplifying permutations and for analysing equations |
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
6 |
involving permutations. |
19494 | 7 |
*) |
17870 | 8 |
|
20431 | 9 |
(* |
10 |
FIXMES: |
|
11 |
||
12 |
- allow the user to give an explicit set S in the |
|
13 |
fresh_guess tactic which is then verified |
|
14 |
||
15 |
- the perm_compose tactic does not do an "outermost |
|
16 |
rewriting" and can therefore not deal with goals |
|
17 |
like |
|
18 |
||
19 |
[(a,b)] o pi1 o pi2 = .... |
|
20 |
||
21 |
rather it tries to permute pi1 over pi2, which |
|
22 |
results in a failure when used with the |
|
23 |
perm_(full)_simp tactics |
|
24 |
||
25 |
*) |
|
26 |
||
27 |
||
19987
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
28 |
signature NOMINAL_PERMEQ = |
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
29 |
sig |
25997 | 30 |
val perm_simproc_fun : simproc |
31 |
val perm_simproc_app : simproc |
|
32 |
||
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
33 |
val perm_simp_tac : Proof.context -> int -> tactic |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
34 |
val perm_extend_simp_tac : Proof.context -> int -> tactic |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
35 |
val supports_tac : Proof.context -> int -> tactic |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
36 |
val finite_guess_tac : Proof.context -> int -> tactic |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
37 |
val fresh_guess_tac : Proof.context -> int -> tactic |
17870 | 38 |
|
30549 | 39 |
val perm_simp_meth : (Proof.context -> Proof.method) context_parser |
40 |
val perm_simp_meth_debug : (Proof.context -> Proof.method) context_parser |
|
41 |
val perm_extend_simp_meth : (Proof.context -> Proof.method) context_parser |
|
42 |
val perm_extend_simp_meth_debug : (Proof.context -> Proof.method) context_parser |
|
43 |
val supports_meth : (Proof.context -> Proof.method) context_parser |
|
44 |
val supports_meth_debug : (Proof.context -> Proof.method) context_parser |
|
45 |
val finite_guess_meth : (Proof.context -> Proof.method) context_parser |
|
46 |
val finite_guess_meth_debug : (Proof.context -> Proof.method) context_parser |
|
47 |
val fresh_guess_meth : (Proof.context -> Proof.method) context_parser |
|
48 |
val fresh_guess_meth_debug : (Proof.context -> Proof.method) context_parser |
|
19987
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
49 |
end |
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
50 |
|
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
51 |
structure NominalPermeq : NOMINAL_PERMEQ = |
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
52 |
struct |
b97607d4d9a5
- put declarations inside a structure (NominalPermeq)
berghofe
parents:
19858
diff
changeset
|
53 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
54 |
(* some lemmas needed below *) |
24519 | 55 |
val finite_emptyI = @{thm "finite.emptyI"}; |
56 |
val finite_Un = @{thm "finite_Un"}; |
|
57 |
val conj_absorb = @{thm "conj_absorb"}; |
|
58 |
val not_false = @{thm "not_False_eq_True"} |
|
44684
8dde3352d5c4
assert Pure equations for theorem references; tuned
haftmann
parents:
43278
diff
changeset
|
59 |
val perm_fun_def = Simpdata.mk_eq @{thm "Nominal.perm_fun_def"}; |
24519 | 60 |
val perm_eq_app = @{thm "Nominal.pt_fun_app_eq"}; |
44684
8dde3352d5c4
assert Pure equations for theorem references; tuned
haftmann
parents:
43278
diff
changeset
|
61 |
val supports_def = Simpdata.mk_eq @{thm "Nominal.supports_def"}; |
8dde3352d5c4
assert Pure equations for theorem references; tuned
haftmann
parents:
43278
diff
changeset
|
62 |
val fresh_def = Simpdata.mk_eq @{thm "Nominal.fresh_def"}; |
24519 | 63 |
val fresh_prod = @{thm "Nominal.fresh_prod"}; |
64 |
val fresh_unit = @{thm "Nominal.fresh_unit"}; |
|
65 |
val supports_rule = @{thm "supports_finite"}; |
|
66 |
val supp_prod = @{thm "supp_prod"}; |
|
67 |
val supp_unit = @{thm "supp_unit"}; |
|
68 |
val pt_perm_compose_aux = @{thm "pt_perm_compose_aux"}; |
|
69 |
val cp1_aux = @{thm "cp1_aux"}; |
|
70 |
val perm_aux_fold = @{thm "perm_aux_fold"}; |
|
71 |
val supports_fresh_rule = @{thm "supports_fresh"}; |
|
21669 | 72 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
73 |
(* needed in the process of fully simplifying permutations *) |
24519 | 74 |
val strong_congs = [@{thm "if_cong"}] |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
75 |
(* needed to avoid warnings about overwritten congs *) |
24519 | 76 |
val weak_congs = [@{thm "if_weak_cong"}] |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
77 |
|
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
78 |
(* debugging *) |
56492 | 79 |
fun DEBUG ctxt (msg,tac) = |
56491 | 80 |
CHANGED (EVERY [print_tac ctxt ("before "^msg), tac, print_tac ctxt ("after "^msg)]); |
56492 | 81 |
fun NO_DEBUG _ (_,tac) = CHANGED tac; |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
82 |
|
19477 | 83 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
84 |
(* simproc that deals with instances of permutations in front *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
85 |
(* of applications; just adding this rule to the simplifier *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
86 |
(* would loop; it also needs careful tuning with the simproc *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
87 |
(* for functions to avoid further possibilities for looping *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
88 |
fun perm_simproc_app' ctxt redex = |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
89 |
let |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
90 |
val thy = Proof_Context.theory_of ctxt; |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
91 |
(* the "application" case is only applicable when the head of f is not a *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
92 |
(* constant or when (f x) is a permuation with two or more arguments *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
93 |
fun applicable_app t = |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
94 |
(case (strip_comb t) of |
56253 | 95 |
(Const (@{const_name Nominal.perm},_),ts) => (length ts) >= 2 |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
96 |
| (Const _,_) => false |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
97 |
| _ => true) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
98 |
in |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
99 |
case redex of |
19169
20a73345dd6e
fixed a problem where a permutation is not analysed
urbanc
parents:
19163
diff
changeset
|
100 |
(* case pi o (f x) == (pi o f) (pi o x) *) |
56253 | 101 |
(Const(@{const_name Nominal.perm}, |
102 |
Type(@{type_name fun}, |
|
103 |
[Type(@{type_name list}, [Type(@{type_name prod},[Type(n,_),_])]),_])) $ pi $ (f $ x)) => |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
104 |
(if (applicable_app f) then |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
105 |
let |
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30280
diff
changeset
|
106 |
val name = Long_Name.base_name n |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
107 |
val at_inst = Global_Theory.get_thm thy ("at_" ^ name ^ "_inst") |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
108 |
val pt_inst = Global_Theory.get_thm thy ("pt_" ^ name ^ "_inst") |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
109 |
in SOME ((at_inst RS (pt_inst RS perm_eq_app)) RS eq_reflection) end |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
110 |
else NONE) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
111 |
| _ => NONE |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
112 |
end |
19139 | 113 |
|
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
37678
diff
changeset
|
114 |
val perm_simproc_app = Simplifier.simproc_global @{theory} "perm_simproc_app" |
25997 | 115 |
["Nominal.perm pi x"] perm_simproc_app'; |
116 |
||
24519 | 117 |
(* a simproc that deals with permutation instances in front of functions *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
118 |
fun perm_simproc_fun' ctxt redex = |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
119 |
let |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
120 |
fun applicable_fun t = |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
121 |
(case (strip_comb t) of |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
122 |
(Abs _ ,[]) => true |
56253 | 123 |
| (Const (@{const_name Nominal.perm},_),_) => false |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
124 |
| (Const _, _) => true |
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
125 |
| _ => false) |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
126 |
in |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
127 |
case redex of |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
128 |
(* case pi o f == (%x. pi o (f ((rev pi)o x))) *) |
56253 | 129 |
(Const(@{const_name Nominal.perm},_) $ pi $ f) => |
44830 | 130 |
(if applicable_fun f then SOME perm_fun_def else NONE) |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
131 |
| _ => NONE |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
132 |
end |
19139 | 133 |
|
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
37678
diff
changeset
|
134 |
val perm_simproc_fun = Simplifier.simproc_global @{theory} "perm_simproc_fun" |
25997 | 135 |
["Nominal.perm pi x"] perm_simproc_fun'; |
136 |
||
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
137 |
(* function for simplyfying permutations *) |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
138 |
(* stac contains the simplifiation tactic that is *) |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
139 |
(* applied (see (no_asm) options below *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
140 |
fun perm_simp_gen stac dyn_thms eqvt_thms ctxt i = |
56230 | 141 |
("general simplification of permutations", fn st => SUBGOAL (fn _ => |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
142 |
let |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
143 |
val ctxt' = ctxt |
60359 | 144 |
addsimps (maps (Proof_Context.get_thms ctxt) dyn_thms @ eqvt_thms) |
25997 | 145 |
addsimprocs [perm_simproc_fun, perm_simproc_app] |
45620
f2a587696afb
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
wenzelm
parents:
44830
diff
changeset
|
146 |
|> fold Simplifier.del_cong weak_congs |
f2a587696afb
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
wenzelm
parents:
44830
diff
changeset
|
147 |
|> fold Simplifier.add_cong strong_congs |
19477 | 148 |
in |
56230 | 149 |
stac ctxt' i |
150 |
end) i st); |
|
19477 | 151 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
152 |
(* general simplification of permutations and permutation that arose from eqvt-problems *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
153 |
fun perm_simp stac ctxt = |
22610 | 154 |
let val simps = ["perm_swap","perm_fresh_fresh","perm_bij","perm_pi_simp","swap_simps"] |
155 |
in |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
156 |
perm_simp_gen stac simps [] ctxt |
22610 | 157 |
end; |
158 |
||
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
159 |
fun eqvt_simp stac ctxt = |
22610 | 160 |
let val simps = ["perm_swap","perm_fresh_fresh","perm_pi_simp"] |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
161 |
val eqvts_thms = NominalThmDecls.get_eqvt_thms ctxt; |
22610 | 162 |
in |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
163 |
perm_simp_gen stac simps eqvts_thms ctxt |
22610 | 164 |
end; |
22562
80b814fe284b
rename bij and fresh into bijs and freshs and lookup for eqvts lemma using the ml value instead of the name
narboux
parents:
22541
diff
changeset
|
165 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
166 |
|
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
167 |
(* main simplification tactics for permutations *) |
56491 | 168 |
fun perm_simp_tac_gen_i stac tactical ctxt i = DETERM (tactical ctxt (perm_simp stac ctxt i)); |
169 |
fun eqvt_simp_tac_gen_i stac tactical ctxt i = DETERM (tactical ctxt (eqvt_simp stac ctxt i)); |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
170 |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
171 |
val perm_simp_tac_i = perm_simp_tac_gen_i simp_tac |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
172 |
val perm_asm_simp_tac_i = perm_simp_tac_gen_i asm_simp_tac |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
173 |
val perm_full_simp_tac_i = perm_simp_tac_gen_i full_simp_tac |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
174 |
val perm_asm_lr_simp_tac_i = perm_simp_tac_gen_i asm_lr_simp_tac |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
175 |
val perm_asm_full_simp_tac_i = perm_simp_tac_gen_i asm_full_simp_tac |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
176 |
val eqvt_asm_full_simp_tac_i = eqvt_simp_tac_gen_i asm_full_simp_tac |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
177 |
|
19477 | 178 |
(* applies the perm_compose rule such that *) |
179 |
(* pi o (pi' o lhs) = rhs *) |
|
180 |
(* is transformed to *) |
|
181 |
(* (pi o pi') o (pi' o lhs) = rhs *) |
|
182 |
(* *) |
|
183 |
(* this rule would loop in the simplifier, so some trick is used with *) |
|
184 |
(* generating perm_aux'es for the outermost permutation and then un- *) |
|
185 |
(* folding the definition *) |
|
25997 | 186 |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
187 |
fun perm_compose_simproc' ctxt redex = |
25997 | 188 |
(case redex of |
56253 | 189 |
(Const (@{const_name Nominal.perm}, Type (@{type_name fun}, [Type (@{type_name list}, |
190 |
[Type (@{type_name Product_Type.prod}, [T as Type (tname,_),_])]),_])) $ pi1 $ (Const (@{const_name Nominal.perm}, |
|
191 |
Type (@{type_name fun}, [Type (@{type_name list}, [Type (@{type_name Product_Type.prod}, [U as Type (uname,_),_])]),_])) $ |
|
25997 | 192 |
pi2 $ t)) => |
19477 | 193 |
let |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
194 |
val thy = Proof_Context.theory_of ctxt |
30364
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30280
diff
changeset
|
195 |
val tname' = Long_Name.base_name tname |
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents:
30280
diff
changeset
|
196 |
val uname' = Long_Name.base_name uname |
25997 | 197 |
in |
198 |
if pi1 <> pi2 then (* only apply the composition rule in this case *) |
|
199 |
if T = U then |
|
60801 | 200 |
SOME (Thm.instantiate' |
59621
291934bac95e
Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents:
59582
diff
changeset
|
201 |
[SOME (Thm.global_ctyp_of thy (fastype_of t))] |
291934bac95e
Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents:
59582
diff
changeset
|
202 |
[SOME (Thm.global_cterm_of thy pi1), SOME (Thm.global_cterm_of thy pi2), SOME (Thm.global_cterm_of thy t)] |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
203 |
(mk_meta_eq ([Global_Theory.get_thm thy ("pt_"^tname'^"_inst"), |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
204 |
Global_Theory.get_thm thy ("at_"^tname'^"_inst")] MRS pt_perm_compose_aux))) |
25997 | 205 |
else |
60801 | 206 |
SOME (Thm.instantiate' |
59621
291934bac95e
Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents:
59582
diff
changeset
|
207 |
[SOME (Thm.global_ctyp_of thy (fastype_of t))] |
291934bac95e
Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents:
59582
diff
changeset
|
208 |
[SOME (Thm.global_cterm_of thy pi1), SOME (Thm.global_cterm_of thy pi2), SOME (Thm.global_cterm_of thy t)] |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
209 |
(mk_meta_eq (Global_Theory.get_thm thy ("cp_"^tname'^"_"^uname'^"_inst") RS |
25997 | 210 |
cp1_aux))) |
211 |
else NONE |
|
212 |
end |
|
213 |
| _ => NONE); |
|
19477 | 214 |
|
38715
6513ea67d95d
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents:
37678
diff
changeset
|
215 |
val perm_compose_simproc = Simplifier.simproc_global @{theory} "perm_compose" |
25997 | 216 |
["Nominal.perm pi1 (Nominal.perm pi2 t)"] perm_compose_simproc'; |
19477 | 217 |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
218 |
fun perm_compose_tac ctxt i = |
25997 | 219 |
("analysing permutation compositions on the lhs", |
220 |
fn st => EVERY |
|
60754 | 221 |
[resolve_tac ctxt [trans] i, |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
222 |
asm_full_simp_tac (empty_simpset ctxt addsimprocs [perm_compose_simproc]) i, |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
223 |
asm_full_simp_tac (put_simpset HOL_basic_ss ctxt addsimps [perm_aux_fold]) i] st); |
18012 | 224 |
|
58956
a816aa3ff391
proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);
wenzelm
parents:
56492
diff
changeset
|
225 |
fun apply_cong_tac ctxt i = ("application of congruence", cong_tac ctxt i); |
17870 | 226 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
227 |
|
19477 | 228 |
(* unfolds the definition of permutations *) |
229 |
(* applied to functions such that *) |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
230 |
(* pi o f = rhs *) |
19477 | 231 |
(* is transformed to *) |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
232 |
(* %x. pi o (f ((rev pi) o x)) = rhs *) |
60754 | 233 |
fun unfold_perm_fun_def_tac ctxt i = |
24519 | 234 |
("unfolding of permutations on functions", |
60754 | 235 |
resolve_tac ctxt [perm_fun_def RS meta_eq_to_obj_eq RS trans] i) |
17870 | 236 |
|
19477 | 237 |
(* applies the ext-rule such that *) |
238 |
(* *) |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
239 |
(* f = g goes to /\x. f x = g x *) |
60754 | 240 |
fun ext_fun_tac ctxt i = |
241 |
("extensionality expansion of functions", resolve_tac ctxt @{thms ext} i); |
|
17870 | 242 |
|
243 |
||
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
244 |
(* perm_extend_simp_tac_i is perm_simp plus additional tactics *) |
19477 | 245 |
(* to decide equation that come from support problems *) |
246 |
(* since it contains looping rules the "recursion" - depth is set *) |
|
247 |
(* to 10 - this seems to be sufficient in most cases *) |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
248 |
fun perm_extend_simp_tac_i tactical ctxt = |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
249 |
let fun perm_extend_simp_tac_aux tactical ctxt n = |
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
250 |
if n=0 then K all_tac |
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32733
diff
changeset
|
251 |
else DETERM o |
60754 | 252 |
(FIRST' |
253 |
[fn i => tactical ctxt ("splitting conjunctions on the rhs", resolve_tac ctxt [conjI] i), |
|
254 |
fn i => tactical ctxt (perm_simp asm_full_simp_tac ctxt i), |
|
255 |
fn i => tactical ctxt (perm_compose_tac ctxt i), |
|
256 |
fn i => tactical ctxt (apply_cong_tac ctxt i), |
|
257 |
fn i => tactical ctxt (unfold_perm_fun_def_tac ctxt i), |
|
258 |
fn i => tactical ctxt (ext_fun_tac ctxt i)] |
|
259 |
THEN_ALL_NEW (TRY o (perm_extend_simp_tac_aux tactical ctxt (n-1)))) |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
260 |
in perm_extend_simp_tac_aux tactical ctxt 10 end; |
19151 | 261 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
262 |
|
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
263 |
(* tactic that tries to solve "supports"-goals; first it *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
264 |
(* unfolds the support definition and strips off the *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
265 |
(* intros, then applies eqvt_simp_tac *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
266 |
fun supports_tac_i tactical ctxt i = |
18012 | 267 |
let |
36945 | 268 |
val simps = [supports_def, Thm.symmetric fresh_def, fresh_prod] |
17870 | 269 |
in |
56491 | 270 |
EVERY [tactical ctxt ("unfolding of supports ", simp_tac (put_simpset HOL_basic_ss ctxt addsimps simps) i), |
60754 | 271 |
tactical ctxt ("stripping of foralls ", REPEAT_DETERM (resolve_tac ctxt [allI] i)), |
272 |
tactical ctxt ("geting rid of the imps ", resolve_tac ctxt [impI] i), |
|
273 |
tactical ctxt ("eliminating conjuncts ", REPEAT_DETERM (eresolve_tac ctxt [conjE] i)), |
|
274 |
tactical ctxt ("applying eqvt_simp ", eqvt_simp_tac_gen_i asm_full_simp_tac tactical ctxt i)] |
|
17870 | 275 |
end; |
276 |
||
19151 | 277 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
278 |
(* tactic that guesses the finite-support of a goal *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
279 |
(* it first collects all free variables and tries to show *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
280 |
(* that the support of these free variables (op supports) *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
281 |
(* the goal *) |
20854 | 282 |
fun collect_vars i (Bound j) vs = if j < i then vs else insert (op =) (Bound (j - i)) vs |
283 |
| collect_vars i (v as Free _) vs = insert (op =) v vs |
|
284 |
| collect_vars i (v as Var _) vs = insert (op =) v vs |
|
19151 | 285 |
| collect_vars i (Const _) vs = vs |
286 |
| collect_vars i (Abs (_, _, t)) vs = collect_vars (i+1) t vs |
|
287 |
| collect_vars i (t $ u) vs = collect_vars i u (collect_vars i t vs); |
|
288 |
||
43278 | 289 |
(* FIXME proper SUBGOAL/CSUBGOAL instead of cprems_of etc. *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
290 |
fun finite_guess_tac_i tactical ctxt i st = |
42364 | 291 |
let val goal = nth (cprems_of st) (i - 1) |
19151 | 292 |
in |
59582 | 293 |
case Envir.eta_contract (Logic.strip_assums_concl (Thm.term_of goal)) of |
56253 | 294 |
_ $ (Const (@{const_name finite}, _) $ (Const (@{const_name Nominal.supp}, T) $ x)) => |
19151 | 295 |
let |
59582 | 296 |
val ps = Logic.strip_params (Thm.term_of goal); |
19151 | 297 |
val Ts = rev (map snd ps); |
298 |
val vs = collect_vars 0 x []; |
|
33244 | 299 |
val s = fold_rev (fn v => fn s => |
19151 | 300 |
HOLogic.pair_const (fastype_of1 (Ts, v)) (fastype_of1 (Ts, s)) $ v $ s) |
33244 | 301 |
vs HOLogic.unit; |
46219
426ed18eba43
discontinued old-style Term.list_abs in favour of plain Term.abs;
wenzelm
parents:
45620
diff
changeset
|
302 |
val s' = fold_rev Term.abs ps |
56253 | 303 |
(Const (@{const_name Nominal.supp}, fastype_of1 (Ts, s) --> |
44692
ccfc7c193d2b
modify nominal packages to better respect set/pred distinction
huffman
parents:
43278
diff
changeset
|
304 |
Term.range_type T) $ s); |
19151 | 305 |
val supports_rule' = Thm.lift_rule goal supports_rule; |
306 |
val _ $ (_ $ S $ _) = |
|
59582 | 307 |
Logic.strip_assums_concl (hd (Thm.prems_of supports_rule')); |
60787 | 308 |
val supports_rule'' = |
309 |
infer_instantiate ctxt |
|
310 |
[(#1 (dest_Var (head_of S)), Thm.cterm_of ctxt s')] supports_rule'; |
|
60359 | 311 |
val fin_supp = Proof_Context.get_thms ctxt "fin_supp" |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
312 |
val ctxt' = ctxt addsimps [supp_prod,supp_unit,finite_Un,finite_emptyI,conj_absorb]@fin_supp |
19151 | 313 |
in |
56491 | 314 |
(tactical ctxt ("guessing of the right supports-set", |
58956
a816aa3ff391
proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);
wenzelm
parents:
56492
diff
changeset
|
315 |
EVERY [compose_tac ctxt (false, supports_rule'', 2) i, |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
316 |
asm_full_simp_tac ctxt' (i+1), |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
317 |
supports_tac_i tactical ctxt i])) st |
19151 | 318 |
end |
319 |
| _ => Seq.empty |
|
320 |
end |
|
43278 | 321 |
handle General.Subscript => Seq.empty |
322 |
(* FIXME proper SUBGOAL/CSUBGOAL instead of cprems_of etc. *) |
|
19151 | 323 |
|
22595
293934e41dfd
make fresh_guess fail if it does not solve the subgoal
narboux
parents:
22578
diff
changeset
|
324 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
325 |
(* tactic that guesses whether an atom is fresh for an expression *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
326 |
(* it first collects all free variables and tries to show that the *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
327 |
(* support of these free variables (op supports) the goal *) |
43278 | 328 |
(* FIXME proper SUBGOAL/CSUBGOAL instead of cprems_of etc. *) |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
329 |
fun fresh_guess_tac_i tactical ctxt i st = |
19857 | 330 |
let |
42364 | 331 |
val goal = nth (cprems_of st) (i - 1) |
60359 | 332 |
val fin_supp = Proof_Context.get_thms ctxt "fin_supp" |
333 |
val fresh_atm = Proof_Context.get_thms ctxt "fresh_atm" |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
334 |
val ctxt1 = ctxt addsimps [Thm.symmetric fresh_def,fresh_prod,fresh_unit,conj_absorb,not_false]@fresh_atm |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
335 |
val ctxt2 = ctxt addsimps [supp_prod,supp_unit,finite_Un,finite_emptyI,conj_absorb]@fin_supp |
19857 | 336 |
in |
59582 | 337 |
case Logic.strip_assums_concl (Thm.term_of goal) of |
56253 | 338 |
_ $ (Const (@{const_name Nominal.fresh}, Type ("fun", [T, _])) $ _ $ t) => |
19857 | 339 |
let |
59582 | 340 |
val ps = Logic.strip_params (Thm.term_of goal); |
19857 | 341 |
val Ts = rev (map snd ps); |
342 |
val vs = collect_vars 0 t []; |
|
33244 | 343 |
val s = fold_rev (fn v => fn s => |
19857 | 344 |
HOLogic.pair_const (fastype_of1 (Ts, v)) (fastype_of1 (Ts, s)) $ v $ s) |
33244 | 345 |
vs HOLogic.unit; |
46219
426ed18eba43
discontinued old-style Term.list_abs in favour of plain Term.abs;
wenzelm
parents:
45620
diff
changeset
|
346 |
val s' = |
426ed18eba43
discontinued old-style Term.list_abs in favour of plain Term.abs;
wenzelm
parents:
45620
diff
changeset
|
347 |
fold_rev Term.abs ps |
56253 | 348 |
(Const (@{const_name Nominal.supp}, fastype_of1 (Ts, s) --> HOLogic.mk_setT T) $ s); |
19857 | 349 |
val supports_fresh_rule' = Thm.lift_rule goal supports_fresh_rule; |
350 |
val _ $ (_ $ S $ _) = |
|
59582 | 351 |
Logic.strip_assums_concl (hd (Thm.prems_of supports_fresh_rule')); |
60787 | 352 |
val supports_fresh_rule'' = |
353 |
infer_instantiate ctxt |
|
354 |
[(#1 (dest_Var (head_of S)), Thm.cterm_of ctxt s')] supports_fresh_rule'; |
|
19857 | 355 |
in |
56491 | 356 |
(tactical ctxt ("guessing of the right set that supports the goal", |
58956
a816aa3ff391
proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);
wenzelm
parents:
56492
diff
changeset
|
357 |
(EVERY [compose_tac ctxt (false, supports_fresh_rule'', 3) i, |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
358 |
asm_full_simp_tac ctxt1 (i+2), |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
359 |
asm_full_simp_tac ctxt2 (i+1), |
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
360 |
supports_tac_i tactical ctxt i]))) st |
19857 | 361 |
end |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
362 |
(* when a term-constructor contains more than one binder, it is useful *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
363 |
(* in nominal_primrecs to try whether the goal can be solved by an hammer *) |
56491 | 364 |
| _ => (tactical ctxt ("if it is not of the form _\<sharp>_, then try the simplifier", |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
365 |
(asm_full_simp_tac (put_simpset HOL_ss ctxt addsimps [fresh_prod]@fresh_atm) i))) st |
19857 | 366 |
end |
43278 | 367 |
handle General.Subscript => Seq.empty; |
368 |
(* FIXME proper SUBGOAL/CSUBGOAL instead of cprems_of etc. *) |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
369 |
|
56492 | 370 |
val eqvt_simp_tac = eqvt_asm_full_simp_tac_i NO_DEBUG; |
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
371 |
|
56492 | 372 |
val perm_simp_tac = perm_asm_full_simp_tac_i NO_DEBUG; |
373 |
val perm_extend_simp_tac = perm_extend_simp_tac_i NO_DEBUG; |
|
374 |
val supports_tac = supports_tac_i NO_DEBUG; |
|
375 |
val finite_guess_tac = finite_guess_tac_i NO_DEBUG; |
|
376 |
val fresh_guess_tac = fresh_guess_tac_i NO_DEBUG; |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
377 |
|
56492 | 378 |
val dperm_simp_tac = perm_asm_full_simp_tac_i DEBUG; |
379 |
val dperm_extend_simp_tac = perm_extend_simp_tac_i DEBUG; |
|
380 |
val dsupports_tac = supports_tac_i DEBUG; |
|
381 |
val dfinite_guess_tac = finite_guess_tac_i DEBUG; |
|
382 |
val dfresh_guess_tac = fresh_guess_tac_i DEBUG; |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
383 |
|
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
384 |
(* Code opied from the Simplifer for setting up the perm_simp method *) |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
385 |
(* behaves nearly identical to the simp-method, for example can handle *) |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
386 |
(* options like (no_asm) etc. *) |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
387 |
val no_asmN = "no_asm"; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
388 |
val no_asm_useN = "no_asm_use"; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
389 |
val no_asm_simpN = "no_asm_simp"; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
390 |
val asm_lrN = "asm_lr"; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
391 |
|
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
392 |
val perm_simp_options = |
56492 | 393 |
(Args.parens (Args.$$$ no_asmN) >> K (perm_simp_tac_i NO_DEBUG) || |
394 |
Args.parens (Args.$$$ no_asm_simpN) >> K (perm_asm_simp_tac_i NO_DEBUG) || |
|
395 |
Args.parens (Args.$$$ no_asm_useN) >> K (perm_full_simp_tac_i NO_DEBUG) || |
|
396 |
Args.parens (Args.$$$ asm_lrN) >> K (perm_asm_lr_simp_tac_i NO_DEBUG) || |
|
397 |
Scan.succeed (perm_asm_full_simp_tac_i NO_DEBUG)); |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
398 |
|
30549 | 399 |
val perm_simp_meth = |
33554 | 400 |
Scan.lift perm_simp_options --| Method.sections (Simplifier.simp_modifiers') >> |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
401 |
(fn tac => fn ctxt => SIMPLE_METHOD' (CHANGED_PROP o tac ctxt)); |
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
402 |
|
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
403 |
(* setup so that the simpset is used which is active at the moment when the tactic is called *) |
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
404 |
fun local_simp_meth_setup tac = |
30549 | 405 |
Method.sections (Simplifier.simp_modifiers' @ Splitter.split_modifiers) >> |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
406 |
(K (SIMPLE_METHOD' o tac)); |
17870 | 407 |
|
22595
293934e41dfd
make fresh_guess fail if it does not solve the subgoal
narboux
parents:
22578
diff
changeset
|
408 |
(* uses HOL_basic_ss only and fails if the tactic does not solve the subgoal *) |
293934e41dfd
make fresh_guess fail if it does not solve the subgoal
narboux
parents:
22578
diff
changeset
|
409 |
|
22656
13302b2d0948
debug versions of finite_guess and fresh_guess do not fail if they can not solve the goal
narboux
parents:
22610
diff
changeset
|
410 |
fun basic_simp_meth_setup debug tac = |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
411 |
Scan.depend (fn context => Scan.succeed (Simplifier.map_ss (put_simpset HOL_basic_ss) context, ())) -- |
30549 | 412 |
Method.sections (Simplifier.simp_modifiers' @ Splitter.split_modifiers) >> |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
46219
diff
changeset
|
413 |
(K (SIMPLE_METHOD' o (if debug then tac else SOLVED' o tac))); |
22418
49e2d9744ae1
major update of the nominal package; there is now an infrastructure
urbanc
parents:
22274
diff
changeset
|
414 |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
415 |
val perm_simp_meth_debug = local_simp_meth_setup dperm_simp_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
416 |
val perm_extend_simp_meth = local_simp_meth_setup perm_extend_simp_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
417 |
val perm_extend_simp_meth_debug = local_simp_meth_setup dperm_extend_simp_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
418 |
val supports_meth = local_simp_meth_setup supports_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
419 |
val supports_meth_debug = local_simp_meth_setup dsupports_tac; |
24571 | 420 |
|
28322
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
421 |
val finite_guess_meth = basic_simp_meth_setup false finite_guess_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
422 |
val finite_guess_meth_debug = basic_simp_meth_setup true dfinite_guess_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
423 |
val fresh_guess_meth = basic_simp_meth_setup false fresh_guess_tac; |
6f4cf302c798
made the perm_simp tactic to understand options such as (no_asm)
urbanc
parents:
28262
diff
changeset
|
424 |
val fresh_guess_meth_debug = basic_simp_meth_setup true dfresh_guess_tac; |
17870 | 425 |
|
20289 | 426 |
end |