author | wenzelm |
Fri, 20 Sep 2024 14:28:13 +0200 | |
changeset 80910 | 406a85a25189 |
parent 80540 | f86bcf439837 |
child 81254 | d3c0734059ee |
permissions | -rw-r--r-- |
55287 | 1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML |
52555 | 2 |
Author: Jasmin Blanchette, TU Muenchen |
3 |
Author: Steffen Juilf Smolka, TU Muenchen |
|
4 |
||
5 |
Reconstructors. |
|
6 |
*) |
|
7 |
||
55287 | 8 |
signature SLEDGEHAMMER_PROOF_METHODS = |
52555 | 9 |
sig |
10 |
type stature = ATP_Problem_Generate.stature |
|
11 |
||
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
12 |
datatype SMT_backend = |
72798
e732c98b02e6
tuned proof preplay to explicitly refer to Z3 backend
desharna
parents:
72518
diff
changeset
|
13 |
SMT_Z3 | |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
14 |
SMT_Verit of string |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
15 |
|
55285 | 16 |
datatype proof_method = |
17 |
Metis_Method of string option * string option | |
|
18 |
Meson_Method | |
|
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
19 |
SMT_Method of SMT_backend | |
56852
b38c5b9cf590
added 'satx' to Sledgehammer's portfolio (cf. 'isar_try0')
blanchet
parents:
56093
diff
changeset
|
20 |
SATx_Method | |
78695 | 21 |
Argo_Method | |
55323
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
22 |
Blast_Method | |
55285 | 23 |
Simp_Method | |
24 |
Auto_Method | |
|
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
25 |
Fastforce_Method | |
55285 | 26 |
Force_Method | |
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
27 |
Moura_Method | |
55323
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
28 |
Linarith_Method | |
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
29 |
Presburger_Method | |
79942
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
30 |
Algebra_Method | |
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
31 |
Order_Method |
52555 | 32 |
|
54824 | 33 |
datatype play_outcome = |
34 |
Played of Time.time | |
|
35 |
Play_Timed_Out of Time.time | |
|
56093 | 36 |
Play_Failed |
52555 | 37 |
|
54824 | 38 |
type one_line_params = |
57739 | 39 |
((string * stature) list * (proof_method * play_outcome)) * string * int * int |
52555 | 40 |
|
57287
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
41 |
val is_proof_method_direct : proof_method -> bool |
72401
2783779b7dd3
removed obsolete unmaintained experimental prover Pirate
blanchet
parents:
70586
diff
changeset
|
42 |
val string_of_proof_method : string list -> proof_method -> string |
57054 | 43 |
val tac_of_proof_method : Proof.context -> thm list * thm list -> proof_method -> int -> tactic |
55211 | 44 |
val string_of_play_outcome : play_outcome -> string |
70586 | 45 |
val play_outcome_ord : play_outcome ord |
56985
82c83978fbd9
correctly add extra facts to lemmas (cf. conjecture and hypotheses) in Z3 Isar proofs
blanchet
parents:
56983
diff
changeset
|
46 |
val one_line_proof_text : Proof.context -> int -> one_line_params -> string |
54495 | 47 |
end; |
52555 | 48 |
|
55287 | 49 |
structure Sledgehammer_Proof_Methods : SLEDGEHAMMER_PROOF_METHODS = |
52555 | 50 |
struct |
51 |
||
54828 | 52 |
open ATP_Util |
52555 | 53 |
open ATP_Problem_Generate |
55211 | 54 |
open ATP_Proof_Reconstruct |
52555 | 55 |
|
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
56 |
datatype SMT_backend = |
72798
e732c98b02e6
tuned proof preplay to explicitly refer to Z3 backend
desharna
parents:
72518
diff
changeset
|
57 |
SMT_Z3 | |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
58 |
SMT_Verit of string |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
59 |
|
55285 | 60 |
datatype proof_method = |
61 |
Metis_Method of string option * string option | |
|
62 |
Meson_Method | |
|
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
63 |
SMT_Method of SMT_backend | |
56852
b38c5b9cf590
added 'satx' to Sledgehammer's portfolio (cf. 'isar_try0')
blanchet
parents:
56093
diff
changeset
|
64 |
SATx_Method | |
78695 | 65 |
Argo_Method | |
55323
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
66 |
Blast_Method | |
55285 | 67 |
Simp_Method | |
68 |
Auto_Method | |
|
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
69 |
Fastforce_Method | |
55285 | 70 |
Force_Method | |
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
71 |
Moura_Method | |
55323
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
72 |
Linarith_Method | |
253a029335a2
split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)
blanchet
parents:
55315
diff
changeset
|
73 |
Presburger_Method | |
79942
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
74 |
Algebra_Method | |
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
75 |
Order_Method |
52555 | 76 |
|
54824 | 77 |
datatype play_outcome = |
78 |
Played of Time.time | |
|
79 |
Play_Timed_Out of Time.time | |
|
56093 | 80 |
Play_Failed |
52555 | 81 |
|
57739 | 82 |
type one_line_params = |
83 |
((string * stature) list * (proof_method * play_outcome)) * string * int * int |
|
55211 | 84 |
|
57287
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
85 |
fun is_proof_method_direct (Metis_Method _) = true |
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
86 |
| is_proof_method_direct Meson_Method = true |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
87 |
| is_proof_method_direct (SMT_Method _) = true |
57287
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
88 |
| is_proof_method_direct Simp_Method = true |
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
89 |
| is_proof_method_direct _ = false |
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
90 |
|
58499
094efe6ac459
don't affect other subgoals with 'auto' in one-liner proofs
blanchet
parents:
58092
diff
changeset
|
91 |
fun is_proof_method_multi_goal Auto_Method = true |
094efe6ac459
don't affect other subgoals with 'auto' in one-liner proofs
blanchet
parents:
58092
diff
changeset
|
92 |
| is_proof_method_multi_goal _ = false |
094efe6ac459
don't affect other subgoals with 'auto' in one-liner proofs
blanchet
parents:
58092
diff
changeset
|
93 |
|
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
94 |
fun maybe_paren s = s |> not (Symbol_Pos.is_identifier s) ? enclose "(" ")" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
95 |
|
80207
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
96 |
(* |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
97 |
Combine indexed fact names for pretty-printing. |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
98 |
Example: [... "assms(1)" "assms(3)" ...] becomes [... "assms(1,3)" ...] |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
99 |
Combines only adjacent same names. |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
100 |
Input should not have same name with and without index. |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
101 |
*) |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
102 |
fun merge_indexed_facts (ss: string list) :string list = |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
103 |
let |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
104 |
|
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
105 |
fun split (s: string) : string * string = |
80540 | 106 |
if String.isPrefix "\<open>" s then (s,"") |
107 |
else |
|
108 |
case first_field "(" s of |
|
109 |
NONE => (s,"") |
|
110 |
| SOME (name,isp) => (name, String.substring (isp, 0, size isp - 1)) |
|
80207
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
111 |
|
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
112 |
fun merge ((name1,is1) :: (name2,is2) :: zs) = |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
113 |
if name1 = name2 |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
114 |
then merge ((name1,is1 ^ "," ^ is2) :: zs) |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
115 |
else (name1,is1) :: merge ((name2,is2) :: zs) |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
116 |
| merge xs = xs; |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
117 |
|
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
118 |
fun parents is = if is = "" then "" else "(" ^ is ^ ")" |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
119 |
|
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
120 |
in |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
121 |
map (fn (name,is) => name ^ parents is) (merge (map split ss)) |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
122 |
end |
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
123 |
|
72401
2783779b7dd3
removed obsolete unmaintained experimental prover Pirate
blanchet
parents:
70586
diff
changeset
|
124 |
fun string_of_proof_method ss meth = |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
125 |
let |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
126 |
val meth_s = |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
127 |
(case meth of |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
128 |
Metis_Method (NONE, NONE) => "metis" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
129 |
| Metis_Method (type_enc_opt, lam_trans_opt) => |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
130 |
"metis (" ^ commas (map_filter I [type_enc_opt, lam_trans_opt]) ^ ")" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
131 |
| Meson_Method => "meson" |
72798
e732c98b02e6
tuned proof preplay to explicitly refer to Z3 backend
desharna
parents:
72518
diff
changeset
|
132 |
| SMT_Method SMT_Z3 => "smt (z3)" |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
133 |
| SMT_Method (SMT_Verit strategy) => |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
134 |
"smt (" ^ commas ("verit" :: (if strategy = "default" then [] else [strategy])) ^ ")" |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
135 |
| SATx_Method => "satx" |
78695 | 136 |
| Argo_Method => "argo" |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
137 |
| Blast_Method => "blast" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
138 |
| Simp_Method => if null ss then "simp" else "simp add:" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
139 |
| Auto_Method => "auto" |
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
140 |
| Fastforce_Method => "fastforce" |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
141 |
| Force_Method => "force" |
58092
4ae52c60603a
renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
blanchet
parents:
58075
diff
changeset
|
142 |
| Moura_Method => "moura" |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
143 |
| Linarith_Method => "linarith" |
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
144 |
| Presburger_Method => "presburger" |
79942
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
145 |
| Algebra_Method => "algebra" |
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
146 |
| Order_Method => "order") |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
147 |
in |
80910 | 148 |
maybe_paren (implode_space (meth_s :: merge_indexed_facts ss)) |
56983
132142089ea6
use 'simp add:' syntax in Sledgehammer rather than 'using'
blanchet
parents:
56965
diff
changeset
|
149 |
end |
55285 | 150 |
|
57054 | 151 |
fun tac_of_proof_method ctxt (local_facts, global_facts) meth = |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
152 |
let |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
153 |
fun tac_of_metis (type_enc_opt, lam_trans_opt) = |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
154 |
let |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
155 |
val ctxt = ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
156 |
|> Config.put Metis_Tactic.verbose false |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
157 |
|> Config.put Metis_Tactic.trace false |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
158 |
in |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
159 |
SELECT_GOAL (Metis_Tactic.metis_method ((Option.map single type_enc_opt, lam_trans_opt), |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
160 |
global_facts) ctxt local_facts) |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
161 |
end |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
162 |
|
72798
e732c98b02e6
tuned proof preplay to explicitly refer to Z3 backend
desharna
parents:
72518
diff
changeset
|
163 |
fun tac_of_smt SMT_Z3 = SMT_Solver.smt_tac |
75956
1e2a9d2251b0
remove duplicate parsing for alethe; fix skolemization;
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents:
75040
diff
changeset
|
164 |
| tac_of_smt (SMT_Verit strategy) = Verit_Strategies.verit_tac_stgy strategy |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
165 |
in |
55285 | 166 |
(case meth of |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
167 |
Metis_Method options => tac_of_metis options |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
168 |
| SMT_Method backend => tac_of_smt backend ctxt (local_facts @ global_facts) |
62219
dbac573b27e7
preplaying of 'smt' and 'metis' more in sync with actual method
blanchet
parents:
61841
diff
changeset
|
169 |
| _ => |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
170 |
Method.insert_tac ctxt local_facts THEN' |
62219
dbac573b27e7
preplaying of 'smt' and 'metis' more in sync with actual method
blanchet
parents:
61841
diff
changeset
|
171 |
(case meth of |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
172 |
Meson_Method => Meson_Tactic.meson_general_tac ctxt global_facts |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
173 |
| Simp_Method => Simplifier.asm_full_simp_tac (ctxt addsimps global_facts) |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
174 |
| _ => |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
175 |
Method.insert_tac ctxt global_facts THEN' |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
176 |
(case meth of |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
177 |
SATx_Method => SAT.satx_tac ctxt |
78695 | 178 |
| Argo_Method => Argo_Tactic.argo_tac ctxt [] |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
179 |
| Blast_Method => blast_tac ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
180 |
| Auto_Method => SELECT_GOAL (Clasimp.auto_tac ctxt) |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
181 |
| Fastforce_Method => Clasimp.fast_force_tac ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
182 |
| Force_Method => Clasimp.force_tac ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
183 |
| Moura_Method => moura_tac ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
184 |
| Linarith_Method => Lin_Arith.tac ctxt |
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
185 |
| Presburger_Method => Cooper.tac true [] [] ctxt |
79942
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
186 |
| Algebra_Method => Groebner.algebra_tac [] [] ctxt |
7793e3161d2b
try proof method "order" in Sledgehammer's proof reconstruction
desharna
parents:
78736
diff
changeset
|
187 |
| Order_Method => HOL_Order_Tac.tac [] ctxt))) |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
188 |
end |
55211 | 189 |
|
54828 | 190 |
fun string_of_play_outcome (Played time) = string_of_ext_time (false, time) |
56093 | 191 |
| string_of_play_outcome (Play_Timed_Out time) = |
192 |
if time = Time.zeroTime then "" else string_of_ext_time (true, time) ^ ", timed out" |
|
54828 | 193 |
| string_of_play_outcome Play_Failed = "failed" |
194 |
||
78736
45867a453a3f
used standard Time.compare in Sledgehammer's preplay
desharna
parents:
78695
diff
changeset
|
195 |
fun play_outcome_ord (Played time1, Played time2) = Time.compare (time1, time2) |
55269 | 196 |
| play_outcome_ord (Played _, _) = LESS |
197 |
| play_outcome_ord (_, Played _) = GREATER |
|
78736
45867a453a3f
used standard Time.compare in Sledgehammer's preplay
desharna
parents:
78695
diff
changeset
|
198 |
| play_outcome_ord (Play_Timed_Out time1, Play_Timed_Out time2) = Time.compare (time1, time2) |
55269 | 199 |
| play_outcome_ord (Play_Timed_Out _, _) = LESS |
200 |
| play_outcome_ord (_, Play_Timed_Out _) = GREATER |
|
201 |
| play_outcome_ord (Play_Failed, Play_Failed) = EQUAL |
|
202 |
||
55211 | 203 |
fun apply_on_subgoal _ 1 = "by " |
204 |
| apply_on_subgoal 1 _ = "apply " |
|
57287
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
205 |
| apply_on_subgoal i n = "prefer " ^ string_of_int i ^ " " ^ apply_on_subgoal 1 n |
55211 | 206 |
|
55285 | 207 |
(* FIXME *) |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
208 |
fun proof_method_command meth i n used_chaineds _(*num_chained*) extras = |
60252
2c468c062589
improved one-line preplaying (don't rely on 'using x by simp' to mean 'by (simp add: x)' and beware of inaccessible '(local.)this')
blanchet
parents:
59058
diff
changeset
|
209 |
let |
2c468c062589
improved one-line preplaying (don't rely on 'using x by simp' to mean 'by (simp add: x)' and beware of inaccessible '(local.)this')
blanchet
parents:
59058
diff
changeset
|
210 |
val (indirect_ss, direct_ss) = |
73975
8d93f9ca6518
revisited ac28714b7478: more faithful preplaying with chained facts
blanchet
parents:
72798
diff
changeset
|
211 |
if is_proof_method_direct meth then ([], extras) else (extras, []) |
60252
2c468c062589
improved one-line preplaying (don't rely on 'using x by simp' to mean 'by (simp add: x)' and beware of inaccessible '(local.)this')
blanchet
parents:
59058
diff
changeset
|
212 |
in |
80207
ca7e7e41374e
pretty-printing sledgehammer command: merge indexed theorems
nipkow
parents:
79942
diff
changeset
|
213 |
(if null indirect_ss then "" |
80910 | 214 |
else "using " ^ implode_space (merge_indexed_facts indirect_ss) ^ " ") ^ |
72401
2783779b7dd3
removed obsolete unmaintained experimental prover Pirate
blanchet
parents:
70586
diff
changeset
|
215 |
apply_on_subgoal i n ^ string_of_proof_method direct_ss meth ^ |
58499
094efe6ac459
don't affect other subgoals with 'auto' in one-liner proofs
blanchet
parents:
58092
diff
changeset
|
216 |
(if is_proof_method_multi_goal meth andalso n <> 1 then "[1]" else "") |
57287
68aa585269ac
given two one-liners, only show the best of the two
blanchet
parents:
57054
diff
changeset
|
217 |
end |
55211 | 218 |
|
56093 | 219 |
fun try_command_line banner play command = |
220 |
let val s = string_of_play_outcome play in |
|
75040 | 221 |
banner ^ Active.sendback_markup_command command ^ (s |> s <> "" ? enclose " (" ")") |
56093 | 222 |
end |
52555 | 223 |
|
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
224 |
fun one_line_proof_text _ num_chained |
57739 | 225 |
((used_facts, (meth, play)), banner, subgoal, subgoal_count) = |
57777 | 226 |
let val (chained, extra) = List.partition (fn (_, (sc, _)) => sc = Chained) used_facts in |
57735
056a55b44ec7
eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
blanchet
parents:
57720
diff
changeset
|
227 |
map fst extra |
72518
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
desharna
parents:
72401
diff
changeset
|
228 |
|> proof_method_command meth subgoal subgoal_count (map fst chained) num_chained |
63692 | 229 |
|> (if play = Play_Failed then prefix "One-line proof reconstruction failed: " |
57735
056a55b44ec7
eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
blanchet
parents:
57720
diff
changeset
|
230 |
else try_command_line banner play) |
55211 | 231 |
end |
52555 | 232 |
|
54495 | 233 |
end; |