author | blanchet |
Tue, 24 Aug 2010 21:40:03 +0200 | |
changeset 38737 | bdcb23701448 |
parent 38691 | fe5929dacd43 |
child 38740 | e2d58749194b |
permissions | -rw-r--r-- |
38047 | 1 |
(* Title: HOL/Tools/ATP/atp_systems.ML |
28592 | 2 |
Author: Fabian Immler, TU Muenchen |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
3 |
Author: Jasmin Blanchette, TU Muenchen |
28592 | 4 |
|
36376 | 5 |
Setup for supported ATPs. |
28592 | 6 |
*) |
7 |
||
36376 | 8 |
signature ATP_SYSTEMS = |
28592 | 9 |
sig |
38023 | 10 |
datatype failure = |
38519 | 11 |
Unprovable | IncompleteUnprovable | CantConnect | TimedOut | |
12 |
OutOfResources | SpassTooOld | VampireTooOld | NoPerl | NoLibwwwPerl | |
|
13 |
MalformedInput | MalformedOutput | UnknownError |
|
38023 | 14 |
|
15 |
type prover_config = |
|
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:
38090
diff
changeset
|
16 |
{exec: string * string, |
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:
38090
diff
changeset
|
17 |
required_execs: (string * string) list, |
38023 | 18 |
arguments: bool -> Time.time -> string, |
38645 | 19 |
has_incomplete_mode: bool, |
38023 | 20 |
proof_delims: (string * string) list, |
21 |
known_failures: (failure * string) list, |
|
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
22 |
default_max_relevant_per_iter: int, |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
23 |
default_theory_relevant: bool, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
24 |
explicit_forall: bool, |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
25 |
use_conjecture_for_hypotheses: bool} |
38023 | 26 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
27 |
val string_for_failure : failure -> string |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
28 |
val known_failure_in_output : |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
29 |
string -> (failure * string) list -> failure option |
38023 | 30 |
val add_prover: string * prover_config -> theory -> theory |
31 |
val get_prover: theory -> string -> prover_config |
|
32 |
val available_atps: theory -> unit |
|
35867 | 33 |
val refresh_systems_on_tptp : unit -> unit |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
34 |
val default_atps_param_value : unit -> string |
35867 | 35 |
val setup : theory -> theory |
28592 | 36 |
end; |
37 |
||
36376 | 38 |
structure ATP_Systems : ATP_SYSTEMS = |
28592 | 39 |
struct |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
40 |
|
38023 | 41 |
(* prover configuration *) |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
42 |
|
38023 | 43 |
datatype failure = |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
44 |
Unprovable | IncompleteUnprovable | CantConnect | TimedOut | OutOfResources | |
38519 | 45 |
SpassTooOld | VampireTooOld | NoPerl | NoLibwwwPerl | MalformedInput | |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
46 |
MalformedOutput | UnknownError |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
47 |
|
32941
72d48e333b77
eliminated extraneous wrapping of public records;
wenzelm
parents:
32936
diff
changeset
|
48 |
type prover_config = |
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:
38090
diff
changeset
|
49 |
{exec: string * string, |
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:
38090
diff
changeset
|
50 |
required_execs: (string * string) list, |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
51 |
arguments: bool -> Time.time -> string, |
38645 | 52 |
has_incomplete_mode: bool, |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
53 |
proof_delims: (string * string) list, |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
54 |
known_failures: (failure * string) list, |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
55 |
default_max_relevant_per_iter: int, |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
56 |
default_theory_relevant: bool, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
57 |
explicit_forall: bool, |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
58 |
use_conjecture_for_hypotheses: bool} |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
59 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
60 |
val missing_message_tail = |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
61 |
" appears to be missing. You will need to install it if you want to run \ |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
62 |
\ATPs remotely." |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
63 |
|
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
64 |
fun string_for_failure Unprovable = "The ATP problem is unprovable." |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
65 |
| string_for_failure IncompleteUnprovable = |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
66 |
"The ATP cannot prove the problem." |
38094 | 67 |
| string_for_failure CantConnect = "Can't connect to remote server." |
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
68 |
| string_for_failure TimedOut = "Timed out." |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
69 |
| string_for_failure OutOfResources = "The ATP ran out of resources." |
38519 | 70 |
| string_for_failure SpassTooOld = |
38096 | 71 |
"Isabelle requires a more recent version of SPASS with support for the \ |
72 |
\TPTP syntax. To install it, download and extract the package \ |
|
73 |
\\"http://isabelle.in.tum.de/dist/contrib/spass-3.7.tar.gz\" and add the \ |
|
74 |
\\"spass-3.7\" directory's absolute path to " ^ |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
75 |
quote (Path.implode (Path.expand (Path.appends |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
76 |
(Path.variable "ISABELLE_HOME_USER" :: |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
77 |
map Path.basic ["etc", "components"])))) ^ |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
78 |
" on a line of its own." |
38519 | 79 |
| string_for_failure VampireTooOld = |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
80 |
"Isabelle requires a more recent version of Vampire. To install it, follow \ |
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
81 |
\the instructions from the Sledgehammer manual (\"isabelle doc\ |
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
82 |
\ sledgehammer\")." |
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
83 |
| string_for_failure NoPerl = "Perl" ^ missing_message_tail |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
84 |
| string_for_failure NoLibwwwPerl = |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
85 |
"The Perl module \"libwww-perl\"" ^ missing_message_tail |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
86 |
| string_for_failure MalformedInput = |
38096 | 87 |
"The ATP problem is malformed. Please report this to the Isabelle \ |
88 |
\developers." |
|
89 |
| string_for_failure MalformedOutput = "The ATP output is malformed." |
|
90 |
| string_for_failure UnknownError = "An unknown ATP error occurred." |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
91 |
|
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
92 |
fun known_failure_in_output output = |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
93 |
find_first (fn (_, pattern) => String.isSubstring pattern output) |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
94 |
#> Option.map fst |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
95 |
|
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
96 |
val known_perl_failures = |
38094 | 97 |
[(CantConnect, "HTTP error"), |
98 |
(NoPerl, "env: perl"), |
|
38065 | 99 |
(NoLibwwwPerl, "Can't locate HTTP")] |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
100 |
|
38023 | 101 |
(* named provers *) |
38001
a9b47b85ca24
reintroduced more preprocessing steps to Sledgehammer, adapted to the new FOF setting
blanchet
parents:
38000
diff
changeset
|
102 |
|
38023 | 103 |
structure Data = Theory_Data |
104 |
( |
|
105 |
type T = (prover_config * stamp) Symtab.table |
|
106 |
val empty = Symtab.empty |
|
107 |
val extend = I |
|
108 |
fun merge data : T = Symtab.merge (eq_snd op =) data |
|
109 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name ^ ".") |
|
110 |
) |
|
38017
3ad3e3ca2451
move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
blanchet
parents:
38015
diff
changeset
|
111 |
|
38023 | 112 |
fun add_prover (name, config) thy = |
113 |
Data.map (Symtab.update_new (name, (config, stamp ()))) thy |
|
114 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name ^ ".") |
|
38017
3ad3e3ca2451
move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
blanchet
parents:
38015
diff
changeset
|
115 |
|
38023 | 116 |
fun get_prover thy name = |
117 |
the (Symtab.lookup (Data.get thy) name) |> fst |
|
118 |
handle Option.Option => error ("Unknown ATP: " ^ name ^ ".") |
|
37962
d7dbe01f48d7
keep track of clause numbers for SPASS now that we generate FOF rather than CNF problems;
blanchet
parents:
37926
diff
changeset
|
119 |
|
38023 | 120 |
fun available_atps thy = |
121 |
priority ("Available ATPs: " ^ |
|
122 |
commas (sort_strings (Symtab.keys (Data.get thy))) ^ ".") |
|
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
123 |
|
38023 | 124 |
fun available_atps thy = |
125 |
priority ("Available ATPs: " ^ |
|
126 |
commas (sort_strings (Symtab.keys (Data.get thy))) ^ ".") |
|
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
127 |
|
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
128 |
fun to_secs bonus time = (Time.toMilliseconds time + bonus + 999) div 1000 |
36142
f5e15e9aae10
make Sledgehammer "minimize" output less confusing + round up (not down) time limits to nearest second
blanchet
parents:
36064
diff
changeset
|
129 |
|
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
130 |
(* E prover *) |
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
131 |
|
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
132 |
(* Give older versions of E an extra second, because the "eproof" script wrongly |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
133 |
subtracted an entire second to account for the overhead of the script |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
134 |
itself, which is in fact much lower. *) |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
135 |
fun e_bonus () = |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
136 |
case getenv "E_VERSION" of |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
137 |
"" => 1000 |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
138 |
| version => |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
139 |
if exists (fn s => String.isPrefix s version) ["0.9", "1.0"] then 1000 |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
140 |
else 0 |
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
141 |
|
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
142 |
val tstp_proof_delims = |
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
143 |
("# SZS output start CNFRefutation.", "# SZS output end CNFRefutation") |
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
144 |
|
35969 | 145 |
val e_config : prover_config = |
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:
38090
diff
changeset
|
146 |
{exec = ("E_HOME", "eproof"), |
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:
38090
diff
changeset
|
147 |
required_execs = [], |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
148 |
arguments = fn _ => fn timeout => |
38691 | 149 |
"--tstp-in --tstp-out -l5 -xAutoDev -tAutoDev --silent \ |
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
150 |
\--cpu-limit=" ^ string_of_int (to_secs (e_bonus ()) timeout), |
38645 | 151 |
has_incomplete_mode = false, |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
152 |
proof_delims = [tstp_proof_delims], |
36265
41c9e755e552
distinguish between the different ATP errors in the user interface;
blanchet
parents:
36264
diff
changeset
|
153 |
known_failures = |
37995
06f02b15ef8a
generate full first-order formulas (FOF) in Sledgehammer
blanchet
parents:
37994
diff
changeset
|
154 |
[(Unprovable, "SZS status: CounterSatisfiable"), |
06f02b15ef8a
generate full first-order formulas (FOF) in Sledgehammer
blanchet
parents:
37994
diff
changeset
|
155 |
(Unprovable, "SZS status CounterSatisfiable"), |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
156 |
(TimedOut, "Failure: Resource limit exceeded (time)"), |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
157 |
(TimedOut, "time limit exceeded"), |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
158 |
(OutOfResources, |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
159 |
"# Cannot determine problem status within resource limit"), |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
160 |
(OutOfResources, "SZS status: ResourceOut"), |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
161 |
(OutOfResources, "SZS status ResourceOut")], |
38685
87a1e97a3ef3
adjust fudge factors in the light of experiments
blanchet
parents:
38680
diff
changeset
|
162 |
default_max_relevant_per_iter = 80 (* FUDGE *), |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
163 |
default_theory_relevant = false, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
164 |
explicit_forall = false, |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
165 |
use_conjecture_for_hypotheses = true} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
166 |
|
38023 | 167 |
val e = ("e", e_config) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
168 |
|
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
169 |
|
36219
16670b4f0baa
set SPASS option on the command-line, so that it doesn't vanish when moving to TPTP format
blanchet
parents:
36190
diff
changeset
|
170 |
(* The "-VarWeight=3" option helps the higher-order problems, probably by |
16670b4f0baa
set SPASS option on the command-line, so that it doesn't vanish when moving to TPTP format
blanchet
parents:
36190
diff
changeset
|
171 |
counteracting the presence of "hAPP". *) |
37498
b426cbdb5a23
removed Sledgehammer's support for the DFG syntax;
blanchet
parents:
37480
diff
changeset
|
172 |
val spass_config : prover_config = |
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:
38090
diff
changeset
|
173 |
{exec = ("ISABELLE_ATP", "scripts/spass"), |
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:
38090
diff
changeset
|
174 |
required_execs = [("SPASS_HOME", "SPASS")], |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
175 |
arguments = fn complete => fn timeout => |
37962
d7dbe01f48d7
keep track of clause numbers for SPASS now that we generate FOF rather than CNF problems;
blanchet
parents:
37926
diff
changeset
|
176 |
("-Auto -PGiven=0 -PProblem=0 -Splits=0 -FullRed=0 -DocProof \ |
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
177 |
\-VarWeight=3 -TimeLimit=" ^ string_of_int (to_secs 0 timeout)) |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
178 |
|> not complete ? prefix "-SOS=1 ", |
38645 | 179 |
has_incomplete_mode = true, |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
180 |
proof_delims = [("Here is a proof", "Formulae used in the proof")], |
36289
f75b6a3e1450
set "atps" reference's default value to "(remote_)e (remote_)spass (remote_)vampire", based on what is installed
blanchet
parents:
36287
diff
changeset
|
181 |
known_failures = |
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
182 |
known_perl_failures @ |
37413 | 183 |
[(IncompleteUnprovable, "SPASS beiseite: Completion found"), |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
184 |
(TimedOut, "SPASS beiseite: Ran out of time"), |
36965 | 185 |
(OutOfResources, "SPASS beiseite: Maximal number of loops exceeded"), |
37413 | 186 |
(MalformedInput, "Undefined symbol"), |
37414
d0cea0796295
expect SPASS 3.7, and give a friendly warning if an older version is used
blanchet
parents:
37413
diff
changeset
|
187 |
(MalformedInput, "Free Variable"), |
38519 | 188 |
(SpassTooOld, "tptp2dfg")], |
38685
87a1e97a3ef3
adjust fudge factors in the light of experiments
blanchet
parents:
38680
diff
changeset
|
189 |
default_max_relevant_per_iter = 40 (* FUDGE *), |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
190 |
default_theory_relevant = true, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
191 |
explicit_forall = true, |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
192 |
use_conjecture_for_hypotheses = true} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
193 |
|
38023 | 194 |
val spass = ("spass", spass_config) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
195 |
|
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
196 |
|
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
197 |
(* Vampire *) |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
198 |
|
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
199 |
val vampire_config : prover_config = |
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:
38090
diff
changeset
|
200 |
{exec = ("VAMPIRE_HOME", "vampire"), |
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:
38090
diff
changeset
|
201 |
required_execs = [], |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
202 |
arguments = fn _ => fn timeout => |
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
203 |
"--mode casc -t " ^ string_of_int (to_secs 0 timeout) ^ |
38588 | 204 |
" --thanks Andrei --input_file", |
38645 | 205 |
has_incomplete_mode = false, |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
206 |
proof_delims = |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
207 |
[("=========== Refutation ==========", |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
208 |
"======= End of refutation ======="), |
38033 | 209 |
("% SZS output start Refutation", "% SZS output end Refutation"), |
210 |
("% SZS output start Proof", "% SZS output end Proof")], |
|
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
211 |
known_failures = |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
212 |
[(Unprovable, "UNPROVABLE"), |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
213 |
(IncompleteUnprovable, "CANNOT PROVE"), |
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:
38090
diff
changeset
|
214 |
(TimedOut, "SZS status Timeout"), |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
215 |
(Unprovable, "Satisfiability detected"), |
38647
5500241da479
play with fudge factor + parse one more Vampire error
blanchet
parents:
38646
diff
changeset
|
216 |
(Unprovable, "Termination reason: Satisfiable"), |
38519 | 217 |
(VampireTooOld, "not a valid option")], |
38646 | 218 |
default_max_relevant_per_iter = 45 (* FUDGE *), |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
219 |
default_theory_relevant = false, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
220 |
explicit_forall = false, |
38680 | 221 |
use_conjecture_for_hypotheses = true} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
222 |
|
38023 | 223 |
val vampire = ("vampire", vampire_config) |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
224 |
|
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
225 |
|
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
226 |
(* Remote prover invocation via SystemOnTPTP *) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
227 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
228 |
val systems = Synchronized.var "atp_systems" ([] : string list) |
31835 | 229 |
|
230 |
fun get_systems () = |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
231 |
case bash_output "\"$ISABELLE_ATP/scripts/remote_atp\" -w 2>&1" of |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
232 |
(answer, 0) => split_lines answer |
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
233 |
| (answer, _) => |
38065 | 234 |
error (case known_failure_in_output answer known_perl_failures of |
235 |
SOME failure => string_for_failure failure |
|
236 |
| NONE => perhaps (try (unsuffix "\n")) answer ^ ".") |
|
31835 | 237 |
|
35867 | 238 |
fun refresh_systems_on_tptp () = |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
239 |
Synchronized.change systems (fn _ => get_systems ()) |
31835 | 240 |
|
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
241 |
fun find_system name [] systems = find_first (String.isPrefix name) systems |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
242 |
| find_system name (version :: versions) systems = |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
243 |
case find_first (String.isPrefix (name ^ "---" ^ version)) systems of |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
244 |
NONE => find_system name versions systems |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
245 |
| res => res |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
246 |
|
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
247 |
fun get_system name versions = |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
248 |
Synchronized.change_result systems |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
249 |
(fn systems => (if null systems then get_systems () else systems) |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
250 |
|> `(find_system name versions)) |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
251 |
|
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
252 |
fun the_system name versions = |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
253 |
case get_system name versions of |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
254 |
NONE => error ("System " ^ quote name ^ " not available at SystemOnTPTP.") |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
255 |
| SOME sys => sys |
31835 | 256 |
|
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
257 |
fun remote_config system_name system_versions proof_delims known_failures |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
258 |
default_max_relevant_per_iter default_theory_relevant |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
259 |
use_conjecture_for_hypotheses = |
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:
38090
diff
changeset
|
260 |
{exec = ("ISABELLE_ATP", "scripts/remote_atp"), |
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:
38090
diff
changeset
|
261 |
required_execs = [], |
37514
b147d01b8ebc
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
blanchet
parents:
37509
diff
changeset
|
262 |
arguments = fn _ => fn timeout => |
38737
bdcb23701448
better workaround for E's off-by-one-second issue
blanchet
parents:
38691
diff
changeset
|
263 |
" -t " ^ string_of_int (to_secs 0 timeout) ^ " -s " ^ |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
264 |
the_system system_name system_versions, |
38645 | 265 |
has_incomplete_mode = false, |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
266 |
proof_delims = insert (op =) tstp_proof_delims proof_delims, |
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
267 |
known_failures = |
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
268 |
known_failures @ known_perl_failures @ |
38094 | 269 |
[(TimedOut, "says Timeout")], |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
270 |
default_max_relevant_per_iter = default_max_relevant_per_iter, |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
271 |
default_theory_relevant = default_theory_relevant, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
272 |
explicit_forall = true, |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
273 |
use_conjecture_for_hypotheses = use_conjecture_for_hypotheses} |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
274 |
|
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
275 |
fun remotify_config system_name system_versions |
38598 | 276 |
({proof_delims, known_failures, default_max_relevant_per_iter, |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
277 |
default_theory_relevant, use_conjecture_for_hypotheses, ...} |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
278 |
: prover_config) : prover_config = |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
279 |
remote_config system_name system_versions proof_delims known_failures |
38598 | 280 |
default_max_relevant_per_iter default_theory_relevant |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
281 |
use_conjecture_for_hypotheses |
38023 | 282 |
|
38598 | 283 |
val remotify_name = prefix "remote_" |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
284 |
fun remote_prover name system_name system_versions proof_delims known_failures |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
285 |
default_max_relevant_per_iter default_theory_relevant |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
286 |
use_conjecture_for_hypotheses = |
38598 | 287 |
(remotify_name name, |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
288 |
remote_config system_name system_versions proof_delims known_failures |
38631
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
289 |
default_max_relevant_per_iter default_theory_relevant |
979a0b37f981
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
blanchet
parents:
38603
diff
changeset
|
290 |
use_conjecture_for_hypotheses) |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
291 |
fun remotify_prover (name, config) system_name system_versions = |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
292 |
(remotify_name name, remotify_config system_name system_versions config) |
28592 | 293 |
|
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
294 |
val remote_e = remotify_prover e "EP" ["1.0", "1.1", "1.2"] |
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
295 |
val remote_vampire = remotify_prover vampire "Vampire" ["9.9", "0.6", "1.0"] |
38603
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
296 |
val remote_sine_e = |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
297 |
remote_prover "sine_e" "SInE" [] [] |
38646 | 298 |
[(Unprovable, "says Unknown")] 150 (* FUDGE *) false true |
38598 | 299 |
val remote_snark = |
38690
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
300 |
remote_prover "snark" "SNARK---" [] [("refutation.", "end_refutation.")] [] |
38646 | 301 |
50 (* FUDGE *) false true |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
302 |
|
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
303 |
(* Setup *) |
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
304 |
|
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:
38090
diff
changeset
|
305 |
fun is_installed ({exec, required_execs, ...} : prover_config) = |
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:
38090
diff
changeset
|
306 |
forall (curry (op <>) "" o getenv o fst) (exec :: required_execs) |
38041
3b80d6082131
remove "remote_spass" because there's no way to find out which clauses come from which facts + rename scripts
blanchet
parents:
38033
diff
changeset
|
307 |
fun maybe_remote (name, config) = |
38598 | 308 |
name |> not (is_installed config) ? remotify_name |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
309 |
|
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
310 |
fun default_atps_param_value () = |
38041
3b80d6082131
remove "remote_spass" because there's no way to find out which clauses come from which facts + rename scripts
blanchet
parents:
38033
diff
changeset
|
311 |
space_implode " " ([maybe_remote e] @ |
3b80d6082131
remove "remote_spass" because there's no way to find out which clauses come from which facts + rename scripts
blanchet
parents:
38033
diff
changeset
|
312 |
(if is_installed (snd spass) then [fst spass] else []) @ |
38603
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
313 |
[if forall (is_installed o snd) [e, spass] then |
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
314 |
remotify_name (fst vampire) |
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
315 |
else |
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
316 |
maybe_remote vampire, |
a57d04dd1b25
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
blanchet
parents:
38598
diff
changeset
|
317 |
fst remote_sine_e]) |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
318 |
|
38598 | 319 |
val provers = [e, spass, vampire, remote_e, remote_vampire, remote_sine_e, |
320 |
remote_snark] |
|
38023 | 321 |
val setup = fold add_prover provers |
35867 | 322 |
|
28592 | 323 |
end; |