author | wenzelm |
Sun, 27 Dec 2020 14:04:27 +0100 | |
changeset 73010 | a569465f8b57 |
parent 72400 | abfeed05c323 |
child 73939 | 9231ea46e041 |
permissions | -rw-r--r-- |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer_prover_minimize.ML |
31037
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
2 |
Author: Philipp Meyer, TU Muenchen |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
3 |
Author: Jasmin Blanchette, TU Muenchen |
31037
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
4 |
|
40977 | 5 |
Minimization of fact list for Metis using external provers. |
31037
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
6 |
*) |
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
7 |
|
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
8 |
signature SLEDGEHAMMER_PROVER_MINIMIZE = |
32525 | 9 |
sig |
46340 | 10 |
type stature = ATP_Problem_Generate.stature |
55287 | 11 |
type proof_method = Sledgehammer_Proof_Methods.proof_method |
12 |
type play_outcome = Sledgehammer_Proof_Methods.play_outcome |
|
55201 | 13 |
type mode = Sledgehammer_Prover.mode |
14 |
type params = Sledgehammer_Prover.params |
|
15 |
type prover = Sledgehammer_Prover.prover |
|
35867 | 16 |
|
55205 | 17 |
val is_prover_supported : Proof.context -> string -> bool |
18 |
val is_prover_installed : Proof.context -> string -> bool |
|
19 |
val default_max_facts_of_prover : Proof.context -> string -> int |
|
20 |
val get_prover : Proof.context -> mode -> string -> prover |
|
21 |
||
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
22 |
val binary_min_facts : int Config.T |
54824 | 23 |
val minimize_facts : (thm list -> unit) -> string -> params -> bool -> int -> int -> |
57734
18bb3e1ff6f6
rationalized preplaying by eliminating (now superfluous) laziness
blanchet
parents:
57732
diff
changeset
|
24 |
Proof.state -> thm -> ((string * stature) * thm list) list -> |
57739 | 25 |
((string * stature) * thm list) list option |
57750 | 26 |
* ((unit -> (string * stature) list * (proof_method * play_outcome)) -> string) |
54503 | 27 |
val get_minimizing_prover : Proof.context -> mode -> (thm list -> unit) -> string -> prover |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
28 |
end; |
32525 | 29 |
|
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
30 |
structure Sledgehammer_Prover_Minimize : SLEDGEHAMMER_PROVER_MINIMIZE = |
31037
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
31 |
struct |
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
32 |
|
43085
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
blanchet
parents:
43064
diff
changeset
|
33 |
open ATP_Util |
39496
a52a4e4399c1
got caught once again by SML's pattern maching (ctor vs. var)
blanchet
parents:
39491
diff
changeset
|
34 |
open ATP_Proof |
46320 | 35 |
open ATP_Problem_Generate |
55212 | 36 |
open ATP_Proof_Reconstruct |
36142
f5e15e9aae10
make Sledgehammer "minimize" output less confusing + round up (not down) time limits to nearest second
blanchet
parents:
36063
diff
changeset
|
37 |
open Sledgehammer_Util |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
38 |
open Sledgehammer_Fact |
55287 | 39 |
open Sledgehammer_Proof_Methods |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
40 |
open Sledgehammer_Isar |
72400 | 41 |
open Sledgehammer_ATP_Systems |
55201 | 42 |
open Sledgehammer_Prover |
55205 | 43 |
open Sledgehammer_Prover_ATP |
58061 | 44 |
open Sledgehammer_Prover_SMT |
55205 | 45 |
|
46 |
fun is_prover_supported ctxt = |
|
47 |
let val thy = Proof_Context.theory_of ctxt in |
|
58061 | 48 |
is_atp thy orf is_smt_prover ctxt |
55205 | 49 |
end |
50 |
||
51 |
fun is_prover_installed ctxt = |
|
58061 | 52 |
is_smt_prover ctxt orf is_atp_installed (Proof_Context.theory_of ctxt) |
55205 | 53 |
|
54 |
fun default_max_facts_of_prover ctxt name = |
|
55 |
let val thy = Proof_Context.theory_of ctxt in |
|
57732 | 56 |
if is_atp thy name then |
55205 | 57 |
fold (Integer.max o fst o #1 o fst o snd) (#best_slices (get_atp thy name ()) ctxt) 0 |
58061 | 58 |
else if is_smt_prover ctxt name then |
59 |
SMT_Solver.default_max_relevant ctxt name |
|
56081 | 60 |
else |
63692 | 61 |
error ("No such prover: " ^ name) |
55205 | 62 |
end |
63 |
||
64 |
fun get_prover ctxt mode name = |
|
65 |
let val thy = Proof_Context.theory_of ctxt in |
|
57732 | 66 |
if is_atp thy name then run_atp mode name |
58061 | 67 |
else if is_smt_prover ctxt name then run_smt_solver mode name |
63692 | 68 |
else error ("No such prover: " ^ name) |
55205 | 69 |
end |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
70 |
|
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
71 |
(* wrapper for calling external prover *) |
31236 | 72 |
|
40061
71cc5aac8b76
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
blanchet
parents:
40060
diff
changeset
|
73 |
fun n_facts names = |
38698
d19c3a7ce38b
clean handling of whether a fact is chained or not;
blanchet
parents:
38696
diff
changeset
|
74 |
let val n = length names in |
40061
71cc5aac8b76
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
blanchet
parents:
40060
diff
changeset
|
75 |
string_of_int n ^ " fact" ^ plural_s n ^ |
57781 | 76 |
(if n > 0 then ": " ^ (names |> map fst |> sort string_ord |> space_implode " ") else "") |
38092
81a003f7de0d
speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents:
38084
diff
changeset
|
77 |
end |
81a003f7de0d
speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents:
38084
diff
changeset
|
78 |
|
58843 | 79 |
fun print silent f = if silent then () else writeln (f ()) |
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
80 |
|
54824 | 81 |
fun test_facts ({debug, verbose, overlord, spy, provers, max_mono_iters, max_new_mono_instances, |
57245 | 82 |
type_enc, strict, lam_trans, uncurried_aliases, isar_proofs, compress, try0, smt_proofs, |
57673
858c1a63967f
don't lose 'minimize' flag before it reaches Isar proof text generation
blanchet
parents:
57245
diff
changeset
|
83 |
minimize, preplay_timeout, ...} : params) |
54824 | 84 |
silent (prover : prover) timeout i n state goal facts = |
31236 | 85 |
let |
57054 | 86 |
val _ = print silent (fn () => "Testing " ^ n_facts (map fst facts) ^ |
87 |
(if verbose then " (timeout: " ^ string_of_time timeout ^ ")" else "") ^ "...") |
|
88 |
||
51005
ce4290c33d73
eliminated needless speed optimization -- and simplified code quite a bit
blanchet
parents:
50669
diff
changeset
|
89 |
val facts = facts |> maps (fn (n, ths) => map (pair n) ths) |
38100
e458a0dd3dc1
use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents:
38094
diff
changeset
|
90 |
val params = |
61311
150aa3015c47
removed legacy asynchronous mode in Sledgehammer
blanchet
parents:
60924
diff
changeset
|
91 |
{debug = debug, verbose = verbose, overlord = overlord, spy = spy, provers = provers, |
150aa3015c47
removed legacy asynchronous mode in Sledgehammer
blanchet
parents:
60924
diff
changeset
|
92 |
type_enc = type_enc, strict = strict, lam_trans = lam_trans, |
53800 | 93 |
uncurried_aliases = uncurried_aliases, learn = false, fact_filter = NONE, |
94 |
max_facts = SOME (length facts), fact_thresholds = (1.01, 1.01), |
|
95 |
max_mono_iters = max_mono_iters, max_new_mono_instances = max_new_mono_instances, |
|
57245 | 96 |
isar_proofs = isar_proofs, compress = compress, try0 = try0, smt_proofs = smt_proofs, |
57673
858c1a63967f
don't lose 'minimize' flag before it reaches Isar proof text generation
blanchet
parents:
57245
diff
changeset
|
97 |
slice = false, minimize = minimize, timeout = timeout, preplay_timeout = preplay_timeout, |
57245 | 98 |
expect = ""} |
40065 | 99 |
val problem = |
54141
f57f8e7a879f
generate a comment storing the goal nickname in "learn_prover"
blanchet
parents:
54130
diff
changeset
|
100 |
{comment = "", state = state, goal = goal, subgoal = i, subgoal_count = n, |
62735 | 101 |
factss = [("", facts)], found_proof = I} |
58654
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
102 |
val result0 as {outcome = outcome0, used_facts, used_from, preferred_methss, run_time, |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
103 |
message} = |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
104 |
prover params problem |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
105 |
val result as {outcome, ...} = |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
106 |
if is_none outcome0 andalso |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
107 |
forall (member (fn ((s, _), ((s', _), _)) => s = s') used_from) used_facts then |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
108 |
result0 |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
109 |
else |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
110 |
{outcome = SOME MaybeUnprovable, used_facts = [], used_from = used_from, |
3e1cad27fc2f
special treatment of extensionality in minimizer
blanchet
parents:
58494
diff
changeset
|
111 |
preferred_methss = preferred_methss, run_time = run_time, message = message} |
36223
217ca1273786
make Sledgehammer's minimizer also minimize Isar proofs
blanchet
parents:
36143
diff
changeset
|
112 |
in |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
113 |
print silent (fn () => |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
114 |
(case outcome of |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
115 |
SOME failure => string_of_atp_failure failure |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
116 |
| NONE => |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
117 |
"Found proof" ^ |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
118 |
(if length used_facts = length facts then "" else " with " ^ n_facts used_facts) ^ |
63692 | 119 |
" (" ^ string_of_time run_time ^ ")")); |
38092
81a003f7de0d
speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents:
38084
diff
changeset
|
120 |
result |
36223
217ca1273786
make Sledgehammer's minimizer also minimize Isar proofs
blanchet
parents:
36143
diff
changeset
|
121 |
end |
31236 | 122 |
|
40204
da97d75e20e6
standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
blanchet
parents:
40200
diff
changeset
|
123 |
(* minimalization of facts *) |
31236 | 124 |
|
45372 | 125 |
(* Give the external prover some slack. The ATP gets further slack because the |
126 |
Sledgehammer preprocessing time is included in the estimate below but isn't |
|
127 |
part of the timeout. *) |
|
128 |
val slack_msecs = 200 |
|
129 |
||
54816
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
130 |
fun new_timeout timeout run_time = |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
131 |
Int.min (Time.toMilliseconds timeout, Time.toMilliseconds run_time + slack_msecs) |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
132 |
|> Time.fromMilliseconds |
45372 | 133 |
|
45367 | 134 |
(* The linear algorithm usually outperforms the binary algorithm when over 60% |
135 |
of the facts are actually needed. The binary algorithm is much more |
|
136 |
appropriate for provers that cannot return the list of used facts and hence |
|
137 |
returns all facts as used. Since we cannot know in advance how many facts are |
|
138 |
actually needed, we heuristically set the threshold to 10 facts. *) |
|
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
139 |
val binary_min_facts = |
69593 | 140 |
Attrib.setup_config_int \<^binding>\<open>sledgehammer_minimize_binary_min_facts\<close> (K 20) |
40977 | 141 |
|
45368 | 142 |
fun linear_minimize test timeout result xs = |
143 |
let |
|
144 |
fun min _ [] p = p |
|
145 |
| min timeout (x :: xs) (seen, result) = |
|
54816
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
146 |
(case test timeout (xs @ seen) of |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
147 |
result as {outcome = NONE, used_facts, run_time, ...} : prover_result => |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
148 |
min (new_timeout timeout run_time) (filter_used_facts true used_facts xs) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
149 |
(filter_used_facts false used_facts seen, result) |
54816
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
150 |
| _ => min timeout xs (x :: seen, result)) |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
151 |
in |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
152 |
min timeout xs ([], result) |
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
153 |
end |
38015 | 154 |
|
45368 | 155 |
fun binary_minimize test timeout result xs = |
40977 | 156 |
let |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
157 |
fun min depth (result as {run_time, ...} : prover_result) sup (xs as _ :: _ :: _) = |
41743 | 158 |
let |
45367 | 159 |
val (l0, r0) = chop (length xs div 2) xs |
41743 | 160 |
(* |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
161 |
val _ = warning (replicate_string depth " " ^ "{ " ^ "sup: " ^ n_facts (map fst sup)) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
162 |
val _ = warning (replicate_string depth " " ^ " " ^ "xs: " ^ n_facts (map fst xs)) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
163 |
val _ = warning (replicate_string depth " " ^ " " ^ "l0: " ^ n_facts (map fst l0)) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
164 |
val _ = warning (replicate_string depth " " ^ " " ^ "r0: " ^ n_facts (map fst r0)) |
41743 | 165 |
*) |
45367 | 166 |
val depth = depth + 1 |
45372 | 167 |
val timeout = new_timeout timeout run_time |
41743 | 168 |
in |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
169 |
(case test timeout (sup @ l0) of |
45372 | 170 |
result as {outcome = NONE, used_facts, ...} => |
48798 | 171 |
min depth result (filter_used_facts true used_facts sup) |
57781 | 172 |
(filter_used_facts true used_facts l0) |
45367 | 173 |
| _ => |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
174 |
(case test timeout (sup @ r0) of |
45367 | 175 |
result as {outcome = NONE, used_facts, ...} => |
48798 | 176 |
min depth result (filter_used_facts true used_facts sup) |
57054 | 177 |
(filter_used_facts true used_facts r0) |
45367 | 178 |
| _ => |
179 |
let |
|
180 |
val (sup_r0, (l, result)) = min depth result (sup @ r0) l0 |
|
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58843
diff
changeset
|
181 |
val (sup, r0) = (sup, r0) |> apply2 (filter_used_facts true (map fst sup_r0)) |
45367 | 182 |
val (sup_l, (r, result)) = min depth result (sup @ l) r0 |
48798 | 183 |
val sup = sup |> filter_used_facts true (map fst sup_l) |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
184 |
in (sup, (l @ r, result)) end)) |
40977 | 185 |
end |
41743 | 186 |
(* |
187 |
|> tap (fn _ => warning (replicate_string depth " " ^ "}")) |
|
188 |
*) |
|
45367 | 189 |
| min _ result sup xs = (sup, (xs, result)) |
190 |
in |
|
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
191 |
(case snd (min 0 result [] xs) of |
45372 | 192 |
([x], result as {run_time, ...}) => |
193 |
(case test (new_timeout timeout run_time) [] of |
|
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
194 |
result as {outcome = NONE, ...} => ([], result) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
195 |
| _ => ([x], result)) |
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
196 |
| p => p) |
45367 | 197 |
end |
40977 | 198 |
|
54816
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
199 |
fun minimize_facts do_learn prover_name (params as {learn, timeout, ...}) silent i n state goal |
57734
18bb3e1ff6f6
rationalized preplaying by eliminating (now superfluous) laziness
blanchet
parents:
57732
diff
changeset
|
200 |
facts = |
31236 | 201 |
let |
40941
a3e6f8634a11
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet
parents:
40553
diff
changeset
|
202 |
val ctxt = Proof.context_of state |
58085 | 203 |
val prover = get_prover ctxt Minimize prover_name |
48796
0f94b8b69e79
consider removing chained facts last, so that they're more likely to be kept
blanchet
parents:
48399
diff
changeset
|
204 |
val (chained, non_chained) = List.partition is_fact_chained facts |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
205 |
|
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
206 |
fun test timeout non_chained = |
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
207 |
test_facts params silent prover timeout i n state goal (chained @ non_chained) |
31236 | 208 |
in |
63692 | 209 |
(print silent (fn () => "Sledgehammer minimizer: " ^ quote prover_name); |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
210 |
(case test timeout non_chained of |
45371 | 211 |
result as {outcome = NONE, used_facts, run_time, ...} => |
38015 | 212 |
let |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
213 |
val non_chained = filter_used_facts true used_facts non_chained |
45372 | 214 |
val min = |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
215 |
if length non_chained >= Config.get ctxt binary_min_facts then binary_minimize |
54815 | 216 |
else linear_minimize |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
217 |
val (min_facts, {message, ...}) = |
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
218 |
min test (new_timeout timeout run_time) result non_chained |
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
219 |
val min_facts_and_chained = chained @ min_facts |
48321 | 220 |
in |
221 |
print silent (fn () => cat_lines |
|
57750 | 222 |
["Minimized to " ^ n_facts (map fst min_facts)] ^ |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
223 |
(case length chained of |
57750 | 224 |
0 => "" |
63692 | 225 |
| n => " (plus " ^ string_of_int n ^ " chained)")); |
59355
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
226 |
(if learn then do_learn (maps snd min_facts_and_chained) else ()); |
533f6cfc04c0
don't minimize chained facts -- this leads to subtle failures, e.g. if a method succeeds without a chained fact but fails with it
blanchet
parents:
59058
diff
changeset
|
227 |
(SOME min_facts_and_chained, message) |
48321 | 228 |
end |
57734
18bb3e1ff6f6
rationalized preplaying by eliminating (now superfluous) laziness
blanchet
parents:
57732
diff
changeset
|
229 |
| {outcome = SOME TimedOut, ...} => |
57738 | 230 |
(NONE, fn _ => |
54816
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
blanchet
parents:
54815
diff
changeset
|
231 |
"Timeout: You can increase the time limit using the \"timeout\" option (e.g., \ |
63692 | 232 |
\timeout = " ^ string_of_int (10 + Time.toMilliseconds timeout div 1000) ^ "\")") |
57738 | 233 |
| {message, ...} => (NONE, (prefix "Prover error: " o message)))) |
234 |
handle ERROR msg => (NONE, fn _ => "Error: " ^ msg) |
|
31236 | 235 |
end |
236 |
||
57732 | 237 |
fun maybe_minimize mode do_learn name (params as {verbose, minimize, ...}) |
55205 | 238 |
({state, goal, subgoal, subgoal_count, ...} : prover_problem) |
57738 | 239 |
(result as {outcome, used_facts, used_from, preferred_methss, run_time, message} |
57734
18bb3e1ff6f6
rationalized preplaying by eliminating (now superfluous) laziness
blanchet
parents:
57732
diff
changeset
|
240 |
: prover_result) = |
58494
ed380b9594b5
always minimize, to reinvoke the prover with nicer options and yield a nicer Isar proof (potentially -- cf. 'full_proof')
blanchet
parents:
58085
diff
changeset
|
241 |
if is_some outcome then |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
242 |
result |
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
243 |
else |
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
244 |
let |
57738 | 245 |
val (used_facts, message) = |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
246 |
if minimize then |
57732 | 247 |
minimize_facts do_learn name params |
54824 | 248 |
(not verbose orelse (mode <> Normal andalso mode <> MaSh)) subgoal subgoal_count state |
57734
18bb3e1ff6f6
rationalized preplaying by eliminating (now superfluous) laziness
blanchet
parents:
57732
diff
changeset
|
249 |
goal (filter_used_facts true used_facts (map (apsnd single) used_from)) |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
250 |
|>> Option.map (map fst) |
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
251 |
else |
57738 | 252 |
(SOME used_facts, message) |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
253 |
in |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
254 |
(case used_facts of |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
255 |
SOME used_facts => |
60924
610794dff23c
tuned signature, in accordance to sortBy in Scala;
wenzelm
parents:
59355
diff
changeset
|
256 |
{outcome = NONE, used_facts = sort_by fst used_facts, used_from = used_from, |
57738 | 257 |
preferred_methss = preferred_methss, run_time = run_time, message = message} |
55202
824c48a539c9
renamed many Sledgehammer ML files to clarify structure
blanchet
parents:
55201
diff
changeset
|
258 |
| NONE => result) |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
259 |
end |
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
260 |
|
57735
056a55b44ec7
eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
blanchet
parents:
57734
diff
changeset
|
261 |
fun get_minimizing_prover ctxt mode do_learn name params problem = |
056a55b44ec7
eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
blanchet
parents:
57734
diff
changeset
|
262 |
get_prover ctxt mode name params problem |
57732 | 263 |
|> maybe_minimize mode do_learn name params problem |
48250
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
blanchet
parents:
48085
diff
changeset
|
264 |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
265 |
end; |