author | blanchet |
Thu, 21 Oct 2010 16:25:40 +0200 | |
changeset 40060 | 5ef6747aa619 |
parent 40059 | 6ad9081665db |
child 40061 | 71cc5aac8b76 |
permissions | -rw-r--r-- |
38021
e024504943d1
rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents:
38020
diff
changeset
|
1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer.ML |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
2 |
Author: Fabian Immler, TU Muenchen |
32996
d2e48879e65a
removed disjunctive group cancellation -- provers run independently;
wenzelm
parents:
32995
diff
changeset
|
3 |
Author: Makarius |
35969 | 4 |
Author: Jasmin Blanchette, TU Muenchen |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
5 |
|
38021
e024504943d1
rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents:
38020
diff
changeset
|
6 |
Sledgehammer's heart. |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
7 |
*) |
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
8 |
|
38021
e024504943d1
rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents:
38020
diff
changeset
|
9 |
signature SLEDGEHAMMER = |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
10 |
sig |
38023 | 11 |
type failure = ATP_Systems.failure |
38988 | 12 |
type locality = Sledgehammer_Filter.locality |
13 |
type relevance_override = Sledgehammer_Filter.relevance_override |
|
39004
f1b465f889b5
translate the axioms to FOF once and for all ATPs
blanchet
parents:
39003
diff
changeset
|
14 |
type fol_formula = Sledgehammer_Translate.fol_formula |
38988 | 15 |
type minimize_command = Sledgehammer_Reconstruct.minimize_command |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
16 |
|
35969 | 17 |
type params = |
38982
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
18 |
{blocking: bool, |
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
19 |
debug: bool, |
35969 | 20 |
verbose: bool, |
36143
6490319b1703
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet
parents:
36064
diff
changeset
|
21 |
overlord: bool, |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
22 |
provers: string list, |
35969 | 23 |
full_types: bool, |
36235
61159615a0c5
added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)
blanchet
parents:
36231
diff
changeset
|
24 |
explicit_apply: bool, |
38745
ad577fd62ee4
reorganize options regarding to the relevance threshold and decay
blanchet
parents:
38744
diff
changeset
|
25 |
relevance_thresholds: real * real, |
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
26 |
max_relevant: int option, |
35969 | 27 |
isar_proof: bool, |
36924 | 28 |
isar_shrink_factor: int, |
38985
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
29 |
timeout: Time.time, |
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
30 |
expect: string} |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
31 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
32 |
type atp_problem = |
39318 | 33 |
{state: Proof.state, |
38998 | 34 |
goal: thm, |
35 |
subgoal: int, |
|
39366
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
36 |
axioms: (term * ((string * locality) * fol_formula) option) list, |
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
37 |
only: bool} |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
38 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
39 |
type atp_result = |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
40 |
{outcome: failure option, |
35969 | 41 |
message: string, |
37926
e6ff246c0cdb
renamings + only need second component of name pool to reconstruct proofs
blanchet
parents:
37627
diff
changeset
|
42 |
pool: string Symtab.table, |
38752
6628adcae4a7
consider "locality" when assigning weights to facts
blanchet
parents:
38748
diff
changeset
|
43 |
used_thm_names: (string * locality) list, |
35969 | 44 |
atp_run_time_in_msecs: int, |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
45 |
output: string, |
39452 | 46 |
tstplike_proof: string, |
38818
61cf050f8b2e
improve SPASS hack, when a clause comes from several facts
blanchet
parents:
38752
diff
changeset
|
47 |
axiom_names: (string * locality) list vector, |
38083
c4b57f68ddb3
remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents:
38061
diff
changeset
|
48 |
conjecture_shape: int list list} |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
49 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
50 |
type atp = params -> minimize_command -> atp_problem -> atp_result |
35867 | 51 |
|
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
52 |
val smtN : string |
38023 | 53 |
val dest_dir : string Config.T |
54 |
val problem_prefix : string Config.T |
|
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
55 |
val measure_run_time : bool Config.T |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
56 |
val available_provers : theory -> unit |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
57 |
val kill_provers : unit -> unit |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
58 |
val running_provers : unit -> unit |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
59 |
val messages : int option -> unit |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
60 |
val run_atp : theory -> string -> atp |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
61 |
val run_smt_solver : |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
62 |
Proof.context -> bool -> Time.time -> ('a * thm) list -> string * 'a list |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
63 |
val is_smt_solver_installed : unit -> bool |
38044 | 64 |
val run_sledgehammer : |
39318 | 65 |
params -> bool -> int -> relevance_override -> (string -> minimize_command) |
66 |
-> Proof.state -> bool * Proof.state |
|
38023 | 67 |
val setup : theory -> theory |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
68 |
end; |
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
69 |
|
38021
e024504943d1
rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents:
38020
diff
changeset
|
70 |
structure Sledgehammer : SLEDGEHAMMER = |
28477
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
71 |
struct |
9339d4dcec8b
version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff
changeset
|
72 |
|
38028 | 73 |
open ATP_Problem |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39453
diff
changeset
|
74 |
open ATP_Proof |
38028 | 75 |
open ATP_Systems |
39494
bf7dd4902321
rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
blanchet
parents:
39493
diff
changeset
|
76 |
open Metis_Translate |
38023 | 77 |
open Sledgehammer_Util |
38988 | 78 |
open Sledgehammer_Filter |
38282
319c59682c51
move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents:
38277
diff
changeset
|
79 |
open Sledgehammer_Translate |
38988 | 80 |
open Sledgehammer_Reconstruct |
37583
9ce2451647d5
factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents:
37581
diff
changeset
|
81 |
|
38023 | 82 |
|
37583
9ce2451647d5
factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents:
37581
diff
changeset
|
83 |
(** The Sledgehammer **) |
9ce2451647d5
factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents:
37581
diff
changeset
|
84 |
|
38102
019a49759829
fix bug in the newly introduced "bound concealing" code
blanchet
parents:
38100
diff
changeset
|
85 |
(* Identifier to distinguish Sledgehammer from other tools using |
019a49759829
fix bug in the newly introduced "bound concealing" code
blanchet
parents:
38100
diff
changeset
|
86 |
"Async_Manager". *) |
37585 | 87 |
val das_Tool = "Sledgehammer" |
88 |
||
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
89 |
val smtN = "smt" |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
90 |
val smt_names = [smtN, remote_prefix ^ smtN] |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
91 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
92 |
fun available_provers thy = |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
93 |
let |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
94 |
val (remote_provers, local_provers) = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
95 |
sort_strings (available_atps thy) @ smt_names |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
96 |
|> List.partition (String.isPrefix remote_prefix) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
97 |
in |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
98 |
priority ("Available provers: " ^ commas (local_provers @ remote_provers) ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
99 |
".") |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
100 |
end |
35969 | 101 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
102 |
fun kill_provers () = Async_Manager.kill_threads das_Tool "provers" |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
103 |
fun running_provers () = Async_Manager.running_threads das_Tool "provers" |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
104 |
val messages = Async_Manager.thread_messages das_Tool "prover" |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
105 |
|
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
106 |
(** problems, results, ATPs, etc. **) |
35969 | 107 |
|
108 |
type params = |
|
38982
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
109 |
{blocking: bool, |
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
110 |
debug: bool, |
35969 | 111 |
verbose: bool, |
36143
6490319b1703
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet
parents:
36064
diff
changeset
|
112 |
overlord: bool, |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
113 |
provers: string list, |
35969 | 114 |
full_types: bool, |
36235
61159615a0c5
added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)
blanchet
parents:
36231
diff
changeset
|
115 |
explicit_apply: bool, |
38745
ad577fd62ee4
reorganize options regarding to the relevance threshold and decay
blanchet
parents:
38744
diff
changeset
|
116 |
relevance_thresholds: real * real, |
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
117 |
max_relevant: int option, |
35969 | 118 |
isar_proof: bool, |
36924 | 119 |
isar_shrink_factor: int, |
38985
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
120 |
timeout: Time.time, |
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
121 |
expect: string} |
35867 | 122 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
123 |
type atp_problem = |
39318 | 124 |
{state: Proof.state, |
38998 | 125 |
goal: thm, |
126 |
subgoal: int, |
|
39366
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
127 |
axioms: (term * ((string * locality) * fol_formula) option) list, |
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
128 |
only: bool} |
35867 | 129 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
130 |
type atp_result = |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
131 |
{outcome: failure option, |
35969 | 132 |
message: string, |
37926
e6ff246c0cdb
renamings + only need second component of name pool to reconstruct proofs
blanchet
parents:
37627
diff
changeset
|
133 |
pool: string Symtab.table, |
38752
6628adcae4a7
consider "locality" when assigning weights to facts
blanchet
parents:
38748
diff
changeset
|
134 |
used_thm_names: (string * locality) list, |
35969 | 135 |
atp_run_time_in_msecs: int, |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
136 |
output: string, |
39452 | 137 |
tstplike_proof: string, |
38818
61cf050f8b2e
improve SPASS hack, when a clause comes from several facts
blanchet
parents:
38752
diff
changeset
|
138 |
axiom_names: (string * locality) list vector, |
38083
c4b57f68ddb3
remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents:
38061
diff
changeset
|
139 |
conjecture_shape: int list list} |
35867 | 140 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
141 |
type atp = params -> minimize_command -> atp_problem -> atp_result |
35867 | 142 |
|
38023 | 143 |
(* configuration attributes *) |
144 |
||
38991 | 145 |
val (dest_dir, dest_dir_setup) = |
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
146 |
Attrib.config_string "sledgehammer_dest_dir" (K "") |
38991 | 147 |
(* Empty string means create files in Isabelle's temporary files directory. *) |
38023 | 148 |
|
149 |
val (problem_prefix, problem_prefix_setup) = |
|
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
150 |
Attrib.config_string "sledgehammer_problem_prefix" (K "prob") |
38023 | 151 |
|
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
152 |
val (measure_run_time, measure_run_time_setup) = |
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
153 |
Attrib.config_bool "sledgehammer_measure_run_time" (K false) |
28484 | 154 |
|
38023 | 155 |
fun with_path cleanup after f path = |
156 |
Exn.capture f path |
|
157 |
|> tap (fn _ => cleanup path) |
|
158 |
|> Exn.release |
|
159 |
|> tap (after path) |
|
160 |
||
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
161 |
fun prover_description ctxt ({blocking, verbose, ...} : params) name num_axioms |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
162 |
i n goal = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
163 |
quote name ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
164 |
(if verbose then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
165 |
" with " ^ string_of_int num_axioms ^ " fact" ^ plural_s num_axioms |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
166 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
167 |
"") ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
168 |
" on " ^ (if n = 1 then "goal" else "subgoal " ^ string_of_int i) ^ ":" ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
169 |
(if blocking then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
170 |
"" |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
171 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
172 |
"\n" ^ Syntax.string_of_term ctxt (Thm.term_of (Thm.cprem_of goal i))) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
173 |
|
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
174 |
fun proof_banner auto = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
175 |
if auto then "Sledgehammer found a proof" else "Try this command" |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
176 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
177 |
(* generic TPTP-based ATPs *) |
38023 | 178 |
|
39492 | 179 |
(* Important messages are important but not so important that users want to see |
180 |
them each time. *) |
|
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
181 |
val important_message_keep_factor = 0.1 |
39492 | 182 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
183 |
fun atp_fun auto atp_name |
38645 | 184 |
{exec, required_execs, arguments, has_incomplete_mode, proof_delims, |
38997 | 185 |
known_failures, default_max_relevant, explicit_forall, |
186 |
use_conjecture_for_hypotheses} |
|
38455 | 187 |
({debug, verbose, overlord, full_types, explicit_apply, |
38998 | 188 |
max_relevant, isar_proof, isar_shrink_factor, timeout, ...} : params) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
189 |
minimize_command ({state, goal, subgoal, axioms, only} : atp_problem) = |
38023 | 190 |
let |
39318 | 191 |
val ctxt = Proof.context_of state |
38998 | 192 |
val (_, hyp_ts, concl_t) = strip_subgoal goal subgoal |
39366
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
193 |
val axioms = axioms |> not only |
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
194 |
? take (the_default default_max_relevant max_relevant) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
195 |
val dest_dir = if overlord then getenv "ISABELLE_HOME_USER" |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
196 |
else Config.get ctxt dest_dir |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
197 |
val problem_prefix = Config.get ctxt problem_prefix |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
198 |
val atp_problem_file_name = |
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
199 |
Path.basic ((if overlord then "prob_" ^ atp_name |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
200 |
else problem_prefix ^ serial_string ()) |
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
201 |
^ "_" ^ string_of_int subgoal) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
202 |
val atp_problem_path_name = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
203 |
if dest_dir = "" then |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
204 |
File.tmp_path atp_problem_file_name |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
205 |
else if File.exists (Path.explode dest_dir) then |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
206 |
Path.append (Path.explode dest_dir) atp_problem_file_name |
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
207 |
else |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
208 |
error ("No such directory: " ^ quote dest_dir ^ ".") |
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
209 |
val measure_run_time = verbose orelse Config.get ctxt measure_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:
38091
diff
changeset
|
210 |
val command = Path.explode (getenv (fst exec) ^ "/" ^ snd exec) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
211 |
(* write out problem file and call ATP *) |
38645 | 212 |
fun command_line complete timeout probfile = |
38023 | 213 |
let |
214 |
val core = File.shell_path command ^ " " ^ arguments complete timeout ^ |
|
215 |
" " ^ File.shell_path probfile |
|
216 |
in |
|
39010 | 217 |
(if measure_run_time then "TIMEFORMAT='%3R'; { time " ^ core ^ " ; }" |
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
218 |
else "exec " ^ core) ^ " 2>&1" |
38023 | 219 |
end |
220 |
fun split_time s = |
|
221 |
let |
|
222 |
val split = String.tokens (fn c => str c = "\n"); |
|
223 |
val (output, t) = s |> split |> split_last |> apfst cat_lines; |
|
224 |
fun as_num f = f >> (fst o read_int); |
|
225 |
val num = as_num (Scan.many1 Symbol.is_ascii_digit); |
|
226 |
val digit = Scan.one Symbol.is_ascii_digit; |
|
227 |
val num3 = as_num (digit ::: digit ::: (digit >> single)); |
|
228 |
val time = num --| Scan.$$ "." -- num3 >> (fn (a, b) => a * 1000 + b); |
|
229 |
val as_time = the_default 0 o Scan.read Symbol.stopper time o explode; |
|
230 |
in (output, as_time t) end; |
|
231 |
fun run_on probfile = |
|
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:
38091
diff
changeset
|
232 |
case filter (curry (op =) "" o getenv o fst) (exec :: required_execs) of |
38032 | 233 |
(home_var, _) :: _ => |
38023 | 234 |
error ("The environment variable " ^ quote home_var ^ " is not set.") |
38032 | 235 |
| [] => |
236 |
if File.exists command then |
|
237 |
let |
|
39318 | 238 |
fun run complete timeout = |
38032 | 239 |
let |
38645 | 240 |
val command = command_line complete timeout probfile |
38032 | 241 |
val ((output, msecs), res_code) = |
242 |
bash_output command |
|
243 |
|>> (if overlord then |
|
244 |
prefix ("% " ^ command ^ "\n% " ^ timestamp () ^ "\n") |
|
245 |
else |
|
246 |
I) |
|
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
247 |
|>> (if measure_run_time then split_time else rpair 0) |
39452 | 248 |
val (tstplike_proof, outcome) = |
249 |
extract_tstplike_proof_and_outcome complete res_code |
|
250 |
proof_delims known_failures output |
|
251 |
in (output, msecs, tstplike_proof, outcome) end |
|
38032 | 252 |
val readable_names = debug andalso overlord |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
253 |
val (atp_problem, pool, conjecture_offset, axiom_names) = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
254 |
prepare_atp_problem ctxt readable_names explicit_forall full_types |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
255 |
explicit_apply hyp_ts concl_t axioms |
39452 | 256 |
val ss = tptp_strings_for_atp_problem use_conjecture_for_hypotheses |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
257 |
atp_problem |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38600
diff
changeset
|
258 |
val _ = File.write_list probfile ss |
38032 | 259 |
val conjecture_shape = |
260 |
conjecture_offset + 1 upto conjecture_offset + length hyp_ts + 1 |
|
38040
174568533593
fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
blanchet
parents:
38039
diff
changeset
|
261 |
|> map single |
39318 | 262 |
val run_twice = has_incomplete_mode andalso not auto |
38645 | 263 |
val timer = Timer.startRealTimer () |
38032 | 264 |
val result = |
39318 | 265 |
run false (if run_twice then |
266 |
Time.fromMilliseconds |
|
38645 | 267 |
(2 * Time.toMilliseconds timeout div 3) |
39318 | 268 |
else |
269 |
timeout) |
|
270 |
|> run_twice |
|
38645 | 271 |
? (fn (_, msecs0, _, SOME _) => |
39318 | 272 |
run true (Time.- (timeout, Timer.checkRealTimer timer)) |
39452 | 273 |
|> (fn (output, msecs, tstplike_proof, outcome) => |
274 |
(output, msecs0 + msecs, tstplike_proof, outcome)) |
|
38645 | 275 |
| result => result) |
38282
319c59682c51
move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents:
38277
diff
changeset
|
276 |
in ((pool, conjecture_shape, axiom_names), result) end |
38032 | 277 |
else |
278 |
error ("Bad executable: " ^ Path.implode command ^ ".") |
|
38023 | 279 |
|
280 |
(* If the problem file has not been exported, remove it; otherwise, export |
|
281 |
the proof file too. *) |
|
282 |
fun cleanup probfile = |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
283 |
if dest_dir = "" then try File.rm probfile else NONE |
38023 | 284 |
fun export probfile (_, (output, _, _, _)) = |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
285 |
if dest_dir = "" then |
38023 | 286 |
() |
287 |
else |
|
288 |
File.write (Path.explode (Path.implode probfile ^ "_proof")) output |
|
38282
319c59682c51
move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents:
38277
diff
changeset
|
289 |
val ((pool, conjecture_shape, axiom_names), |
39452 | 290 |
(output, msecs, tstplike_proof, outcome)) = |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
291 |
with_path cleanup export run_on atp_problem_path_name |
38282
319c59682c51
move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents:
38277
diff
changeset
|
292 |
val (conjecture_shape, axiom_names) = |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
293 |
repair_conjecture_shape_and_axiom_names output conjecture_shape |
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
294 |
axiom_names |
39492 | 295 |
val important_message = |
39493
cb2208f2c07d
move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
blanchet
parents:
39492
diff
changeset
|
296 |
if random () <= important_message_keep_factor then |
39492 | 297 |
extract_important_message output |
298 |
else |
|
299 |
"" |
|
38023 | 300 |
val (message, used_thm_names) = |
301 |
case outcome of |
|
302 |
NONE => |
|
303 |
proof_text isar_proof |
|
304 |
(pool, debug, isar_shrink_factor, ctxt, conjecture_shape) |
|
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
305 |
(proof_banner auto, full_types, minimize_command, tstplike_proof, |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
306 |
axiom_names, goal, subgoal) |
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
307 |
|>> (fn message => |
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
308 |
message ^ (if verbose then |
39371 | 309 |
"\nATP real CPU time: " ^ string_of_int msecs ^ |
310 |
" ms." |
|
38744
2b6333f78a9e
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
blanchet
parents:
38741
diff
changeset
|
311 |
else |
39107
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
312 |
"") ^ |
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
313 |
(if important_message <> "" then |
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
314 |
"\n\nImportant message from Dr. Geoff Sutcliffe:\n" ^ |
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
315 |
important_message |
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
316 |
else |
0a62f8a94af3
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
blanchet
parents:
39010
diff
changeset
|
317 |
"")) |
38597
db482afec7f0
no spurious trailing "\n" at the end of Sledgehammer's output
blanchet
parents:
38590
diff
changeset
|
318 |
| SOME failure => (string_for_failure failure, []) |
38023 | 319 |
in |
320 |
{outcome = outcome, message = message, pool = pool, |
|
321 |
used_thm_names = used_thm_names, atp_run_time_in_msecs = msecs, |
|
39452 | 322 |
output = output, tstplike_proof = tstplike_proof, |
323 |
axiom_names = axiom_names, conjecture_shape = conjecture_shape} |
|
38023 | 324 |
end |
325 |
||
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
326 |
fun run_atp thy name = atp_fun false name (get_atp thy name) |
38023 | 327 |
|
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
328 |
fun run_atp_somehow (params as {blocking, debug, max_relevant, timeout, |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
329 |
expect, ...}) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
330 |
auto i n minimize_command |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
331 |
(atp_problem as {state, goal, axioms, ...}) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
332 |
(atp as {default_max_relevant, ...}, atp_name) = |
36379
20ef039bccff
make "ATP_Manager.get_prover" a total function, since we always want to show the same error text
blanchet
parents:
36373
diff
changeset
|
333 |
let |
39318 | 334 |
val ctxt = Proof.context_of state |
37584 | 335 |
val birth_time = Time.now () |
336 |
val death_time = Time.+ (birth_time, timeout) |
|
39110
a74bd9bfa880
show the number of facts for each prover in "verbose" mode
blanchet
parents:
39108
diff
changeset
|
337 |
val max_relevant = the_default default_max_relevant max_relevant |
a74bd9bfa880
show the number of facts for each prover in "verbose" mode
blanchet
parents:
39108
diff
changeset
|
338 |
val num_axioms = Int.min (length axioms, max_relevant) |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
339 |
val desc = prover_description ctxt params atp_name num_axioms i n goal |
39318 | 340 |
fun go () = |
38982
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
341 |
let |
39453
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
342 |
fun really_go () = |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
343 |
atp_fun auto atp_name atp params (minimize_command atp_name) |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
344 |
atp_problem |
38985
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
345 |
|> (fn {outcome, message, ...} => |
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
346 |
(if is_some outcome then "none" else "some", message)) |
39453
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
347 |
val (outcome_code, message) = |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
348 |
if debug then |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
349 |
really_go () |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
350 |
else |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
351 |
(really_go () |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
352 |
handle ERROR message => ("unknown", "Error: " ^ message ^ "\n") |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
353 |
| exn => ("unknown", "Internal error:\n" ^ |
1740a2d6bef9
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
blanchet
parents:
39452
diff
changeset
|
354 |
ML_Compiler.exn_message exn ^ "\n")) |
39318 | 355 |
val _ = |
356 |
if expect = "" orelse outcome_code = expect then |
|
357 |
() |
|
358 |
else if blocking then |
|
359 |
error ("Unexpected outcome: " ^ quote outcome_code ^ ".") |
|
360 |
else |
|
361 |
warning ("Unexpected outcome: " ^ quote outcome_code ^ "."); |
|
362 |
in (outcome_code = "some", message) end |
|
363 |
in |
|
364 |
if auto then |
|
365 |
let val (success, message) = TimeLimit.timeLimit timeout go () in |
|
366 |
(success, state |> success ? Proof.goal_message (fn () => |
|
367 |
Pretty.chunks [Pretty.str "", Pretty.mark Markup.hilite |
|
39327 | 368 |
(Pretty.str message)])) |
38982
820b8221ed48
added "blocking" option to Sledgehammer to run in synchronous mode;
blanchet
parents:
38893
diff
changeset
|
369 |
end |
39318 | 370 |
else if blocking then |
371 |
let val (success, message) = TimeLimit.timeLimit timeout go () in |
|
39370
f8292d3020db
use same hack as in "Async_Manager" to work around Proof General bug
blanchet
parents:
39366
diff
changeset
|
372 |
List.app priority |
f8292d3020db
use same hack as in "Async_Manager" to work around Proof General bug
blanchet
parents:
39366
diff
changeset
|
373 |
(Async_Manager.break_into_chunks [desc ^ "\n" ^ message]); |
f8292d3020db
use same hack as in "Async_Manager" to work around Proof General bug
blanchet
parents:
39366
diff
changeset
|
374 |
(success, state) |
39318 | 375 |
end |
376 |
else |
|
377 |
(Async_Manager.launch das_Tool birth_time death_time desc (snd o go); |
|
378 |
(false, state)) |
|
37584 | 379 |
end |
28582 | 380 |
|
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
381 |
(* FIXME: dummy *) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
382 |
fun run_smt_solver ctxt remote timeout axioms = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
383 |
("", axioms |> take 5 |> map fst) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
384 |
|
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
385 |
(* FIXME: dummy *) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
386 |
fun is_smt_solver_installed () = true |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
387 |
|
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
388 |
fun run_smt_solver_somehow ctxt (params as {timeout, ...}) i n goal axioms |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
389 |
(remote, name) = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
390 |
let |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
391 |
val desc = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
392 |
prover_description ctxt params name (length axioms) i n goal |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
393 |
val (failure, used_thm_names) = run_smt_solver ctxt remote timeout axioms |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
394 |
val success = (failure = "") |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
395 |
val message = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
396 |
das_Tool ^ ": " ^ desc ^ "\n" ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
397 |
(if success then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
398 |
sendback_line (proof_banner false) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
399 |
(apply_on_subgoal i n ^ |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
400 |
command_call "smt" (map fst used_thm_names)) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
401 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
402 |
"Error: " ^ failure) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
403 |
in priority message; success end |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
404 |
|
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
405 |
val smt_default_max_relevant = 300 (* FUDGE *) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
406 |
val auto_max_relevant_divisor = 2 (* FUDGE *) |
39318 | 407 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
408 |
fun run_sledgehammer (params as {blocking, provers, full_types, |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
409 |
relevance_thresholds, max_relevant, timeout, |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
410 |
...}) |
39366
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
411 |
auto i (relevance_override as {only, ...}) minimize_command |
f58fbb959826
handle relevance filter corner cases more gracefully;
blanchet
parents:
39364
diff
changeset
|
412 |
state = |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
413 |
if null provers then |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
414 |
error "No prover is set." |
39318 | 415 |
else case subgoal_count state of |
416 |
0 => (priority "No subgoal!"; (false, state)) |
|
417 |
| n => |
|
418 |
let |
|
39364 | 419 |
val _ = Proof.assert_backward state |
39318 | 420 |
val thy = Proof.theory_of state |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
421 |
val {context = ctxt, facts = chained_ths, goal} = Proof.goal state |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
422 |
val (_, hyp_ts, concl_t) = strip_subgoal goal i |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39494
diff
changeset
|
423 |
val _ = () |> not blocking ? kill_provers |
39318 | 424 |
val _ = if auto then () else priority "Sledgehammering..." |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
425 |
val (smts, atps) = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
426 |
provers |> List.partition (member (op =) smt_names) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
427 |
|>> (take 1 #> map (`(String.isPrefix remote_prefix))) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
428 |
||> map (`(get_atp thy)) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
429 |
fun run_atps (res as (success, state)) = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
430 |
if success orelse null atps then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
431 |
res |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
432 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
433 |
let |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
434 |
val max_max_relevant = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
435 |
case max_relevant of |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
436 |
SOME n => n |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
437 |
| NONE => |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
438 |
0 |> fold (Integer.max o #default_max_relevant o fst) atps |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
439 |
|> auto ? (fn n => n div auto_max_relevant_divisor) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
440 |
val axioms = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
441 |
relevant_facts ctxt full_types relevance_thresholds |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
442 |
max_max_relevant relevance_override chained_ths |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
443 |
hyp_ts concl_t |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
444 |
val atp_problem = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
445 |
{state = state, goal = goal, subgoal = i, |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
446 |
axioms = map (prepare_axiom ctxt) axioms, only = only} |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
447 |
val run_atp_somehow = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
448 |
run_atp_somehow params auto i n minimize_command atp_problem |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
449 |
in |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
450 |
if auto then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
451 |
fold (fn atp => fn (true, state) => (true, state) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
452 |
| (false, _) => run_atp_somehow atp) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
453 |
atps (false, state) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
454 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
455 |
atps |> (if blocking then Par_List.map else map) run_atp_somehow |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
456 |
|> exists fst |> rpair state |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
457 |
end |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
458 |
fun run_smt_solvers (res as (success, state)) = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
459 |
if success orelse null smts then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
460 |
res |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
461 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
462 |
let |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
463 |
val max_relevant = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
464 |
max_relevant |> the_default smt_default_max_relevant |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
465 |
val axioms = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
466 |
relevant_facts ctxt full_types relevance_thresholds |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
467 |
max_relevant relevance_override chained_ths |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
468 |
hyp_ts concl_t |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
469 |
in |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
470 |
smts |> map (run_smt_solver_somehow ctxt params i n goal axioms) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
471 |
|> exists I |> rpair state |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
472 |
end |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
473 |
fun run_atps_and_smt_solvers () = |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
474 |
[run_atps, run_smt_solvers] |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
475 |
|> Par_List.map (fn f => f (false, state) |> K ()) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
476 |
in |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
477 |
if blocking then |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
478 |
(false, state) |> run_atps |> not auto ? run_smt_solvers |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
479 |
else |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
480 |
Future.fork (tap run_atps_and_smt_solvers) |> K (false, state) |
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
481 |
end |
38044 | 482 |
|
38023 | 483 |
val setup = |
484 |
dest_dir_setup |
|
485 |
#> problem_prefix_setup |
|
39003
c2aebd79981f
run relevance filter in a thread, to avoid blocking
blanchet
parents:
39000
diff
changeset
|
486 |
#> measure_run_time_setup |
38023 | 487 |
|
28582 | 488 |
end; |