author | blanchet |
Mon, 30 May 2011 17:00:38 +0200 | |
changeset 43052 | 8d6a4978cc65 |
parent 43051 | d7075adac3bd |
child 43058 | 5f8bac7a2945 |
permissions | -rw-r--r-- |
38988 | 1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer_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 |
|
38988 | 8 |
signature SLEDGEHAMMER_MINIMIZE = |
32525 | 9 |
sig |
38988 | 10 |
type locality = Sledgehammer_Filter.locality |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
11 |
type play = Sledgehammer_ATP_Reconstruct.play |
41087
d7b5fd465198
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
blanchet
parents:
40983
diff
changeset
|
12 |
type params = Sledgehammer_Provers.params |
35867 | 13 |
|
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
14 |
val binary_min_facts : int Config.T |
40061
71cc5aac8b76
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
blanchet
parents:
40060
diff
changeset
|
15 |
val minimize_facts : |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
16 |
string -> params -> bool option -> bool -> int -> int -> Proof.state |
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
17 |
-> ((string * locality) * thm list) list |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
18 |
-> ((string * locality) * thm list) list option |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
19 |
* ((unit -> play) * (play -> string)) |
38996 | 20 |
val run_minimize : |
21 |
params -> int -> (Facts.ref * Attrib.src list) list -> Proof.state -> unit |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
22 |
end; |
32525 | 23 |
|
38988 | 24 |
structure Sledgehammer_Minimize : SLEDGEHAMMER_MINIMIZE = |
31037
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
25 |
struct |
ac8669134e7a
added Philipp Meyer's implementation of AtpMinimal
immler@in.tum.de
parents:
diff
changeset
|
26 |
|
39496
a52a4e4399c1
got caught once again by SML's pattern maching (ctor vs. var)
blanchet
parents:
39491
diff
changeset
|
27 |
open ATP_Proof |
36142
f5e15e9aae10
make Sledgehammer "minimize" output less confusing + round up (not down) time limits to nearest second
blanchet
parents:
36063
diff
changeset
|
28 |
open Sledgehammer_Util |
38988 | 29 |
open Sledgehammer_Filter |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
30 |
open Sledgehammer_ATP_Reconstruct |
41087
d7b5fd465198
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
blanchet
parents:
40983
diff
changeset
|
31 |
open Sledgehammer_Provers |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
32 |
|
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
33 |
(* wrapper for calling external prover *) |
31236 | 34 |
|
40061
71cc5aac8b76
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
blanchet
parents:
40060
diff
changeset
|
35 |
fun n_facts names = |
38698
d19c3a7ce38b
clean handling of whether a fact is chained or not;
blanchet
parents:
38696
diff
changeset
|
36 |
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
|
37 |
string_of_int n ^ " fact" ^ plural_s n ^ |
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
|
38 |
(if n > 0 then |
38698
d19c3a7ce38b
clean handling of whether a fact is chained or not;
blanchet
parents:
38696
diff
changeset
|
39 |
": " ^ (names |> map fst |
d19c3a7ce38b
clean handling of whether a fact is chained or not;
blanchet
parents:
38696
diff
changeset
|
40 |
|> sort_distinct string_ord |> space_implode " ") |
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
|
41 |
else |
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
|
42 |
"") |
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
|
43 |
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
|
44 |
|
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
45 |
fun print silent f = if silent then () else Output.urgent_message (f ()) |
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
46 |
|
42724
4d6bcf846759
added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option
blanchet
parents:
42646
diff
changeset
|
47 |
fun test_facts ({debug, verbose, overlord, provers, max_mono_iters, |
42740
31334a7b109d
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
blanchet
parents:
42724
diff
changeset
|
48 |
max_new_mono_instances, type_sys, isar_proof, |
43015
21b6baec55b1
renamed "metis_timeout" to "preplay_timeout" and continued implementation
blanchet
parents:
43011
diff
changeset
|
49 |
isar_shrink_factor, preplay_timeout, ...} : params) |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
50 |
explicit_apply_opt silent (prover : prover) timeout i n state facts = |
31236 | 51 |
let |
43004
20e9caff1f86
fix soundness bug in Sledgehammer: distinguish params in goals from fixed variables in context
blanchet
parents:
42740
diff
changeset
|
52 |
val ctxt = Proof.context_of state |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
53 |
val thy = Proof.theory_of state |
41277
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
54 |
val _ = |
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
55 |
print silent (fn () => |
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
56 |
"Testing " ^ n_facts (map fst facts) ^ |
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
57 |
(if verbose then " (timeout: " ^ string_from_time timeout ^ ")" |
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
58 |
else "") ^ "...") |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
59 |
val {goal, ...} = Proof.goal state |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
60 |
val explicit_apply = |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
61 |
case explicit_apply_opt of |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
62 |
SOME explicit_apply => explicit_apply |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
63 |
| NONE => |
43004
20e9caff1f86
fix soundness bug in Sledgehammer: distinguish params in goals from fixed variables in context
blanchet
parents:
42740
diff
changeset
|
64 |
let val (_, hyp_ts, concl_t) = strip_subgoal ctxt goal i in |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
65 |
not (forall (Meson.is_fol_term thy) |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
66 |
(concl_t :: hyp_ts @ maps (map prop_of o snd) facts)) |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
67 |
end |
38100
e458a0dd3dc1
use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents:
38094
diff
changeset
|
68 |
val params = |
42060
889d767ce5f4
make Minimizer honor "verbose" and "debug" options better
blanchet
parents:
41824
diff
changeset
|
69 |
{debug = debug, verbose = verbose, overlord = overlord, blocking = true, |
41138
eb80538166b6
implemented partially-typed "tags" type encoding
blanchet
parents:
41134
diff
changeset
|
70 |
provers = provers, type_sys = type_sys, explicit_apply = explicit_apply, |
eb80538166b6
implemented partially-typed "tags" type encoding
blanchet
parents:
41134
diff
changeset
|
71 |
relevance_thresholds = (1.01, 1.01), max_relevant = NONE, |
42740
31334a7b109d
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
blanchet
parents:
42724
diff
changeset
|
72 |
max_mono_iters = max_mono_iters, |
31334a7b109d
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
blanchet
parents:
42724
diff
changeset
|
73 |
max_new_mono_instances = max_new_mono_instances, isar_proof = isar_proof, |
31334a7b109d
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
blanchet
parents:
42724
diff
changeset
|
74 |
isar_shrink_factor = isar_shrink_factor, slicing = false, |
43015
21b6baec55b1
renamed "metis_timeout" to "preplay_timeout" and continued implementation
blanchet
parents:
43011
diff
changeset
|
75 |
timeout = timeout, preplay_timeout = preplay_timeout, expect = ""} |
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
|
76 |
val facts = |
41090 | 77 |
facts |> maps (fn (n, ths) => ths |> map (Untranslated_Fact o pair n)) |
40065 | 78 |
val problem = |
79 |
{state = state, goal = goal, subgoal = i, subgoal_count = n, |
|
41741 | 80 |
facts = facts, smt_filter = NONE} |
43050
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
81 |
val result as {outcome, used_facts, run_time_in_msecs, ...} = |
43051 | 82 |
prover params (K (K "")) problem |
36223
217ca1273786
make Sledgehammer's minimizer also minimize Isar proofs
blanchet
parents:
36143
diff
changeset
|
83 |
in |
41277
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
84 |
print silent (fn () => |
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
85 |
case outcome of |
41745 | 86 |
SOME failure => string_for_failure failure |
43050
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
87 |
| NONE => "Found proof" ^ |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
88 |
(if length used_facts = length facts then "" |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
89 |
else " with " ^ n_facts used_facts) ^ |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
90 |
(case run_time_in_msecs of |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
91 |
SOME ms => |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
92 |
" (" ^ string_from_time (Time.fromMilliseconds ms) ^ ")" |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
43043
diff
changeset
|
93 |
| NONE => "") ^ "."); |
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
|
94 |
result |
36223
217ca1273786
make Sledgehammer's minimizer also minimize Isar proofs
blanchet
parents:
36143
diff
changeset
|
95 |
end |
31236 | 96 |
|
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
|
97 |
(* minimalization of facts *) |
31236 | 98 |
|
40977 | 99 |
(* The sublinear algorithm works well in almost all situations, except when the |
100 |
external prover cannot return the list of used facts and hence returns all |
|
41267
958fee9ec275
lower threshold where the binary algorithm kick in and use the same value for automatic minimization
blanchet
parents:
41265
diff
changeset
|
101 |
facts as used. In that case, the binary algorithm is much more appropriate. |
958fee9ec275
lower threshold where the binary algorithm kick in and use the same value for automatic minimization
blanchet
parents:
41265
diff
changeset
|
102 |
We can usually detect the situation by looking at the number of used facts |
958fee9ec275
lower threshold where the binary algorithm kick in and use the same value for automatic minimization
blanchet
parents:
41265
diff
changeset
|
103 |
reported by the prover. *) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
104 |
val binary_min_facts = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
105 |
Attrib.setup_config_int @{binding sledgehammer_minimize_binary_min_facts} |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
106 |
(K 20) |
40977 | 107 |
|
38015 | 108 |
fun sublinear_minimize _ [] p = p |
109 |
| sublinear_minimize test (x :: xs) (seen, result) = |
|
110 |
case test (xs @ seen) of |
|
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
|
111 |
result as {outcome = NONE, used_facts, ...} : prover_result => |
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
|
112 |
sublinear_minimize test (filter_used_facts used_facts xs) |
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
|
113 |
(filter_used_facts used_facts seen, result) |
38015 | 114 |
| _ => sublinear_minimize test xs (x :: seen, result) |
115 |
||
40977 | 116 |
fun binary_minimize test xs = |
117 |
let |
|
118 |
fun p xs = #outcome (test xs : prover_result) = NONE |
|
119 |
fun split [] p = p |
|
120 |
| split [h] (l, r) = (h :: l, r) |
|
121 |
| split (h1 :: h2 :: t) (l, r) = split t (h1 :: l, h2 :: r) |
|
41743 | 122 |
fun min _ _ [] = raise Empty |
123 |
| min _ _ [s0] = [s0] |
|
124 |
| min depth sup xs = |
|
125 |
let |
|
126 |
(* |
|
127 |
val _ = warning (replicate_string depth " " ^ "{" ^ (" " ^ |
|
128 |
n_facts (map fst sup) ^ " and " ^ |
|
129 |
n_facts (map fst xs))) |
|
130 |
*) |
|
131 |
val (l0, r0) = split xs ([], []) |
|
132 |
in |
|
40977 | 133 |
if p (sup @ l0) then |
41743 | 134 |
min (depth + 1) sup l0 |
40977 | 135 |
else if p (sup @ r0) then |
41743 | 136 |
min (depth + 1) sup r0 |
40977 | 137 |
else |
138 |
let |
|
41743 | 139 |
val l = min (depth + 1) (sup @ r0) l0 |
140 |
val r = min (depth + 1) (sup @ l) r0 |
|
40977 | 141 |
in l @ r end |
142 |
end |
|
41743 | 143 |
(* |
144 |
|> tap (fn _ => warning (replicate_string depth " " ^ "}")) |
|
145 |
*) |
|
40977 | 146 |
val xs = |
41743 | 147 |
case min 0 [] xs of |
40977 | 148 |
[x] => if p [] then [] else [x] |
149 |
| xs => xs |
|
150 |
in (xs, test xs) end |
|
151 |
||
152 |
(* Give the external prover some slack. The ATP gets further slack because the |
|
153 |
Sledgehammer preprocessing time is included in the estimate below but isn't |
|
154 |
part of the timeout. *) |
|
41277
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
155 |
val slack_msecs = 200 |
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
|
156 |
|
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
157 |
fun minimize_facts prover_name (params as {timeout, ...}) explicit_apply_opt |
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
158 |
silent i n state facts = |
31236 | 159 |
let |
40941
a3e6f8634a11
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet
parents:
40553
diff
changeset
|
160 |
val ctxt = Proof.context_of state |
43021 | 161 |
val prover = get_prover ctxt Minimize prover_name |
38590
bd443b426d56
get rid of "minimize_timeout", now that there's an automatic adaptive timeout mechanism in "minimize"
blanchet
parents:
38589
diff
changeset
|
162 |
val msecs = Time.toMilliseconds timeout |
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
163 |
val _ = print silent (fn () => "Sledgehammer minimize: " ^ |
40977 | 164 |
quote prover_name ^ ".") |
38100
e458a0dd3dc1
use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents:
38094
diff
changeset
|
165 |
fun do_test timeout = |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
166 |
test_facts params explicit_apply_opt silent prover timeout i n state |
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
|
167 |
val timer = Timer.startRealTimer () |
31236 | 168 |
in |
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
|
169 |
(case do_test timeout facts of |
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
|
170 |
result as {outcome = NONE, used_facts, ...} => |
38015 | 171 |
let |
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
|
172 |
val time = Timer.checkRealTimer timer |
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
|
173 |
val new_timeout = |
41277
1369c27c6966
reduce the minimizer slack and add verbose information
blanchet
parents:
41267
diff
changeset
|
174 |
Int.min (msecs, Time.toMilliseconds time + slack_msecs) |
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
|
175 |
|> Time.fromMilliseconds |
40977 | 176 |
val facts = filter_used_facts used_facts facts |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
177 |
val (min_thms, {preplay, message, ...}) = |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42579
diff
changeset
|
178 |
if length facts >= Config.get ctxt binary_min_facts then |
40977 | 179 |
binary_minimize (do_test new_timeout) facts |
180 |
else |
|
181 |
sublinear_minimize (do_test new_timeout) facts ([], result) |
|
38094 | 182 |
val n = length min_thms |
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
183 |
val _ = print silent (fn () => cat_lines |
40061
71cc5aac8b76
generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
blanchet
parents:
40060
diff
changeset
|
184 |
["Minimized: " ^ string_of_int n ^ " fact" ^ plural_s n] ^ |
38752
6628adcae4a7
consider "locality" when assigning weights to facts
blanchet
parents:
38745
diff
changeset
|
185 |
(case length (filter (curry (op =) Chained o snd o fst) min_thms) of |
38698
d19c3a7ce38b
clean handling of whether a fact is chained or not;
blanchet
parents:
38696
diff
changeset
|
186 |
0 => "" |
41491 | 187 |
| n => " (including " ^ string_of_int n ^ " chained)") ^ ".") |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
188 |
in (SOME min_thms, (preplay, message)) end |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
189 |
| {outcome = SOME TimedOut, preplay, ...} => |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
190 |
(NONE, |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
191 |
(preplay, |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
192 |
fn _ => "Timeout: You can increase the time limit using the \ |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
193 |
\\"timeout\" option (e.g., \"timeout = " ^ |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
194 |
string_of_int (10 + msecs div 1000) ^ "\").")) |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
195 |
| {preplay, message, ...} => |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
196 |
(NONE, (preplay, prefix "Prover error: " o message))) |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
197 |
handle ERROR msg => (NONE, (K Failed_to_Play, fn _ => "Error: " ^ msg)) |
31236 | 198 |
end |
199 |
||
41265
a393d6d8e198
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
blanchet
parents:
41259
diff
changeset
|
200 |
fun run_minimize (params as {provers, ...}) i refs state = |
38045 | 201 |
let |
202 |
val ctxt = Proof.context_of state |
|
38696
4c6b65d6a135
quote facts whose names collide with a keyword or command name (cf. "subclass" in "Jinja/J/TypeSafe.thy")
blanchet
parents:
38617
diff
changeset
|
203 |
val reserved = reserved_isar_keyword_table () |
43043
1406f6fc5dc3
normalize indices in chained facts to make sure that backtick facts (which often result in different names) are recognized + changed definition of urgent messages
blanchet
parents:
43033
diff
changeset
|
204 |
val chained_ths = normalize_chained_theorems (#facts (Proof.goal state)) |
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
|
205 |
val facts = |
41091
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
206 |
refs |
0afdf5cde874
implicitly call the minimizer for SMT solvers that don't return an unsat core
blanchet
parents:
41090
diff
changeset
|
207 |
|> maps (map (apsnd single) o fact_from_ref ctxt reserved chained_ths) |
38045 | 208 |
in |
209 |
case subgoal_count state of |
|
40132
7ee65dbffa31
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
wenzelm
parents:
40114
diff
changeset
|
210 |
0 => Output.urgent_message "No subgoal!" |
41265
a393d6d8e198
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
blanchet
parents:
41259
diff
changeset
|
211 |
| n => case provers of |
a393d6d8e198
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
blanchet
parents:
41259
diff
changeset
|
212 |
[] => error "No prover is set." |
a393d6d8e198
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
blanchet
parents:
41259
diff
changeset
|
213 |
| prover :: _ => |
a393d6d8e198
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
blanchet
parents:
41259
diff
changeset
|
214 |
(kill_provers (); |
41742
11e862c68b40
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet
parents:
41741
diff
changeset
|
215 |
minimize_facts prover params NONE false i n state facts |
43052
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
216 |
|> (fn (_, (preplay, message)) => |
8d6a4978cc65
automatically minimize with Metis when this can be done within a few seconds
blanchet
parents:
43051
diff
changeset
|
217 |
Output.urgent_message (message (preplay ())))) |
38045 | 218 |
end |
219 |
||
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35865
diff
changeset
|
220 |
end; |