author | nipkow |
Thu, 21 Mar 2013 10:05:03 +0100 | |
changeset 51468 | 0e8012983c4e |
parent 50112 | 11cd86c5af3a |
child 51580 | 64ef8260dc60 |
permissions | -rw-r--r-- |
9938 | 1 |
(* Title: Provers/classical.ML |
2 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
0 | 3 |
|
4 |
Theorem prover for classical reasoning, including predicate calculus, set |
|
5 |
theory, etc. |
|
6 |
||
9563
216d053992a5
fixed classification of rules in atts and modifiers (final!?);
wenzelm
parents:
9513
diff
changeset
|
7 |
Rules must be classified as intro, elim, safe, hazardous (unsafe). |
0 | 8 |
|
9 |
A rule is unsafe unless it can be applied blindly without harmful results. |
|
10 |
For a rule to be safe, its premises and conclusion should be logically |
|
11 |
equivalent. There should be no variables in the premises that are not in |
|
12 |
the conclusion. |
|
13 |
*) |
|
14 |
||
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
15 |
(*higher precedence than := facilitates use of references*) |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
16 |
infix 4 addSIs addSEs addSDs addIs addEs addDs delrules |
4651 | 17 |
addSWrapper delSWrapper addWrapper delWrapper |
11181
d04f57b91166
renamed addaltern to addafter, addSaltern to addSafter
oheimb
parents:
11168
diff
changeset
|
18 |
addSbefore addSafter addbefore addafter |
5523 | 19 |
addD2 addE2 addSD2 addSE2; |
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
20 |
|
0 | 21 |
signature CLASSICAL_DATA = |
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
22 |
sig |
42790 | 23 |
val imp_elim: thm (* P --> Q ==> (~ R ==> P) ==> (Q ==> R) ==> R *) |
24 |
val not_elim: thm (* ~P ==> P ==> R *) |
|
25 |
val swap: thm (* ~ P ==> (~ R ==> P) ==> R *) |
|
26 |
val classical: thm (* (~ P ==> P) ==> P *) |
|
50062 | 27 |
val sizef: thm -> int (* size function for BEST_FIRST, typically size_of_thm *) |
28 |
val hyp_subst_tacs: (int -> tactic) list (* optional tactics for substitution in |
|
29 |
the hypotheses; assumed to be safe! *) |
|
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
30 |
end; |
0 | 31 |
|
5841 | 32 |
signature BASIC_CLASSICAL = |
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
33 |
sig |
42812 | 34 |
type wrapper = (int -> tactic) -> int -> tactic |
0 | 35 |
type claset |
42793 | 36 |
val print_claset: Proof.context -> unit |
37 |
val addDs: Proof.context * thm list -> Proof.context |
|
38 |
val addEs: Proof.context * thm list -> Proof.context |
|
39 |
val addIs: Proof.context * thm list -> Proof.context |
|
40 |
val addSDs: Proof.context * thm list -> Proof.context |
|
41 |
val addSEs: Proof.context * thm list -> Proof.context |
|
42 |
val addSIs: Proof.context * thm list -> Proof.context |
|
43 |
val delrules: Proof.context * thm list -> Proof.context |
|
44 |
val addSWrapper: claset * (string * (Proof.context -> wrapper)) -> claset |
|
42790 | 45 |
val delSWrapper: claset * string -> claset |
42793 | 46 |
val addWrapper: claset * (string * (Proof.context -> wrapper)) -> claset |
42790 | 47 |
val delWrapper: claset * string -> claset |
48 |
val addSbefore: claset * (string * (int -> tactic)) -> claset |
|
49 |
val addSafter: claset * (string * (int -> tactic)) -> claset |
|
50 |
val addbefore: claset * (string * (int -> tactic)) -> claset |
|
51 |
val addafter: claset * (string * (int -> tactic)) -> claset |
|
52 |
val addD2: claset * (string * thm) -> claset |
|
53 |
val addE2: claset * (string * thm) -> claset |
|
54 |
val addSD2: claset * (string * thm) -> claset |
|
55 |
val addSE2: claset * (string * thm) -> claset |
|
42793 | 56 |
val appSWrappers: Proof.context -> wrapper |
57 |
val appWrappers: Proof.context -> wrapper |
|
982
4fe0b642b7d5
Addition of wrappers for integration with the simplifier.
lcp
parents:
747
diff
changeset
|
58 |
|
42790 | 59 |
val global_claset_of: theory -> claset |
60 |
val claset_of: Proof.context -> claset |
|
42793 | 61 |
val map_claset: (claset -> claset) -> Proof.context -> Proof.context |
62 |
val put_claset: claset -> Proof.context -> Proof.context |
|
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
63 |
|
42793 | 64 |
val fast_tac: Proof.context -> int -> tactic |
65 |
val slow_tac: Proof.context -> int -> tactic |
|
66 |
val astar_tac: Proof.context -> int -> tactic |
|
67 |
val slow_astar_tac: Proof.context -> int -> tactic |
|
68 |
val best_tac: Proof.context -> int -> tactic |
|
69 |
val first_best_tac: Proof.context -> int -> tactic |
|
70 |
val slow_best_tac: Proof.context -> int -> tactic |
|
71 |
val depth_tac: Proof.context -> int -> int -> tactic |
|
72 |
val deepen_tac: Proof.context -> int -> int -> tactic |
|
1587
e7d8a4957bac
Now provides astar versions (thanks to Norbert Voelker)
paulson
parents:
1524
diff
changeset
|
73 |
|
42790 | 74 |
val contr_tac: int -> tactic |
75 |
val dup_elim: thm -> thm |
|
76 |
val dup_intr: thm -> thm |
|
42793 | 77 |
val dup_step_tac: Proof.context -> int -> tactic |
42790 | 78 |
val eq_mp_tac: int -> tactic |
42793 | 79 |
val haz_step_tac: Proof.context -> int -> tactic |
42790 | 80 |
val joinrules: thm list * thm list -> (bool * thm) list |
81 |
val mp_tac: int -> tactic |
|
42793 | 82 |
val safe_tac: Proof.context -> tactic |
83 |
val safe_steps_tac: Proof.context -> int -> tactic |
|
84 |
val safe_step_tac: Proof.context -> int -> tactic |
|
85 |
val clarify_tac: Proof.context -> int -> tactic |
|
86 |
val clarify_step_tac: Proof.context -> int -> tactic |
|
87 |
val step_tac: Proof.context -> int -> tactic |
|
88 |
val slow_step_tac: Proof.context -> int -> tactic |
|
42790 | 89 |
val swapify: thm list -> thm list |
90 |
val swap_res_tac: thm list -> int -> tactic |
|
42793 | 91 |
val inst_step_tac: Proof.context -> int -> tactic |
92 |
val inst0_step_tac: Proof.context -> int -> tactic |
|
93 |
val instp_step_tac: Proof.context -> int -> tactic |
|
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
94 |
end; |
1724 | 95 |
|
5841 | 96 |
signature CLASSICAL = |
97 |
sig |
|
98 |
include BASIC_CLASSICAL |
|
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
99 |
val classical_rule: thm -> thm |
42812 | 100 |
type netpair = (int * (bool * thm)) Net.net * (int * (bool * thm)) Net.net |
101 |
val rep_cs: claset -> |
|
102 |
{safeIs: thm Item_Net.T, |
|
103 |
safeEs: thm Item_Net.T, |
|
104 |
hazIs: thm Item_Net.T, |
|
105 |
hazEs: thm Item_Net.T, |
|
106 |
swrappers: (string * (Proof.context -> wrapper)) list, |
|
107 |
uwrappers: (string * (Proof.context -> wrapper)) list, |
|
108 |
safe0_netpair: netpair, |
|
109 |
safep_netpair: netpair, |
|
110 |
haz_netpair: netpair, |
|
111 |
dup_netpair: netpair, |
|
112 |
xtra_netpair: Context_Rules.netpair} |
|
24021 | 113 |
val get_cs: Context.generic -> claset |
114 |
val map_cs: (claset -> claset) -> Context.generic -> Context.generic |
|
18728 | 115 |
val safe_dest: int option -> attribute |
116 |
val safe_elim: int option -> attribute |
|
117 |
val safe_intro: int option -> attribute |
|
118 |
val haz_dest: int option -> attribute |
|
119 |
val haz_elim: int option -> attribute |
|
120 |
val haz_intro: int option -> attribute |
|
121 |
val rule_del: attribute |
|
30513 | 122 |
val cla_modifiers: Method.modifier parser list |
42793 | 123 |
val cla_method: |
124 |
(Proof.context -> tactic) -> (Proof.context -> Proof.method) context_parser |
|
125 |
val cla_method': |
|
126 |
(Proof.context -> int -> tactic) -> (Proof.context -> Proof.method) context_parser |
|
18708 | 127 |
val setup: theory -> theory |
5841 | 128 |
end; |
129 |
||
0 | 130 |
|
42799 | 131 |
functor Classical(Data: CLASSICAL_DATA): CLASSICAL = |
0 | 132 |
struct |
133 |
||
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
134 |
(** classical elimination rules **) |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
135 |
|
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
136 |
(* |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
137 |
Classical reasoning requires stronger elimination rules. For |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
138 |
instance, make_elim of Pure transforms the HOL rule injD into |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
139 |
|
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
140 |
[| inj f; f x = f y; x = y ==> PROP W |] ==> PROP W |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
141 |
|
26938 | 142 |
Such rules can cause fast_tac to fail and blast_tac to report "PROOF |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
143 |
FAILED"; classical_rule will strenthen this to |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
144 |
|
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
145 |
[| inj f; ~ W ==> f x = f y; x = y ==> W |] ==> W |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
146 |
*) |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
147 |
|
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
148 |
fun classical_rule rule = |
41581
72a02e3dec7e
clarified pretty_statement: more robust treatment of fixes and conclusion of elimination (e.g. for classical rule);
wenzelm
parents:
36960
diff
changeset
|
149 |
if is_some (Object_Logic.elim_concl rule) then |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
150 |
let |
42792 | 151 |
val rule' = rule RS Data.classical; |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
152 |
val concl' = Thm.concl_of rule'; |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
153 |
fun redundant_hyp goal = |
19257 | 154 |
concl' aconv Logic.strip_assums_concl goal orelse |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
155 |
(case Logic.strip_assums_hyp goal of |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
156 |
hyp :: hyps => exists (fn t => t aconv hyp) hyps |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
157 |
| _ => false); |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
158 |
val rule'' = |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
159 |
rule' |> ALLGOALS (SUBGOAL (fn (goal, i) => |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
160 |
if i = 1 orelse redundant_hyp goal |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
161 |
then Tactic.etac thin_rl i |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
162 |
else all_tac)) |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
163 |
|> Seq.hd |
21963 | 164 |
|> Drule.zero_var_indexes; |
22360
26ead7ed4f4b
moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents:
22095
diff
changeset
|
165 |
in if Thm.equiv_thm (rule, rule'') then rule else rule'' end |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
166 |
else rule; |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
167 |
|
23594
e65e466dda01
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
wenzelm
parents:
23178
diff
changeset
|
168 |
(*flatten nested meta connectives in prems*) |
35625 | 169 |
val flat_rule = Conv.fconv_rule (Conv.prems_conv ~1 Object_Logic.atomize_prems); |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
170 |
|
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
171 |
|
1800 | 172 |
(*** Useful tactics for classical reasoning ***) |
0 | 173 |
|
10736 | 174 |
(*Prove goal that assumes both P and ~P. |
4392 | 175 |
No backtracking if it finds an equal assumption. Perhaps should call |
176 |
ematch_tac instead of eresolve_tac, but then cannot prove ZF/cantor.*) |
|
42792 | 177 |
val contr_tac = |
178 |
eresolve_tac [Data.not_elim] THEN' (eq_assume_tac ORELSE' assume_tac); |
|
0 | 179 |
|
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
180 |
(*Finds P-->Q and P in the assumptions, replaces implication by Q. |
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
181 |
Could do the same thing for P<->Q and P... *) |
42792 | 182 |
fun mp_tac i = eresolve_tac [Data.not_elim, Data.imp_elim] i THEN assume_tac i; |
0 | 183 |
|
184 |
(*Like mp_tac but instantiates no variables*) |
|
42792 | 185 |
fun eq_mp_tac i = ematch_tac [Data.not_elim, Data.imp_elim] i THEN eq_assume_tac i; |
0 | 186 |
|
187 |
(*Creates rules to eliminate ~A, from rules to introduce A*) |
|
26412
0918f5c0bbca
pass imp_elim (instead of mp) and swap explicitly -- avoids store_thm;
wenzelm
parents:
24867
diff
changeset
|
188 |
fun swapify intrs = intrs RLN (2, [Data.swap]); |
30528 | 189 |
val swapped = Thm.rule_attribute (fn _ => fn th => th RSN (2, Data.swap)); |
0 | 190 |
|
191 |
(*Uses introduction rules in the normal way, or on negated assumptions, |
|
192 |
trying rules in order. *) |
|
10736 | 193 |
fun swap_res_tac rls = |
42792 | 194 |
let fun addrl rl brls = (false, rl) :: (true, rl RSN (2, Data.swap)) :: brls in |
195 |
assume_tac ORELSE' |
|
196 |
contr_tac ORELSE' |
|
197 |
biresolve_tac (fold_rev addrl rls []) |
|
198 |
end; |
|
0 | 199 |
|
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
200 |
(*Duplication of hazardous rules, for complete provers*) |
42792 | 201 |
fun dup_intr th = zero_var_indexes (th RS Data.classical); |
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
202 |
|
42793 | 203 |
fun dup_elim th = (* FIXME proper context!? *) |
36546 | 204 |
let |
205 |
val rl = (th RSN (2, revcut_rl)) |> Thm.assumption 2 |> Seq.hd; |
|
42361 | 206 |
val ctxt = Proof_Context.init_global (Thm.theory_of_thm rl); |
36546 | 207 |
in rule_by_tactic ctxt (TRYALL (etac revcut_rl)) rl end; |
208 |
||
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
209 |
|
1800 | 210 |
(**** Classical rule sets ****) |
0 | 211 |
|
42812 | 212 |
type netpair = (int * (bool * thm)) Net.net * (int * (bool * thm)) Net.net; |
213 |
type wrapper = (int -> tactic) -> int -> tactic; |
|
214 |
||
0 | 215 |
datatype claset = |
42793 | 216 |
CS of |
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
217 |
{safeIs : thm Item_Net.T, (*safe introduction rules*) |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
218 |
safeEs : thm Item_Net.T, (*safe elimination rules*) |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
219 |
hazIs : thm Item_Net.T, (*unsafe introduction rules*) |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
220 |
hazEs : thm Item_Net.T, (*unsafe elimination rules*) |
42793 | 221 |
swrappers : (string * (Proof.context -> wrapper)) list, (*for transforming safe_step_tac*) |
222 |
uwrappers : (string * (Proof.context -> wrapper)) list, (*for transforming step_tac*) |
|
223 |
safe0_netpair : netpair, (*nets for trivial cases*) |
|
224 |
safep_netpair : netpair, (*nets for >0 subgoals*) |
|
225 |
haz_netpair : netpair, (*nets for unsafe rules*) |
|
226 |
dup_netpair : netpair, (*nets for duplication*) |
|
227 |
xtra_netpair : Context_Rules.netpair}; (*nets for extra rules*) |
|
0 | 228 |
|
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
229 |
(*Desired invariants are |
9938 | 230 |
safe0_netpair = build safe0_brls, |
231 |
safep_netpair = build safep_brls, |
|
232 |
haz_netpair = build (joinrules(hazIs, hazEs)), |
|
10736 | 233 |
dup_netpair = build (joinrules(map dup_intr hazIs, |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
234 |
map dup_elim hazEs)) |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
235 |
|
10736 | 236 |
where build = build_netpair(Net.empty,Net.empty), |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
237 |
safe0_brls contains all brules that solve the subgoal, and |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
238 |
safep_brls contains all brules that generate 1 or more new subgoals. |
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
239 |
The theorem lists are largely comments, though they are used in merge_cs and print_cs. |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
240 |
Nets must be built incrementally, to save space and time. |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
241 |
*) |
0 | 242 |
|
6502 | 243 |
val empty_netpair = (Net.empty, Net.empty); |
244 |
||
10736 | 245 |
val empty_cs = |
42793 | 246 |
CS |
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
247 |
{safeIs = Thm.full_rules, |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
248 |
safeEs = Thm.full_rules, |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
249 |
hazIs = Thm.full_rules, |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
250 |
hazEs = Thm.full_rules, |
42793 | 251 |
swrappers = [], |
252 |
uwrappers = [], |
|
253 |
safe0_netpair = empty_netpair, |
|
254 |
safep_netpair = empty_netpair, |
|
255 |
haz_netpair = empty_netpair, |
|
256 |
dup_netpair = empty_netpair, |
|
257 |
xtra_netpair = empty_netpair}; |
|
0 | 258 |
|
4653 | 259 |
fun rep_cs (CS args) = args; |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
260 |
|
4079
9df5e4f22d96
new implicit claset mechanism based on Sign.sg anytype data;
wenzelm
parents:
4066
diff
changeset
|
261 |
|
1800 | 262 |
(*** Adding (un)safe introduction or elimination rules. |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
263 |
|
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
264 |
In case of overlap, new rules are tried BEFORE old ones!! |
1800 | 265 |
***) |
0 | 266 |
|
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
267 |
(*For use with biresolve_tac. Combines intro rules with swap to handle negated |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
268 |
assumptions. Pairs elim rules with true. *) |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
269 |
fun joinrules (intrs, elims) = |
18557
60a0f9caa0a2
Provers/classical: stricter checks to ensure that supplied intro, dest and
paulson
parents:
18534
diff
changeset
|
270 |
(map (pair true) (elims @ swapify intrs)) @ map (pair false) intrs; |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
271 |
|
12401 | 272 |
fun joinrules' (intrs, elims) = |
18557
60a0f9caa0a2
Provers/classical: stricter checks to ensure that supplied intro, dest and
paulson
parents:
18534
diff
changeset
|
273 |
map (pair true) elims @ map (pair false) intrs; |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
274 |
|
10736 | 275 |
(*Priority: prefer rules with fewest subgoals, |
1231 | 276 |
then rules added most recently (preferring the head of the list).*) |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
277 |
fun tag_brls k [] = [] |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
278 |
| tag_brls k (brl::brls) = |
10736 | 279 |
(1000000*subgoals_of_brl brl + k, brl) :: |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
280 |
tag_brls (k+1) brls; |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
281 |
|
12401 | 282 |
fun tag_brls' _ _ [] = [] |
283 |
| tag_brls' w k (brl::brls) = ((w, k), brl) :: tag_brls' w (k + 1) brls; |
|
10736 | 284 |
|
23178 | 285 |
fun insert_tagged_list rls = fold_rev Tactic.insert_tagged_brl rls; |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
286 |
|
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
287 |
(*Insert into netpair that already has nI intr rules and nE elim rules. |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
288 |
Count the intr rules double (to account for swapify). Negate to give the |
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
289 |
new insertions the lowest priority.*) |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
290 |
fun insert (nI, nE) = insert_tagged_list o (tag_brls (~(2*nI+nE))) o joinrules; |
12401 | 291 |
fun insert' w (nI, nE) = insert_tagged_list o tag_brls' w (~(nI + nE)) o joinrules'; |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
292 |
|
23178 | 293 |
fun delete_tagged_list rls = fold_rev Tactic.delete_tagged_brl rls; |
12362 | 294 |
fun delete x = delete_tagged_list (joinrules x); |
12401 | 295 |
fun delete' x = delete_tagged_list (joinrules' x); |
1800 | 296 |
|
42793 | 297 |
fun string_of_thm NONE = Display.string_of_thm_without_context |
42817 | 298 |
| string_of_thm (SOME context) = Display.string_of_thm (Context.proof_of context); |
42793 | 299 |
|
300 |
fun make_elim context th = |
|
301 |
if has_fewer_prems 1 th then |
|
302 |
error ("Ill-formed destruction rule\n" ^ string_of_thm context th) |
|
303 |
else Tactic.make_elim th; |
|
42790 | 304 |
|
46874 | 305 |
fun warn_thm opt_context msg th = |
306 |
if (case opt_context of SOME context => Context_Position.is_visible_proof context | NONE => false) |
|
307 |
then warning (msg ^ string_of_thm opt_context th) |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
308 |
else (); |
42793 | 309 |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
310 |
fun warn_rules context msg rules th = |
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
311 |
Item_Net.member rules th andalso (warn_thm context msg th; true); |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
312 |
|
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
313 |
fun warn_claset context th (CS {safeIs, safeEs, hazIs, hazEs, ...}) = |
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
314 |
warn_rules context "Rule already declared as safe introduction (intro!)\n" safeIs th orelse |
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
315 |
warn_rules context "Rule already declared as safe elimination (elim!)\n" safeEs th orelse |
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
316 |
warn_rules context "Rule already declared as introduction (intro)\n" hazIs th orelse |
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
317 |
warn_rules context "Rule already declared as elimination (elim)\n" hazEs th; |
1927
6f97cb16e453
New classical reasoner: warns of, and ignores, redundant rules.
paulson
parents:
1814
diff
changeset
|
318 |
|
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
319 |
|
1800 | 320 |
(*** Safe rules ***) |
982
4fe0b642b7d5
Addition of wrappers for integration with the simplifier.
lcp
parents:
747
diff
changeset
|
321 |
|
42793 | 322 |
fun addSI w context th |
42790 | 323 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
324 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
325 |
if warn_rules context "Ignoring duplicate safe introduction (intro!)\n" safeIs th then cs |
1927
6f97cb16e453
New classical reasoner: warns of, and ignores, redundant rules.
paulson
parents:
1814
diff
changeset
|
326 |
else |
42790 | 327 |
let |
328 |
val th' = flat_rule th; |
|
23594
e65e466dda01
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
wenzelm
parents:
23178
diff
changeset
|
329 |
val (safe0_rls, safep_rls) = (*0 subgoals vs 1 or more*) |
42790 | 330 |
List.partition Thm.no_prems [th']; |
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
331 |
val nI = Item_Net.length safeIs + 1; |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
332 |
val nE = Item_Net.length safeEs; |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
333 |
val _ = warn_claset context th cs; |
42790 | 334 |
in |
335 |
CS |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
336 |
{safeIs = Item_Net.update th safeIs, |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
337 |
safe0_netpair = insert (nI,nE) (safe0_rls, []) safe0_netpair, |
9938 | 338 |
safep_netpair = insert (nI,nE) (safep_rls, []) safep_netpair, |
42790 | 339 |
safeEs = safeEs, |
340 |
hazIs = hazIs, |
|
341 |
hazEs = hazEs, |
|
342 |
swrappers = swrappers, |
|
343 |
uwrappers = uwrappers, |
|
344 |
haz_netpair = haz_netpair, |
|
345 |
dup_netpair = dup_netpair, |
|
18691 | 346 |
xtra_netpair = insert' (the_default 0 w) (nI,nE) ([th], []) xtra_netpair} |
42790 | 347 |
end; |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
348 |
|
42793 | 349 |
fun addSE w context th |
42790 | 350 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
351 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
352 |
if warn_rules context "Ignoring duplicate safe elimination (elim!)\n" safeEs th then cs |
18557
60a0f9caa0a2
Provers/classical: stricter checks to ensure that supplied intro, dest and
paulson
parents:
18534
diff
changeset
|
353 |
else if has_fewer_prems 1 th then |
42793 | 354 |
error ("Ill-formed elimination rule\n" ^ string_of_thm context th) |
1927
6f97cb16e453
New classical reasoner: warns of, and ignores, redundant rules.
paulson
parents:
1814
diff
changeset
|
355 |
else |
42790 | 356 |
let |
357 |
val th' = classical_rule (flat_rule th); |
|
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
358 |
val (safe0_rls, safep_rls) = (*0 subgoals vs 1 or more*) |
42790 | 359 |
List.partition (fn rl => nprems_of rl=1) [th']; |
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
360 |
val nI = Item_Net.length safeIs; |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
361 |
val nE = Item_Net.length safeEs + 1; |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
362 |
val _ = warn_claset context th cs; |
42790 | 363 |
in |
364 |
CS |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
365 |
{safeEs = Item_Net.update th safeEs, |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
366 |
safe0_netpair = insert (nI,nE) ([], safe0_rls) safe0_netpair, |
9938 | 367 |
safep_netpair = insert (nI,nE) ([], safep_rls) safep_netpair, |
42790 | 368 |
safeIs = safeIs, |
369 |
hazIs = hazIs, |
|
370 |
hazEs = hazEs, |
|
371 |
swrappers = swrappers, |
|
372 |
uwrappers = uwrappers, |
|
373 |
haz_netpair = haz_netpair, |
|
374 |
dup_netpair = dup_netpair, |
|
18691 | 375 |
xtra_netpair = insert' (the_default 0 w) (nI,nE) ([], [th]) xtra_netpair} |
42790 | 376 |
end; |
0 | 377 |
|
42793 | 378 |
fun addSD w context th = addSE w context (make_elim context th); |
379 |
||
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
380 |
|
1800 | 381 |
(*** Hazardous (unsafe) rules ***) |
0 | 382 |
|
42793 | 383 |
fun addI w context th |
42790 | 384 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
385 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
386 |
if warn_rules context "Ignoring duplicate introduction (intro)\n" hazIs th then cs |
1927
6f97cb16e453
New classical reasoner: warns of, and ignores, redundant rules.
paulson
parents:
1814
diff
changeset
|
387 |
else |
42790 | 388 |
let |
389 |
val th' = flat_rule th; |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
390 |
val nI = Item_Net.length hazIs + 1; |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
391 |
val nE = Item_Net.length hazEs; |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
392 |
val _ = warn_claset context th cs; |
42790 | 393 |
in |
394 |
CS |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
395 |
{hazIs = Item_Net.update th hazIs, |
42790 | 396 |
haz_netpair = insert (nI, nE) ([th'], []) haz_netpair, |
397 |
dup_netpair = insert (nI, nE) ([dup_intr th'], []) dup_netpair, |
|
398 |
safeIs = safeIs, |
|
399 |
safeEs = safeEs, |
|
400 |
hazEs = hazEs, |
|
401 |
swrappers = swrappers, |
|
402 |
uwrappers = uwrappers, |
|
9938 | 403 |
safe0_netpair = safe0_netpair, |
404 |
safep_netpair = safep_netpair, |
|
42790 | 405 |
xtra_netpair = insert' (the_default 1 w) (nI, nE) ([th], []) xtra_netpair} |
406 |
end |
|
407 |
handle THM ("RSN: no unifiers", _, _) => (*from dup_intr*) (* FIXME !? *) |
|
42793 | 408 |
error ("Ill-formed introduction rule\n" ^ string_of_thm context th); |
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
409 |
|
42793 | 410 |
fun addE w context th |
42790 | 411 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
412 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
413 |
if warn_rules context "Ignoring duplicate elimination (elim)\n" hazEs th then cs |
18557
60a0f9caa0a2
Provers/classical: stricter checks to ensure that supplied intro, dest and
paulson
parents:
18534
diff
changeset
|
414 |
else if has_fewer_prems 1 th then |
42793 | 415 |
error ("Ill-formed elimination rule\n" ^ string_of_thm context th) |
1927
6f97cb16e453
New classical reasoner: warns of, and ignores, redundant rules.
paulson
parents:
1814
diff
changeset
|
416 |
else |
42790 | 417 |
let |
418 |
val th' = classical_rule (flat_rule th); |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
419 |
val nI = Item_Net.length hazIs; |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
420 |
val nE = Item_Net.length hazEs + 1; |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
421 |
val _ = warn_claset context th cs; |
42790 | 422 |
in |
423 |
CS |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
424 |
{hazEs = Item_Net.update th hazEs, |
42790 | 425 |
haz_netpair = insert (nI, nE) ([], [th']) haz_netpair, |
426 |
dup_netpair = insert (nI, nE) ([], [dup_elim th']) dup_netpair, |
|
427 |
safeIs = safeIs, |
|
428 |
safeEs = safeEs, |
|
429 |
hazIs = hazIs, |
|
430 |
swrappers = swrappers, |
|
431 |
uwrappers = uwrappers, |
|
9938 | 432 |
safe0_netpair = safe0_netpair, |
433 |
safep_netpair = safep_netpair, |
|
42790 | 434 |
xtra_netpair = insert' (the_default 1 w) (nI, nE) ([], [th]) xtra_netpair} |
435 |
end; |
|
0 | 436 |
|
42793 | 437 |
fun addD w context th = addE w context (make_elim context th); |
438 |
||
0 | 439 |
|
1073
b3f190995bc9
Recoded addSIs, etc., so that nets are built incrementally
lcp
parents:
1010
diff
changeset
|
440 |
|
10736 | 441 |
(*** Deletion of rules |
1800 | 442 |
Working out what to delete, requires repeating much of the code used |
9938 | 443 |
to insert. |
1800 | 444 |
***) |
445 |
||
10736 | 446 |
fun delSI th |
42790 | 447 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
448 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
449 |
if Item_Net.member safeIs th then |
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
450 |
let |
42790 | 451 |
val th' = flat_rule th; |
452 |
val (safe0_rls, safep_rls) = List.partition Thm.no_prems [th']; |
|
453 |
in |
|
454 |
CS |
|
455 |
{safe0_netpair = delete (safe0_rls, []) safe0_netpair, |
|
456 |
safep_netpair = delete (safep_rls, []) safep_netpair, |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
457 |
safeIs = Item_Net.remove th safeIs, |
42790 | 458 |
safeEs = safeEs, |
459 |
hazIs = hazIs, |
|
460 |
hazEs = hazEs, |
|
461 |
swrappers = swrappers, |
|
462 |
uwrappers = uwrappers, |
|
463 |
haz_netpair = haz_netpair, |
|
464 |
dup_netpair = dup_netpair, |
|
465 |
xtra_netpair = delete' ([th], []) xtra_netpair} |
|
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
466 |
end |
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
467 |
else cs; |
1800 | 468 |
|
42790 | 469 |
fun delSE th |
470 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
|
471 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
472 |
if Item_Net.member safeEs th then |
42790 | 473 |
let |
474 |
val th' = classical_rule (flat_rule th); |
|
475 |
val (safe0_rls, safep_rls) = List.partition (fn rl => nprems_of rl = 1) [th']; |
|
476 |
in |
|
477 |
CS |
|
478 |
{safe0_netpair = delete ([], safe0_rls) safe0_netpair, |
|
479 |
safep_netpair = delete ([], safep_rls) safep_netpair, |
|
480 |
safeIs = safeIs, |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
481 |
safeEs = Item_Net.remove th safeEs, |
42790 | 482 |
hazIs = hazIs, |
483 |
hazEs = hazEs, |
|
484 |
swrappers = swrappers, |
|
485 |
uwrappers = uwrappers, |
|
486 |
haz_netpair = haz_netpair, |
|
487 |
dup_netpair = dup_netpair, |
|
488 |
xtra_netpair = delete' ([], [th]) xtra_netpair} |
|
489 |
end |
|
490 |
else cs; |
|
1800 | 491 |
|
42793 | 492 |
fun delI context th |
42790 | 493 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
494 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
495 |
if Item_Net.member hazIs th then |
42790 | 496 |
let val th' = flat_rule th in |
497 |
CS |
|
498 |
{haz_netpair = delete ([th'], []) haz_netpair, |
|
23594
e65e466dda01
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
wenzelm
parents:
23178
diff
changeset
|
499 |
dup_netpair = delete ([dup_intr th'], []) dup_netpair, |
42790 | 500 |
safeIs = safeIs, |
501 |
safeEs = safeEs, |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
502 |
hazIs = Item_Net.remove th hazIs, |
42790 | 503 |
hazEs = hazEs, |
504 |
swrappers = swrappers, |
|
505 |
uwrappers = uwrappers, |
|
9938 | 506 |
safe0_netpair = safe0_netpair, |
507 |
safep_netpair = safep_netpair, |
|
12401 | 508 |
xtra_netpair = delete' ([th], []) xtra_netpair} |
23594
e65e466dda01
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
wenzelm
parents:
23178
diff
changeset
|
509 |
end |
42790 | 510 |
else cs |
511 |
handle THM ("RSN: no unifiers", _, _) => (*from dup_intr*) (* FIXME !? *) |
|
42793 | 512 |
error ("Ill-formed introduction rule\n" ^ string_of_thm context th); |
1800 | 513 |
|
2813
cc4c816dafdc
delrules now deletes ALL occurrences of a rule, since it may appear in any of
paulson
parents:
2689
diff
changeset
|
514 |
fun delE th |
42790 | 515 |
(cs as CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
516 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
517 |
if Item_Net.member hazEs th then |
42790 | 518 |
let val th' = classical_rule (flat_rule th) in |
519 |
CS |
|
520 |
{haz_netpair = delete ([], [th']) haz_netpair, |
|
18534
6799b38ed872
added classical_rule, which replaces Data.make_elim;
wenzelm
parents:
18374
diff
changeset
|
521 |
dup_netpair = delete ([], [dup_elim th']) dup_netpair, |
42790 | 522 |
safeIs = safeIs, |
523 |
safeEs = safeEs, |
|
524 |
hazIs = hazIs, |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
525 |
hazEs = Item_Net.remove th hazEs, |
42790 | 526 |
swrappers = swrappers, |
527 |
uwrappers = uwrappers, |
|
9938 | 528 |
safe0_netpair = safe0_netpair, |
529 |
safep_netpair = safep_netpair, |
|
12401 | 530 |
xtra_netpair = delete' ([], [th]) xtra_netpair} |
42790 | 531 |
end |
532 |
else cs; |
|
1800 | 533 |
|
2813
cc4c816dafdc
delrules now deletes ALL occurrences of a rule, since it may appear in any of
paulson
parents:
2689
diff
changeset
|
534 |
(*Delete ALL occurrences of "th" in the claset (perhaps from several lists)*) |
42793 | 535 |
fun delrule context th (cs as CS {safeIs, safeEs, hazIs, hazEs, ...}) = |
536 |
let val th' = Tactic.make_elim th in |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
537 |
if Item_Net.member safeIs th orelse Item_Net.member safeEs th orelse |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
538 |
Item_Net.member hazIs th orelse Item_Net.member hazEs th orelse |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
539 |
Item_Net.member safeEs th' orelse Item_Net.member hazEs th' |
42793 | 540 |
then delSI th (delSE th (delI context th (delE th (delSE th' (delE th' cs))))) |
42807
e639d91d9073
more precise warnings: observe context visibility;
wenzelm
parents:
42799
diff
changeset
|
541 |
else (warn_thm context "Undeclared classical rule\n" th; cs) |
9938 | 542 |
end; |
1800 | 543 |
|
544 |
||
42793 | 545 |
|
546 |
(** claset data **) |
|
42790 | 547 |
|
42793 | 548 |
(* wrappers *) |
42790 | 549 |
|
22674 | 550 |
fun map_swrappers f |
551 |
(CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
|
552 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
|
553 |
CS {safeIs = safeIs, safeEs = safeEs, hazIs = hazIs, hazEs = hazEs, |
|
4767
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
554 |
swrappers = f swrappers, uwrappers = uwrappers, |
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
555 |
safe0_netpair = safe0_netpair, safep_netpair = safep_netpair, |
6955 | 556 |
haz_netpair = haz_netpair, dup_netpair = dup_netpair, xtra_netpair = xtra_netpair}; |
4767
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
557 |
|
22674 | 558 |
fun map_uwrappers f |
42793 | 559 |
(CS {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, |
22674 | 560 |
safe0_netpair, safep_netpair, haz_netpair, dup_netpair, xtra_netpair}) = |
561 |
CS {safeIs = safeIs, safeEs = safeEs, hazIs = hazIs, hazEs = hazEs, |
|
4767
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
562 |
swrappers = swrappers, uwrappers = f uwrappers, |
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
563 |
safe0_netpair = safe0_netpair, safep_netpair = safep_netpair, |
6955 | 564 |
haz_netpair = haz_netpair, dup_netpair = dup_netpair, xtra_netpair = xtra_netpair}; |
4767
b9f3468c6ee2
introduced functions for updating the wrapper lists
oheimb
parents:
4765
diff
changeset
|
565 |
|
22674 | 566 |
|
42793 | 567 |
(* merge_cs *) |
982
4fe0b642b7d5
Addition of wrappers for integration with the simplifier.
lcp
parents:
747
diff
changeset
|
568 |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
569 |
(*Merge works by adding all new rules of the 2nd claset into the 1st claset, |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
570 |
in order to preserve priorities reliably.*) |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
571 |
|
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
572 |
fun merge_thms add thms1 thms2 = |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
573 |
fold_rev (fn thm => if Item_Net.member thms1 thm then I else add thm) (Item_Net.content thms2); |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
574 |
|
22674 | 575 |
fun merge_cs (cs as CS {safeIs, safeEs, hazIs, hazEs, ...}, |
24358 | 576 |
cs' as CS {safeIs = safeIs2, safeEs = safeEs2, hazIs = hazIs2, hazEs = hazEs2, |
22674 | 577 |
swrappers, uwrappers, ...}) = |
24358 | 578 |
if pointer_eq (cs, cs') then cs |
579 |
else |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
580 |
cs |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
581 |
|> merge_thms (addSI NONE NONE) safeIs safeIs2 |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
582 |
|> merge_thms (addSE NONE NONE) safeEs safeEs2 |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
583 |
|> merge_thms (addI NONE NONE) hazIs hazIs2 |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
584 |
|> merge_thms (addE NONE NONE) hazEs hazEs2 |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
585 |
|> map_swrappers (fn ws => AList.merge (op =) (K true) (ws, swrappers)) |
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
586 |
|> map_uwrappers (fn ws => AList.merge (op =) (K true) (ws, uwrappers)); |
42793 | 587 |
|
588 |
||
589 |
(* data *) |
|
590 |
||
591 |
structure Claset = Generic_Data |
|
592 |
( |
|
593 |
type T = claset; |
|
594 |
val empty = empty_cs; |
|
595 |
val extend = I; |
|
596 |
val merge = merge_cs; |
|
597 |
); |
|
598 |
||
599 |
val global_claset_of = Claset.get o Context.Theory; |
|
600 |
val claset_of = Claset.get o Context.Proof; |
|
601 |
val rep_claset_of = rep_cs o claset_of; |
|
602 |
||
603 |
val get_cs = Claset.get; |
|
604 |
val map_cs = Claset.map; |
|
605 |
||
606 |
fun map_claset f = Context.proof_map (map_cs f); |
|
607 |
fun put_claset cs = map_claset (K cs); |
|
608 |
||
609 |
fun print_claset ctxt = |
|
610 |
let |
|
611 |
val {safeIs, safeEs, hazIs, hazEs, swrappers, uwrappers, ...} = rep_claset_of ctxt; |
|
42810
2425068fe13a
slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
wenzelm
parents:
42807
diff
changeset
|
612 |
val pretty_thms = map (Display.pretty_thm ctxt) o Item_Net.content; |
42793 | 613 |
in |
614 |
[Pretty.big_list "safe introduction rules (intro!):" (pretty_thms safeIs), |
|
615 |
Pretty.big_list "introduction rules (intro):" (pretty_thms hazIs), |
|
616 |
Pretty.big_list "safe elimination rules (elim!):" (pretty_thms safeEs), |
|
617 |
Pretty.big_list "elimination rules (elim):" (pretty_thms hazEs), |
|
618 |
Pretty.strs ("safe wrappers:" :: map #1 swrappers), |
|
619 |
Pretty.strs ("unsafe wrappers:" :: map #1 uwrappers)] |
|
620 |
|> Pretty.chunks |> Pretty.writeln |
|
621 |
end; |
|
622 |
||
623 |
||
624 |
(* old-style declarations *) |
|
625 |
||
626 |
fun decl f (ctxt, ths) = map_claset (fold_rev (f (SOME (Context.Proof ctxt))) ths) ctxt; |
|
627 |
||
628 |
val op addSIs = decl (addSI NONE); |
|
629 |
val op addSEs = decl (addSE NONE); |
|
630 |
val op addSDs = decl (addSD NONE); |
|
631 |
val op addIs = decl (addI NONE); |
|
632 |
val op addEs = decl (addE NONE); |
|
633 |
val op addDs = decl (addD NONE); |
|
634 |
val op delrules = decl delrule; |
|
635 |
||
636 |
||
637 |
||
638 |
(*** Modifying the wrapper tacticals ***) |
|
639 |
||
640 |
fun appSWrappers ctxt = fold (fn (_, w) => w ctxt) (#swrappers (rep_claset_of ctxt)); |
|
641 |
fun appWrappers ctxt = fold (fn (_, w) => w ctxt) (#uwrappers (rep_claset_of ctxt)); |
|
642 |
||
643 |
fun update_warn msg (p as (key : string, _)) xs = |
|
644 |
(if AList.defined (op =) xs key then warning msg else (); AList.update (op =) p xs); |
|
645 |
||
646 |
fun delete_warn msg (key : string) xs = |
|
647 |
if AList.defined (op =) xs key then AList.delete (op =) key xs |
|
648 |
else (warning msg; xs); |
|
649 |
||
650 |
(*Add/replace a safe wrapper*) |
|
651 |
fun cs addSWrapper new_swrapper = |
|
652 |
map_swrappers (update_warn ("Overwriting safe wrapper " ^ fst new_swrapper) new_swrapper) cs; |
|
653 |
||
654 |
(*Add/replace an unsafe wrapper*) |
|
655 |
fun cs addWrapper new_uwrapper = |
|
656 |
map_uwrappers (update_warn ("Overwriting unsafe wrapper " ^ fst new_uwrapper) new_uwrapper) cs; |
|
657 |
||
658 |
(*Remove a safe wrapper*) |
|
659 |
fun cs delSWrapper name = |
|
660 |
map_swrappers (delete_warn ("No such safe wrapper in claset: " ^ name) name) cs; |
|
661 |
||
662 |
(*Remove an unsafe wrapper*) |
|
663 |
fun cs delWrapper name = |
|
664 |
map_uwrappers (delete_warn ("No such unsafe wrapper in claset: " ^ name) name) cs; |
|
665 |
||
666 |
(* compose a safe tactic alternatively before/after safe_step_tac *) |
|
667 |
fun cs addSbefore (name, tac1) = cs addSWrapper (name, fn _ => fn tac2 => tac1 ORELSE' tac2); |
|
668 |
fun cs addSafter (name, tac2) = cs addSWrapper (name, fn _ => fn tac1 => tac1 ORELSE' tac2); |
|
669 |
||
670 |
(*compose a tactic alternatively before/after the step tactic *) |
|
671 |
fun cs addbefore (name, tac1) = cs addWrapper (name, fn _ => fn tac2 => tac1 APPEND' tac2); |
|
672 |
fun cs addafter (name, tac2) = cs addWrapper (name, fn _ => fn tac1 => tac1 APPEND' tac2); |
|
673 |
||
46459 | 674 |
fun cs addD2 (name, thm) = cs addafter (name, dtac thm THEN' assume_tac); |
675 |
fun cs addE2 (name, thm) = cs addafter (name, etac thm THEN' assume_tac); |
|
42793 | 676 |
fun cs addSD2 (name, thm) = cs addSafter (name, dmatch_tac [thm] THEN' eq_assume_tac); |
677 |
fun cs addSE2 (name, thm) = cs addSafter (name, ematch_tac [thm] THEN' eq_assume_tac); |
|
678 |
||
1711 | 679 |
|
982
4fe0b642b7d5
Addition of wrappers for integration with the simplifier.
lcp
parents:
747
diff
changeset
|
680 |
|
1800 | 681 |
(**** Simple tactics for theorem proving ****) |
0 | 682 |
|
683 |
(*Attack subgoals using safe inferences -- matching, not resolution*) |
|
42793 | 684 |
fun safe_step_tac ctxt = |
685 |
let val {safe0_netpair, safep_netpair, ...} = rep_claset_of ctxt in |
|
686 |
appSWrappers ctxt |
|
687 |
(FIRST' |
|
688 |
[eq_assume_tac, |
|
9938 | 689 |
eq_mp_tac, |
690 |
bimatch_from_nets_tac safe0_netpair, |
|
42792 | 691 |
FIRST' Data.hyp_subst_tacs, |
42793 | 692 |
bimatch_from_nets_tac safep_netpair]) |
693 |
end; |
|
0 | 694 |
|
5757 | 695 |
(*Repeatedly attack a subgoal using safe inferences -- it's deterministic!*) |
42793 | 696 |
fun safe_steps_tac ctxt = |
697 |
REPEAT_DETERM1 o (fn i => COND (has_fewer_prems i) no_tac (safe_step_tac ctxt i)); |
|
5757 | 698 |
|
0 | 699 |
(*Repeatedly attack subgoals using safe inferences -- it's deterministic!*) |
42793 | 700 |
fun safe_tac ctxt = REPEAT_DETERM1 (FIRSTGOAL (safe_steps_tac ctxt)); |
747
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
701 |
|
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
702 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
703 |
(*** Clarify_tac: do safe steps without causing branching ***) |
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
704 |
|
42790 | 705 |
fun nsubgoalsP n (k, brl) = (subgoals_of_brl brl = n); |
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
706 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
707 |
(*version of bimatch_from_nets_tac that only applies rules that |
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
708 |
create precisely n subgoals.*) |
10736 | 709 |
fun n_bimatch_from_nets_tac n = |
42790 | 710 |
biresolution_from_nets_tac (order_list o filter (nsubgoalsP n)) true; |
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
711 |
|
42792 | 712 |
fun eq_contr_tac i = ematch_tac [Data.not_elim] i THEN eq_assume_tac i; |
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
713 |
val eq_assume_contr_tac = eq_assume_tac ORELSE' eq_contr_tac; |
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
714 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
715 |
(*Two-way branching is allowed only if one of the branches immediately closes*) |
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
716 |
fun bimatch2_tac netpair i = |
42790 | 717 |
n_bimatch_from_nets_tac 2 netpair i THEN |
718 |
(eq_assume_contr_tac i ORELSE eq_assume_contr_tac (i + 1)); |
|
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
719 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
720 |
(*Attack subgoals using safe inferences -- matching, not resolution*) |
42793 | 721 |
fun clarify_step_tac ctxt = |
722 |
let val {safe0_netpair, safep_netpair, ...} = rep_claset_of ctxt in |
|
723 |
appSWrappers ctxt |
|
724 |
(FIRST' |
|
725 |
[eq_assume_contr_tac, |
|
9938 | 726 |
bimatch_from_nets_tac safe0_netpair, |
42792 | 727 |
FIRST' Data.hyp_subst_tacs, |
9938 | 728 |
n_bimatch_from_nets_tac 1 safep_netpair, |
42793 | 729 |
bimatch2_tac safep_netpair]) |
730 |
end; |
|
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
731 |
|
42793 | 732 |
fun clarify_tac ctxt = SELECT_GOAL (REPEAT_DETERM (clarify_step_tac ctxt 1)); |
3705
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
733 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
734 |
|
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
735 |
(*** Unsafe steps instantiate variables or lose information ***) |
76f3b2803982
Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
paulson
parents:
3546
diff
changeset
|
736 |
|
4066 | 737 |
(*Backtracking is allowed among the various these unsafe ways of |
738 |
proving a subgoal. *) |
|
42793 | 739 |
fun inst0_step_tac ctxt = |
32862 | 740 |
assume_tac APPEND' |
741 |
contr_tac APPEND' |
|
42793 | 742 |
biresolve_from_nets_tac (#safe0_netpair (rep_claset_of ctxt)); |
747
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
743 |
|
4066 | 744 |
(*These unsafe steps could generate more subgoals.*) |
42793 | 745 |
fun instp_step_tac ctxt = |
746 |
biresolve_from_nets_tac (#safep_netpair (rep_claset_of ctxt)); |
|
0 | 747 |
|
748 |
(*These steps could instantiate variables and are therefore unsafe.*) |
|
42793 | 749 |
fun inst_step_tac ctxt = inst0_step_tac ctxt APPEND' instp_step_tac ctxt; |
0 | 750 |
|
42793 | 751 |
fun haz_step_tac ctxt = |
752 |
biresolve_from_nets_tac (#haz_netpair (rep_claset_of ctxt)); |
|
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
753 |
|
0 | 754 |
(*Single step for the prover. FAILS unless it makes progress. *) |
42793 | 755 |
fun step_tac ctxt i = |
756 |
safe_tac ctxt ORELSE appWrappers ctxt (inst_step_tac ctxt ORELSE' haz_step_tac ctxt) i; |
|
0 | 757 |
|
758 |
(*Using a "safe" rule to instantiate variables is unsafe. This tactic |
|
759 |
allows backtracking from "safe" rules to "unsafe" rules here.*) |
|
42793 | 760 |
fun slow_step_tac ctxt i = |
761 |
safe_tac ctxt ORELSE appWrappers ctxt (inst_step_tac ctxt APPEND' haz_step_tac ctxt) i; |
|
0 | 762 |
|
42791
36f787ae5f70
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm
parents:
42790
diff
changeset
|
763 |
|
1800 | 764 |
(**** The following tactics all fail unless they solve one goal ****) |
0 | 765 |
|
766 |
(*Dumb but fast*) |
|
42793 | 767 |
fun fast_tac ctxt = |
768 |
Object_Logic.atomize_prems_tac THEN' SELECT_GOAL (DEPTH_SOLVE (step_tac ctxt 1)); |
|
0 | 769 |
|
770 |
(*Slower but smarter than fast_tac*) |
|
42793 | 771 |
fun best_tac ctxt = |
35625 | 772 |
Object_Logic.atomize_prems_tac THEN' |
42793 | 773 |
SELECT_GOAL (BEST_FIRST (has_fewer_prems 1, Data.sizef) (step_tac ctxt 1)); |
0 | 774 |
|
9402 | 775 |
(*even a bit smarter than best_tac*) |
42793 | 776 |
fun first_best_tac ctxt = |
35625 | 777 |
Object_Logic.atomize_prems_tac THEN' |
42793 | 778 |
SELECT_GOAL (BEST_FIRST (has_fewer_prems 1, Data.sizef) (FIRSTGOAL (step_tac ctxt))); |
9402 | 779 |
|
42793 | 780 |
fun slow_tac ctxt = |
35625 | 781 |
Object_Logic.atomize_prems_tac THEN' |
42793 | 782 |
SELECT_GOAL (DEPTH_SOLVE (slow_step_tac ctxt 1)); |
0 | 783 |
|
42793 | 784 |
fun slow_best_tac ctxt = |
35625 | 785 |
Object_Logic.atomize_prems_tac THEN' |
42793 | 786 |
SELECT_GOAL (BEST_FIRST (has_fewer_prems 1, Data.sizef) (slow_step_tac ctxt 1)); |
0 | 787 |
|
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
788 |
|
10736 | 789 |
(***ASTAR with weight weight_ASTAR, by Norbert Voelker*) |
42791
36f787ae5f70
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm
parents:
42790
diff
changeset
|
790 |
|
36f787ae5f70
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm
parents:
42790
diff
changeset
|
791 |
val weight_ASTAR = 5; |
1587
e7d8a4957bac
Now provides astar versions (thanks to Norbert Voelker)
paulson
parents:
1524
diff
changeset
|
792 |
|
42793 | 793 |
fun astar_tac ctxt = |
35625 | 794 |
Object_Logic.atomize_prems_tac THEN' |
10382
1fb807260ff1
atomize: all automated tactics that "solve" goals;
wenzelm
parents:
10309
diff
changeset
|
795 |
SELECT_GOAL |
42791
36f787ae5f70
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm
parents:
42790
diff
changeset
|
796 |
(ASTAR (has_fewer_prems 1, fn lev => fn thm => size_of_thm thm + weight_ASTAR * lev) |
42793 | 797 |
(step_tac ctxt 1)); |
1587
e7d8a4957bac
Now provides astar versions (thanks to Norbert Voelker)
paulson
parents:
1524
diff
changeset
|
798 |
|
42793 | 799 |
fun slow_astar_tac ctxt = |
35625 | 800 |
Object_Logic.atomize_prems_tac THEN' |
10382
1fb807260ff1
atomize: all automated tactics that "solve" goals;
wenzelm
parents:
10309
diff
changeset
|
801 |
SELECT_GOAL |
42791
36f787ae5f70
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm
parents:
42790
diff
changeset
|
802 |
(ASTAR (has_fewer_prems 1, fn lev => fn thm => size_of_thm thm + weight_ASTAR * lev) |
42793 | 803 |
(slow_step_tac ctxt 1)); |
1587
e7d8a4957bac
Now provides astar versions (thanks to Norbert Voelker)
paulson
parents:
1524
diff
changeset
|
804 |
|
42790 | 805 |
|
1800 | 806 |
(**** Complete tactic, loosely based upon LeanTaP. This tactic is the outcome |
747
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
807 |
of much experimentation! Changing APPEND to ORELSE below would prove |
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
808 |
easy theorems faster, but loses completeness -- and many of the harder |
1800 | 809 |
theorems such as 43. ****) |
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
810 |
|
747
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
811 |
(*Non-deterministic! Could always expand the first unsafe connective. |
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
812 |
That's hard to implement and did not perform better in experiments, due to |
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
813 |
greater search depth required.*) |
42793 | 814 |
fun dup_step_tac ctxt = |
815 |
biresolve_from_nets_tac (#dup_netpair (rep_claset_of ctxt)); |
|
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
816 |
|
5523 | 817 |
(*Searching to depth m. A variant called nodup_depth_tac appears in clasimp.ML*) |
5757 | 818 |
local |
42793 | 819 |
fun slow_step_tac' ctxt = appWrappers ctxt (instp_step_tac ctxt APPEND' dup_step_tac ctxt); |
42790 | 820 |
in |
42793 | 821 |
fun depth_tac ctxt m i state = SELECT_GOAL |
822 |
(safe_steps_tac ctxt 1 THEN_ELSE |
|
823 |
(DEPTH_SOLVE (depth_tac ctxt m 1), |
|
824 |
inst0_step_tac ctxt 1 APPEND COND (K (m = 0)) no_tac |
|
825 |
(slow_step_tac' ctxt 1 THEN DEPTH_SOLVE (depth_tac ctxt (m - 1) 1)))) i state; |
|
5757 | 826 |
end; |
747
bdc066781063
deepen_tac: modified due to outcome of experiments. Its
lcp
parents:
681
diff
changeset
|
827 |
|
10736 | 828 |
(*Search, with depth bound m. |
2173 | 829 |
This is the "entry point", which does safe inferences first.*) |
42793 | 830 |
fun safe_depth_tac ctxt m = SUBGOAL (fn (prem, i) => |
831 |
let |
|
832 |
val deti = (*No Vars in the goal? No need to backtrack between goals.*) |
|
833 |
if exists_subterm (fn Var _ => true | _ => false) prem then DETERM else I; |
|
42790 | 834 |
in |
42793 | 835 |
SELECT_GOAL (TRY (safe_tac ctxt) THEN DEPTH_SOLVE (deti (depth_tac ctxt m 1))) i |
42790 | 836 |
end); |
681
9b02474744ca
Provers/classical: now takes theorem "classical" as argument, proves "swap"
lcp
parents:
469
diff
changeset
|
837 |
|
42793 | 838 |
fun deepen_tac ctxt = DEEPEN (2, 10) (safe_depth_tac ctxt); |
24021 | 839 |
|
840 |
||
5885 | 841 |
(* attributes *) |
842 |
||
42793 | 843 |
fun attrib f = |
844 |
Thm.declaration_attribute (fn th => fn context => map_cs (f (SOME context) th) context); |
|
5885 | 845 |
|
18691 | 846 |
val safe_elim = attrib o addSE; |
847 |
val safe_intro = attrib o addSI; |
|
42793 | 848 |
val safe_dest = attrib o addSD; |
18691 | 849 |
val haz_elim = attrib o addE; |
850 |
val haz_intro = attrib o addI; |
|
42793 | 851 |
val haz_dest = attrib o addD; |
45375
7fe19930dfc9
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
wenzelm
parents:
42817
diff
changeset
|
852 |
|
7fe19930dfc9
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
wenzelm
parents:
42817
diff
changeset
|
853 |
val rule_del = |
7fe19930dfc9
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
wenzelm
parents:
42817
diff
changeset
|
854 |
Thm.declaration_attribute (fn th => fn context => |
7fe19930dfc9
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
wenzelm
parents:
42817
diff
changeset
|
855 |
context |> map_cs (delrule (SOME context) th) |> |
7fe19930dfc9
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
wenzelm
parents:
42817
diff
changeset
|
856 |
Thm.attribute_declaration Context_Rules.rule_del th); |
5885 | 857 |
|
858 |
||
5841 | 859 |
|
5885 | 860 |
(** concrete syntax of attributes **) |
5841 | 861 |
|
862 |
val introN = "intro"; |
|
863 |
val elimN = "elim"; |
|
864 |
val destN = "dest"; |
|
865 |
||
30528 | 866 |
val setup_attrs = |
867 |
Attrib.setup @{binding swapped} (Scan.succeed swapped) |
|
868 |
"classical swap of introduction rule" #> |
|
33369 | 869 |
Attrib.setup @{binding dest} (Context_Rules.add safe_dest haz_dest Context_Rules.dest_query) |
30528 | 870 |
"declaration of Classical destruction rule" #> |
33369 | 871 |
Attrib.setup @{binding elim} (Context_Rules.add safe_elim haz_elim Context_Rules.elim_query) |
30528 | 872 |
"declaration of Classical elimination rule" #> |
33369 | 873 |
Attrib.setup @{binding intro} (Context_Rules.add safe_intro haz_intro Context_Rules.intro_query) |
30528 | 874 |
"declaration of Classical introduction rule" #> |
875 |
Attrib.setup @{binding rule} (Scan.lift Args.del >> K rule_del) |
|
876 |
"remove declaration of intro/elim/dest rule"; |
|
5841 | 877 |
|
878 |
||
879 |
||
7230 | 880 |
(** proof methods **) |
881 |
||
882 |
local |
|
883 |
||
30609
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
884 |
fun some_rule_tac ctxt facts = SUBGOAL (fn (goal, i) => |
5841 | 885 |
let |
33369 | 886 |
val [rules1, rules2, rules4] = Context_Rules.find_rules false facts goal ctxt; |
42793 | 887 |
val {xtra_netpair, ...} = rep_claset_of ctxt; |
33369 | 888 |
val rules3 = Context_Rules.find_rules_netpair true facts goal xtra_netpair; |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
889 |
val rules = rules1 @ rules2 @ rules3 @ rules4; |
18223 | 890 |
val ruleq = Drule.multi_resolves facts rules; |
12376
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
891 |
in |
480303e3fa08
simplified (and clarified) integration with Pure/ContextRules;
wenzelm
parents:
12362
diff
changeset
|
892 |
Method.trace ctxt rules; |
32952 | 893 |
fn st => Seq.maps (fn rule => Tactic.rtac rule i st) ruleq |
18834 | 894 |
end) |
21687 | 895 |
THEN_ALL_NEW Goal.norm_hhf_tac; |
5841 | 896 |
|
30609
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
897 |
in |
7281 | 898 |
|
30609
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
899 |
fun rule_tac ctxt [] facts = some_rule_tac ctxt facts |
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
900 |
| rule_tac _ rules facts = Method.rule_tac rules facts; |
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
901 |
|
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
902 |
fun default_tac ctxt rules facts = |
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
903 |
HEADGOAL (rule_tac ctxt rules facts) ORELSE |
26470 | 904 |
Class.default_intro_tac ctxt facts; |
10309 | 905 |
|
7230 | 906 |
end; |
5841 | 907 |
|
908 |
||
6502 | 909 |
(* automatic methods *) |
5841 | 910 |
|
5927 | 911 |
val cla_modifiers = |
18728 | 912 |
[Args.$$$ destN -- Args.bang_colon >> K ((I, safe_dest NONE): Method.modifier), |
913 |
Args.$$$ destN -- Args.colon >> K (I, haz_dest NONE), |
|
914 |
Args.$$$ elimN -- Args.bang_colon >> K (I, safe_elim NONE), |
|
915 |
Args.$$$ elimN -- Args.colon >> K (I, haz_elim NONE), |
|
916 |
Args.$$$ introN -- Args.bang_colon >> K (I, safe_intro NONE), |
|
917 |
Args.$$$ introN -- Args.colon >> K (I, haz_intro NONE), |
|
918 |
Args.del -- Args.colon >> K (I, rule_del)]; |
|
5927 | 919 |
|
42793 | 920 |
fun cla_method tac = Method.sections cla_modifiers >> K (SIMPLE_METHOD o tac); |
921 |
fun cla_method' tac = Method.sections cla_modifiers >> K (SIMPLE_METHOD' o tac); |
|
5841 | 922 |
|
923 |
||
924 |
||
925 |
(** setup_methods **) |
|
926 |
||
30541 | 927 |
val setup_methods = |
30609
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
928 |
Method.setup @{binding default} |
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
929 |
(Attrib.thms >> (fn rules => fn ctxt => METHOD (default_tac ctxt rules))) |
30541 | 930 |
"apply some intro/elim rule (potentially classical)" #> |
30609
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
931 |
Method.setup @{binding rule} |
983e8b6e4e69
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
wenzelm
parents:
30558
diff
changeset
|
932 |
(Attrib.thms >> (fn rules => fn ctxt => METHOD (HEADGOAL o rule_tac ctxt rules))) |
30541 | 933 |
"apply some intro/elim rule (potentially classical)" #> |
50112
11cd86c5af3a
tuned -- eliminate pointless ML method definition;
wenzelm
parents:
50108
diff
changeset
|
934 |
Method.setup @{binding contradiction} |
11cd86c5af3a
tuned -- eliminate pointless ML method definition;
wenzelm
parents:
50108
diff
changeset
|
935 |
(Scan.succeed (K (Method.rule [Data.not_elim, Drule.rotate_prems 1 Data.not_elim]))) |
30541 | 936 |
"proof by contradiction" #> |
937 |
Method.setup @{binding clarify} (cla_method' (CHANGED_PROP oo clarify_tac)) |
|
938 |
"repeatedly apply safe steps" #> |
|
939 |
Method.setup @{binding fast} (cla_method' fast_tac) "classical prover (depth-first)" #> |
|
940 |
Method.setup @{binding slow} (cla_method' slow_tac) "classical prover (slow depth-first)" #> |
|
941 |
Method.setup @{binding best} (cla_method' best_tac) "classical prover (best-first)" #> |
|
42798 | 942 |
Method.setup @{binding deepen} |
943 |
(Scan.lift (Scan.optional Parse.nat 4) --| Method.sections cla_modifiers |
|
944 |
>> (fn n => fn ctxt => SIMPLE_METHOD' (deepen_tac ctxt n))) |
|
30541 | 945 |
"classical prover (iterative deepening)" #> |
946 |
Method.setup @{binding safe} (cla_method (CHANGED_PROP o safe_tac)) |
|
50108 | 947 |
"classical prover (apply safe rules)" #> |
948 |
Method.setup @{binding safe_step} (cla_method' safe_step_tac) |
|
949 |
"single classical step (safe rules)" #> |
|
950 |
Method.setup @{binding inst_step} (cla_method' inst_step_tac) |
|
951 |
"single classical step (safe rules, allow instantiations)" #> |
|
952 |
Method.setup @{binding step} (cla_method' step_tac) |
|
953 |
"single classical step (safe and unsafe rules)" #> |
|
954 |
Method.setup @{binding slow_step} (cla_method' slow_step_tac) |
|
955 |
"single classical step (safe and unsafe rules, allow backtracking)" #> |
|
956 |
Method.setup @{binding clarify_step} (cla_method' clarify_step_tac) |
|
957 |
"single classical step (safe rules, without splitting)"; |
|
5841 | 958 |
|
959 |
||
960 |
||
961 |
(** theory setup **) |
|
962 |
||
26497
1873915c64a9
purely functional setup of claset/simpset/clasimpset;
wenzelm
parents:
26470
diff
changeset
|
963 |
val setup = setup_attrs #> setup_methods; |
5841 | 964 |
|
965 |
||
8667 | 966 |
|
967 |
(** outer syntax **) |
|
968 |
||
24867 | 969 |
val _ = |
46961
5c6955f487e5
outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents:
46874
diff
changeset
|
970 |
Outer_Syntax.improper_command @{command_spec "print_claset"} "print context of Classical Reasoner" |
26497
1873915c64a9
purely functional setup of claset/simpset/clasimpset;
wenzelm
parents:
26470
diff
changeset
|
971 |
(Scan.succeed (Toplevel.no_timing o Toplevel.unknown_context o |
42439
9efdd0af15ac
eliminated Display.string_of_thm_without_context;
wenzelm
parents:
42361
diff
changeset
|
972 |
Toplevel.keep (fn state => |
9efdd0af15ac
eliminated Display.string_of_thm_without_context;
wenzelm
parents:
42361
diff
changeset
|
973 |
let val ctxt = Toplevel.context_of state |
42793 | 974 |
in print_claset ctxt end))); |
8667 | 975 |
|
5841 | 976 |
end; |