author | blanchet |
Mon, 21 May 2012 11:31:52 +0200 | |
changeset 47948 | 0524790d2112 |
parent 47931 | 406d1df3787e |
child 47949 | fafbb2607366 |
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 |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
10 |
type term_order = ATP_Problem.term_order |
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
11 |
type atp_format = ATP_Problem.atp_format |
42577
78414ec6fa4e
made the format (TFF or FOF) of the TPTP problem a global argument of the problem again and have the ATPs report which formats they support
blanchet
parents:
42571
diff
changeset
|
12 |
type formula_kind = ATP_Problem.formula_kind |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
13 |
type failure = ATP_Proof.failure |
38023 | 14 |
|
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
15 |
type slice_spec = int * atp_format * string * string * bool |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
16 |
type atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
17 |
{exec : string list * string, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
18 |
required_vars : string list list, |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
19 |
arguments : |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
20 |
Proof.context -> bool -> string -> Time.time |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
21 |
-> term_order * (unit -> (string * int) list) |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
22 |
* (unit -> (string * real) list) -> string, |
42578
1eaf4d437d4c
define type system in ATP module so that ATPs can suggest a type system
blanchet
parents:
42577
diff
changeset
|
23 |
proof_delims : (string * string) list, |
1eaf4d437d4c
define type system in ATP module so that ATPs can suggest a type system
blanchet
parents:
42577
diff
changeset
|
24 |
known_failures : (failure * string) list, |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
25 |
prem_kind : formula_kind, |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
26 |
best_slices : |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
27 |
Proof.context -> (real * (bool * (slice_spec * string))) list} |
38023 | 28 |
|
44099 | 29 |
val force_sos : bool Config.T |
47032 | 30 |
val term_order : string Config.T |
43566
a818d5a34cca
filter out some tautologies using an ATP, especially for those theories that are known for producing such things
blanchet
parents:
43529
diff
changeset
|
31 |
val e_smartN : string |
a818d5a34cca
filter out some tautologies using an ATP, especially for those theories that are known for producing such things
blanchet
parents:
43529
diff
changeset
|
32 |
val e_autoN : string |
a818d5a34cca
filter out some tautologies using an ATP, especially for those theories that are known for producing such things
blanchet
parents:
43529
diff
changeset
|
33 |
val e_fun_weightN : string |
a818d5a34cca
filter out some tautologies using an ATP, especially for those theories that are known for producing such things
blanchet
parents:
43529
diff
changeset
|
34 |
val e_sym_offset_weightN : string |
47032 | 35 |
val e_selection_heuristic : string Config.T |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
36 |
val e_default_fun_weight : real Config.T |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
37 |
val e_fun_weight_base : real Config.T |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
38 |
val e_fun_weight_span : real Config.T |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
39 |
val e_default_sym_offs_weight : real Config.T |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
40 |
val e_sym_offs_weight_base : real Config.T |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
41 |
val e_sym_offs_weight_span : real Config.T |
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
42 |
val alt_ergoN : string |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
43 |
val dummy_thfN : string |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
44 |
val eN : string |
44590 | 45 |
val e_sineN : string |
46 |
val e_tofofN : string |
|
45338 | 47 |
val iproverN : string |
48 |
val iprover_eqN : string |
|
44590 | 49 |
val leo2N : string |
50 |
val satallaxN : string |
|
51 |
val snarkN : string |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
52 |
val spassN : string |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
53 |
val spass_oldN : string |
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
54 |
val spass_newN : string |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
55 |
val vampireN : string |
42938 | 56 |
val waldmeisterN : string |
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
57 |
val z3_tptpN : string |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
58 |
val remote_prefix : string |
41738
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
59 |
val remote_atp : |
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
60 |
string -> string -> string list -> (string * string) list |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
61 |
-> (failure * string) list -> formula_kind |
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
62 |
-> (Proof.context -> slice_spec * string) -> string * (unit -> atp_config) |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
63 |
val add_atp : string * (unit -> atp_config) -> theory -> theory |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
64 |
val get_atp : theory -> string -> (unit -> atp_config) |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41725
diff
changeset
|
65 |
val supported_atps : theory -> string list |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
66 |
val is_atp_installed : theory -> string -> bool |
35867 | 67 |
val refresh_systems_on_tptp : unit -> unit |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
68 |
val effective_term_order : Proof.context -> string -> term_order |
35867 | 69 |
val setup : theory -> theory |
28592 | 70 |
end; |
71 |
||
36376 | 72 |
structure ATP_Systems : ATP_SYSTEMS = |
28592 | 73 |
struct |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
74 |
|
42577
78414ec6fa4e
made the format (TFF or FOF) of the TPTP problem a global argument of the problem again and have the ATPs report which formats they support
blanchet
parents:
42571
diff
changeset
|
75 |
open ATP_Problem |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
76 |
open ATP_Proof |
46320 | 77 |
open ATP_Problem_Generate |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
78 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
79 |
(* ATP configuration *) |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
80 |
|
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
81 |
type slice_spec = int * atp_format * string * string * bool |
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
82 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
83 |
type atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
84 |
{exec : string list * string, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
85 |
required_vars : string list list, |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
86 |
arguments : |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
87 |
Proof.context -> bool -> string -> Time.time |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
88 |
-> term_order * (unit -> (string * int) list) |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
89 |
* (unit -> (string * real) list) -> string, |
42578
1eaf4d437d4c
define type system in ATP module so that ATPs can suggest a type system
blanchet
parents:
42577
diff
changeset
|
90 |
proof_delims : (string * string) list, |
1eaf4d437d4c
define type system in ATP module so that ATPs can suggest a type system
blanchet
parents:
42577
diff
changeset
|
91 |
known_failures : (failure * string) list, |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
92 |
prem_kind : formula_kind, |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
93 |
best_slices : Proof.context -> (real * (bool * (slice_spec * string))) list} |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
94 |
|
42723 | 95 |
(* "best_slices" must be found empirically, taking a wholistic approach since |
46407
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
96 |
the ATPs are run in parallel. The "real" component gives the faction of the |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
97 |
time available given to the slice and should add up to 1.0. The first "bool" |
42723 | 98 |
component indicates whether the slice's strategy is complete; the "int", the |
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43567
diff
changeset
|
99 |
preferred number of facts to pass; the first "string", the preferred type |
45521 | 100 |
system (which should be sound or quasi-sound); the second "string", the |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
101 |
preferred lambda translation scheme; the second "bool", whether uncurried |
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
102 |
aliased should be generated; the third "string", extra information to |
45521 | 103 |
the prover (e.g., SOS or no SOS). |
42723 | 104 |
|
105 |
The last slice should be the most "normal" one, because it will get all the |
|
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43567
diff
changeset
|
106 |
time available if the other slices fail early and also because it is used if |
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43567
diff
changeset
|
107 |
slicing is disabled (e.g., by the minimizer). *) |
42710
84fcce345b5d
further improved type system setup based on Judgment Days
blanchet
parents:
42709
diff
changeset
|
108 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
109 |
val known_perl_failures = |
38094 | 110 |
[(CantConnect, "HTTP error"), |
111 |
(NoPerl, "env: perl"), |
|
38065 | 112 |
(NoLibwwwPerl, "Can't locate HTTP")] |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
113 |
|
45203 | 114 |
fun known_szs_failures wrap = |
115 |
[(Unprovable, wrap "CounterSatisfiable"), |
|
116 |
(Unprovable, wrap "Satisfiable"), |
|
117 |
(GaveUp, wrap "GaveUp"), |
|
118 |
(GaveUp, wrap "Unknown"), |
|
119 |
(GaveUp, wrap "Incomplete"), |
|
120 |
(ProofMissing, wrap "Theorem"), |
|
121 |
(ProofMissing, wrap "Unsatisfiable"), |
|
122 |
(TimedOut, wrap "Timeout"), |
|
123 |
(Inappropriate, wrap "Inappropriate"), |
|
124 |
(OutOfResources, wrap "ResourceOut"), |
|
125 |
(OutOfResources, wrap "MemoryOut"), |
|
126 |
(Interrupted, wrap "Forced"), |
|
127 |
(Interrupted, wrap "User")] |
|
128 |
||
129 |
val known_szs_status_failures = known_szs_failures (prefix "SZS status ") |
|
130 |
val known_says_failures = known_szs_failures (prefix " says ") |
|
131 |
||
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
132 |
(* named ATPs *) |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
133 |
|
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
134 |
val alt_ergoN = "alt_ergo" |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
135 |
val dummy_thfN = "dummy_thf" (* for experiments *) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
136 |
val eN = "e" |
44590 | 137 |
val e_sineN = "e_sine" |
138 |
val e_tofofN = "e_tofof" |
|
45338 | 139 |
val iproverN = "iprover" |
140 |
val iprover_eqN = "iprover_eq" |
|
44099 | 141 |
val leo2N = "leo2" |
142 |
val satallaxN = "satallax" |
|
44590 | 143 |
val snarkN = "snark" |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
144 |
val spassN = "spass" |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
145 |
val spass_oldN = "spass_old" (* for experiments *) |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
146 |
val spass_newN = "spass_new" (* for experiments *) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
147 |
val vampireN = "vampire" |
44590 | 148 |
val waldmeisterN = "waldmeister" |
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
149 |
val z3_tptpN = "z3_tptp" |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
150 |
val remote_prefix = "remote_" |
38001
a9b47b85ca24
reintroduced more preprocessing steps to Sledgehammer, adapted to the new FOF setting
blanchet
parents:
38000
diff
changeset
|
151 |
|
38023 | 152 |
structure Data = Theory_Data |
153 |
( |
|
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
154 |
type T = ((unit -> atp_config) * stamp) Symtab.table |
38023 | 155 |
val empty = Symtab.empty |
156 |
val extend = I |
|
46407
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
157 |
fun merge data : T = |
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
158 |
Symtab.merge (eq_snd (op =)) data |
38023 | 159 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name ^ ".") |
160 |
) |
|
38017
3ad3e3ca2451
move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
blanchet
parents:
38015
diff
changeset
|
161 |
|
43981
404ae49ce29f
give E at least two seconds -- anything else risks causing too early timeouts in the minimizer, because of too conservative time computations in E and eproof scripts
blanchet
parents:
43850
diff
changeset
|
162 |
fun to_secs min time = Int.max (min, (Time.toMilliseconds time + 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
|
163 |
|
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
164 |
val sosN = "sos" |
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
165 |
val no_sosN = "no_sos" |
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
166 |
|
44099 | 167 |
val force_sos = Attrib.setup_config_bool @{binding atp_force_sos} (K false) |
168 |
||
47032 | 169 |
val smartN = "smart" |
47073
c73f7b0c7ebc
generate weights and precedences for predicates as well
blanchet
parents:
47055
diff
changeset
|
170 |
(* val kboN = "kbo" *) |
47032 | 171 |
val lpoN = "lpo" |
47034
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
172 |
val xweightsN = "_weights" |
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
173 |
val xprecN = "_prec" |
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
174 |
val xsimpN = "_simp" (* SPASS-specific *) |
47032 | 175 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
176 |
(* Possible values for "atp_term_order": |
47049 | 177 |
"smart", "(kbo|lpo)(_weights)?(_prec|_simp)?" *) |
47032 | 178 |
val term_order = |
179 |
Attrib.setup_config_string @{binding atp_term_order} (K smartN) |
|
180 |
||
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
181 |
(* Alt-Ergo *) |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
182 |
|
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
183 |
val alt_ergo_tff1 = TFF (TPTP_Polymorphic, TPTP_Explicit) |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
184 |
|
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
185 |
val alt_ergo_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
186 |
{exec = (["WHY3_HOME"], "why3"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
187 |
required_vars = [], |
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
188 |
arguments = |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
189 |
fn _ => fn _ => fn _ => fn timeout => fn _ => |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
190 |
"--format tff1 --prover alt-ergo --timelimit " ^ |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
191 |
string_of_int (to_secs 1 timeout), |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
192 |
proof_delims = [], |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
193 |
known_failures = |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
194 |
[(ProofMissing, ": Valid"), |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
195 |
(TimedOut, ": Timeout"), |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
196 |
(GaveUp, ": Unknown")], |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
197 |
prem_kind = Hypothesis, |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
198 |
best_slices = fn _ => |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
199 |
(* FUDGE *) |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
200 |
[(1.0, (false, ((100, alt_ergo_tff1, "poly_native", liftingN, false), "")))]} |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
201 |
|
47646 | 202 |
val alt_ergo = (alt_ergoN, fn () => alt_ergo_config) |
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
203 |
|
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
204 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
205 |
(* E *) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
206 |
|
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
207 |
fun is_new_e_version () = (string_ord (getenv "E_VERSION", "1.2") = GREATER) |
44420 | 208 |
|
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
209 |
val tstp_proof_delims = |
42962
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
blanchet
parents:
42955
diff
changeset
|
210 |
[("# SZS output start CNFRefutation.", "# SZS output end CNFRefutation"), |
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
blanchet
parents:
42955
diff
changeset
|
211 |
("% SZS output start CNFRefutation", "% SZS output end CNFRefutation")] |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
212 |
|
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
213 |
val e_smartN = "smart" |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
214 |
val e_autoN = "auto" |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
215 |
val e_fun_weightN = "fun_weight" |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
216 |
val e_sym_offset_weightN = "sym_offset_weight" |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
217 |
|
47032 | 218 |
val e_selection_heuristic = |
219 |
Attrib.setup_config_string @{binding atp_e_selection_heuristic} (K e_smartN) |
|
41770 | 220 |
(* FUDGE *) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
221 |
val e_default_fun_weight = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
222 |
Attrib.setup_config_real @{binding atp_e_default_fun_weight} (K 20.0) |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
223 |
val e_fun_weight_base = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
224 |
Attrib.setup_config_real @{binding atp_e_fun_weight_base} (K 0.0) |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
225 |
val e_fun_weight_span = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
226 |
Attrib.setup_config_real @{binding atp_e_fun_weight_span} (K 40.0) |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
227 |
val e_default_sym_offs_weight = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
228 |
Attrib.setup_config_real @{binding atp_e_default_sym_offs_weight} (K 1.0) |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
229 |
val e_sym_offs_weight_base = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
230 |
Attrib.setup_config_real @{binding atp_e_sym_offs_weight_base} (K ~20.0) |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
231 |
val e_sym_offs_weight_span = |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
232 |
Attrib.setup_config_real @{binding atp_e_sym_offs_weight_span} (K 60.0) |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
233 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
234 |
fun e_selection_heuristic_case heuristic fw sow = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
235 |
if heuristic = e_fun_weightN then fw |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
236 |
else if heuristic = e_sym_offset_weightN then sow |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
237 |
else raise Fail ("unexpected " ^ quote heuristic) |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
238 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
239 |
fun scaled_e_selection_weight ctxt heuristic w = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
240 |
w * Config.get ctxt (e_selection_heuristic_case heuristic |
47029 | 241 |
e_fun_weight_span e_sym_offs_weight_span) |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
242 |
+ Config.get ctxt (e_selection_heuristic_case heuristic |
47029 | 243 |
e_fun_weight_base e_sym_offs_weight_base) |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
244 |
|> Real.ceil |> signed_string_of_int |
41313
a96ac4d180b7
optionally supply constant weights to E -- turned off by default until properly parameterized
blanchet
parents:
41269
diff
changeset
|
245 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
246 |
fun e_selection_weight_arguments ctxt heuristic sel_weights = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
247 |
if heuristic = e_autoN then |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
248 |
"-xAuto" |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
249 |
else |
43622 | 250 |
(* supplied by Stephan Schulz *) |
41314
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
251 |
"--split-clauses=4 --split-reuse-defs --simul-paramod --forward-context-sr \ |
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
252 |
\--destructive-er-aggressive --destructive-er --presat-simplify \ |
47505
e33d957ae2bf
avoid option introduced in E 1.2 when invoking older versions of E
blanchet
parents:
47499
diff
changeset
|
253 |
\--prefer-initial-clauses -winvfreqrank -c1 -Ginvfreqconjmax -F1 \ |
e33d957ae2bf
avoid option introduced in E 1.2 when invoking older versions of E
blanchet
parents:
47499
diff
changeset
|
254 |
\--delete-bad-limit=150000000 -WSelectMaxLComplexAvoidPosPred -H'(4*" ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
255 |
e_selection_heuristic_case heuristic "FunWeight" "SymOffsetWeight" ^ |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
256 |
"(SimulateSOS, " ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
257 |
(e_selection_heuristic_case heuristic |
47029 | 258 |
e_default_fun_weight e_default_sym_offs_weight |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
259 |
|> Config.get ctxt |> Real.ceil |> signed_string_of_int) ^ |
41314
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
260 |
",20,1.5,1.5,1" ^ |
47030 | 261 |
(sel_weights () |
47029 | 262 |
|> map (fn (s, w) => "," ^ s ^ ":" ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
263 |
scaled_e_selection_weight ctxt heuristic w) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
264 |
|> implode) ^ |
41314
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
265 |
"),3*ConjectureGeneralSymbolWeight(PreferNonGoals,200,100,200,50,50,1,100,\ |
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
266 |
\1.5,1.5,1),1*Clauseweight(PreferProcessed,1,1,1),1*\ |
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
267 |
\FIFOWeight(PreferProcessed))'" |
41313
a96ac4d180b7
optionally supply constant weights to E -- turned off by default until properly parameterized
blanchet
parents:
41269
diff
changeset
|
268 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
269 |
val e_ord_weights = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
270 |
map (fn (s, w) => s ^ ":" ^ string_of_int w) #> space_implode "," |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
271 |
fun e_ord_precedence [_] = "" |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
272 |
| e_ord_precedence info = info |> map fst |> space_implode "<" |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
273 |
|
47039
1b36a05a070d
added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents:
47038
diff
changeset
|
274 |
fun e_term_order_info_arguments false false _ = "" |
1b36a05a070d
added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents:
47038
diff
changeset
|
275 |
| e_term_order_info_arguments gen_weights gen_prec ord_info = |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
276 |
let val ord_info = ord_info () in |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
277 |
(if gen_weights then "--order-weights='" ^ e_ord_weights ord_info ^ "' " |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
278 |
else "") ^ |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
279 |
(if gen_prec then "--precedence='" ^ e_ord_precedence ord_info ^ "' " |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
280 |
else "") |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
281 |
end |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
282 |
|
47032 | 283 |
fun effective_e_selection_heuristic ctxt = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
284 |
if is_new_e_version () then Config.get ctxt e_selection_heuristic else e_autoN |
42443
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42332
diff
changeset
|
285 |
|
47505
e33d957ae2bf
avoid option introduced in E 1.2 when invoking older versions of E
blanchet
parents:
47499
diff
changeset
|
286 |
fun e_kbo () = if is_new_e_version () then "KBO6" else "KBO" |
e33d957ae2bf
avoid option introduced in E 1.2 when invoking older versions of E
blanchet
parents:
47499
diff
changeset
|
287 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
288 |
val e_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
289 |
{exec = (["E_HOME"], "eproof"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
290 |
required_vars = [], |
43354
396aaa15dd8b
pass --trim option to "eproof" script to speed up proof reconstruction
blanchet
parents:
43288
diff
changeset
|
291 |
arguments = |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
292 |
fn ctxt => fn _ => fn heuristic => fn timeout => |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
293 |
fn ({is_lpo, gen_weights, gen_prec, ...}, ord_info, sel_weights) => |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
294 |
"--tstp-in --tstp-out --output-level=5 --silent " ^ |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
295 |
e_selection_weight_arguments ctxt heuristic sel_weights ^ " " ^ |
47039
1b36a05a070d
added "metis_advisory_simp" option to orient as many equations as possible in Metis the right way (cf. "More SPASS with Isabelle")
blanchet
parents:
47038
diff
changeset
|
296 |
e_term_order_info_arguments gen_weights gen_prec ord_info ^ " " ^ |
47505
e33d957ae2bf
avoid option introduced in E 1.2 when invoking older versions of E
blanchet
parents:
47499
diff
changeset
|
297 |
"--term-ordering=" ^ (if is_lpo then "LPO4" else e_kbo ()) ^ " " ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
298 |
"--cpu-limit=" ^ string_of_int (to_secs 2 timeout), |
42962
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
blanchet
parents:
42955
diff
changeset
|
299 |
proof_delims = tstp_proof_delims, |
36265
41c9e755e552
distinguish between the different ATP errors in the user interface;
blanchet
parents:
36264
diff
changeset
|
300 |
known_failures = |
45203 | 301 |
known_szs_status_failures @ |
302 |
[(TimedOut, "Failure: Resource limit exceeded (time)"), |
|
47736 | 303 |
(TimedOut, "time limit exceeded")], |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
304 |
prem_kind = Conjecture, |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
305 |
best_slices = fn ctxt => |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
306 |
let val heuristic = effective_e_selection_heuristic ctxt in |
43474
423cd1ecf714
optimized E's time slicing, based on latest exhaustive Judgment Day results
blanchet
parents:
43473
diff
changeset
|
307 |
(* FUDGE *) |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
308 |
if heuristic = e_smartN then |
46449 | 309 |
[(0.333, (true, ((500, FOF, "mono_tags??", combsN, false), e_fun_weightN))), |
310 |
(0.334, (true, ((50, FOF, "mono_guards??", combsN, false), e_fun_weightN))), |
|
311 |
(0.333, (true, ((1000, FOF, "mono_tags??", combsN, false), e_sym_offset_weightN)))] |
|
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
312 |
else |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
313 |
[(1.0, (true, ((500, FOF, "mono_tags??", combsN, false), heuristic)))] |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
314 |
end} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
315 |
|
47646 | 316 |
val e = (eN, fn () => e_config) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
317 |
|
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
318 |
|
44099 | 319 |
(* LEO-II *) |
320 |
||
44754 | 321 |
val leo2_thf0 = THF (TPTP_Monomorphic, TPTP_Explicit, THF_Without_Choice) |
322 |
||
44099 | 323 |
val leo2_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
324 |
{exec = (["LEO2_HOME"], "leo"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
325 |
required_vars = [], |
44099 | 326 |
arguments = |
47916 | 327 |
fn _ => fn _ => fn _ => fn timeout => fn _ => |
47914
94f37848b7c9
LEO-II's "--sos" option confusingly disables rather than enables SOS, and SOS seems to be ignored anyway; also, pass a number of facts that's more appropriate for each prover
blanchet
parents:
47912
diff
changeset
|
328 |
"--proofoutput 1 --timeout " ^ string_of_int (to_secs 1 timeout), |
44099 | 329 |
proof_delims = tstp_proof_delims, |
45207 | 330 |
known_failures = |
331 |
known_szs_status_failures @ |
|
46481 | 332 |
[(TimedOut, "CPU time limit exceeded, terminating"), |
333 |
(GaveUp, "No.of.Axioms")], |
|
47899 | 334 |
prem_kind = Hypothesis, |
47914
94f37848b7c9
LEO-II's "--sos" option confusingly disables rather than enables SOS, and SOS seems to be ignored anyway; also, pass a number of facts that's more appropriate for each prover
blanchet
parents:
47912
diff
changeset
|
335 |
best_slices = |
44099 | 336 |
(* FUDGE *) |
47914
94f37848b7c9
LEO-II's "--sos" option confusingly disables rather than enables SOS, and SOS seems to be ignored anyway; also, pass a number of facts that's more appropriate for each prover
blanchet
parents:
47912
diff
changeset
|
337 |
K [(1.0, (true, ((20, leo2_thf0, "mono_native_higher", keep_lamsN, false), "")))]} |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
338 |
|
47646 | 339 |
val leo2 = (leo2N, fn () => leo2_config) |
44099 | 340 |
|
341 |
||
342 |
(* Satallax *) |
|
343 |
||
44754 | 344 |
val satallax_thf0 = THF (TPTP_Monomorphic, TPTP_Explicit, THF_With_Choice) |
345 |
||
44099 | 346 |
val satallax_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
347 |
{exec = (["SATALLAX_HOME"], "satallax"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
348 |
required_vars = [], |
44099 | 349 |
arguments = |
350 |
fn _ => fn _ => fn _ => fn timeout => fn _ => |
|
45162 | 351 |
"-p hocore -t " ^ string_of_int (to_secs 1 timeout), |
352 |
proof_delims = |
|
353 |
[("% Higher-Order Unsat Core BEGIN", "% Higher-Order Unsat Core END")], |
|
45203 | 354 |
known_failures = known_szs_status_failures, |
47772
993a44ef9928
tentatively tag hypotheses as definition -- this sometimes help the "tptp_sledgehammer" tool (e.g. SEU466^1.p)
blanchet
parents:
47736
diff
changeset
|
355 |
prem_kind = Definition (* motivated by "isabelle tptp_sledgehammer" tool *), |
44416
cabd06b69c18
added formats to the slice and use TFF for remote Vampire
blanchet
parents:
44391
diff
changeset
|
356 |
best_slices = |
44754 | 357 |
(* FUDGE *) |
47914
94f37848b7c9
LEO-II's "--sos" option confusingly disables rather than enables SOS, and SOS seems to be ignored anyway; also, pass a number of facts that's more appropriate for each prover
blanchet
parents:
47912
diff
changeset
|
358 |
K [(1.0, (true, ((120, satallax_thf0, "mono_native_higher", keep_lamsN, false), "")))]} |
44099 | 359 |
|
47646 | 360 |
val satallax = (satallaxN, fn () => satallax_config) |
44099 | 361 |
|
362 |
||
363 |
(* SPASS *) |
|
42725
64dea91bbe0e
added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
blanchet
parents:
42723
diff
changeset
|
364 |
|
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
365 |
fun is_new_spass_version () = |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
366 |
string_ord (getenv "SPASS_VERSION", "3.7") = GREATER orelse |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
367 |
getenv "SPASS_NEW_HOME" <> "" |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
368 |
|
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
369 |
(* TODO: Legacy: Remove after planned Isabelle2012 release (and don't forget |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
370 |
"required_vars" and "script/spass"). *) |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
371 |
val spass_old_config : atp_config = |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
372 |
{exec = (["ISABELLE_ATP"], "scripts/spass"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
373 |
required_vars = [["SPASS_OLD_HOME", "SPASS_HOME"]], |
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43567
diff
changeset
|
374 |
arguments = fn _ => fn _ => fn sos => fn timeout => fn _ => |
37962
d7dbe01f48d7
keep track of clause numbers for SPASS now that we generate FOF rather than CNF problems;
blanchet
parents:
37926
diff
changeset
|
375 |
("-Auto -PGiven=0 -PProblem=0 -Splits=0 -FullRed=0 -DocProof \ |
43981
404ae49ce29f
give E at least two seconds -- anything else risks causing too early timeouts in the minimizer, because of too conservative time computations in E and eproof scripts
blanchet
parents:
43850
diff
changeset
|
376 |
\-VarWeight=3 -TimeLimit=" ^ string_of_int (to_secs 1 timeout)) |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
377 |
|> sos = sosN ? prefix "-SOS=1 ", |
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
378 |
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
|
379 |
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
|
380 |
known_perl_failures @ |
43050
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
42999
diff
changeset
|
381 |
[(GaveUp, "SPASS beiseite: Completion found"), |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
382 |
(TimedOut, "SPASS beiseite: Ran out of time"), |
36965 | 383 |
(OutOfResources, "SPASS beiseite: Maximal number of loops exceeded"), |
37413 | 384 |
(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
|
385 |
(MalformedInput, "Free Variable"), |
44391 | 386 |
(Unprovable, "No formulae and clauses found in input file"), |
39263
e2a3c435334b
more precise error messages when Vampire is interrupted or SPASS runs into an internal bug
blanchet
parents:
39262
diff
changeset
|
387 |
(InternalError, "Please report this error")], |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
388 |
prem_kind = Conjecture, |
42725
64dea91bbe0e
added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
blanchet
parents:
42723
diff
changeset
|
389 |
best_slices = fn ctxt => |
42723 | 390 |
(* FUDGE *) |
46449 | 391 |
[(0.333, (false, ((150, DFG DFG_Unsorted, "mono_tags??", liftingN, false), sosN))), |
392 |
(0.333, (false, ((300, DFG DFG_Unsorted, "poly_tags??", liftingN, false), sosN))), |
|
393 |
(0.334, (false, ((50, DFG DFG_Unsorted, "mono_tags??", liftingN, false), no_sosN)))] |
|
394 |
|> (if Config.get ctxt force_sos then hd #> apfst (K 1.0) #> single else I)} |
|
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
395 |
|
47646 | 396 |
val spass_old = (spass_oldN, fn () => spass_old_config) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
397 |
|
47149 | 398 |
val spass_new_H1SOS = "-Heuristic=1 -SOS" |
46449 | 399 |
val spass_new_H2 = "-Heuristic=2" |
46455 | 400 |
val spass_new_H2SOS = "-Heuristic=2 -SOS" |
401 |
val spass_new_H2NuVS0 = "-Heuristic=2 -RNuV=1 -Sorts=0" |
|
402 |
val spass_new_H2NuVS0Red2 = |
|
403 |
"-Heuristic=2 -RNuV=1 -Sorts=0 -RFRew=2 -RBRew=2 -RTaut=2" |
|
46449 | 404 |
|
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
405 |
val spass_new_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
406 |
{exec = (["SPASS_NEW_HOME", "SPASS_HOME"], "SPASS"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
407 |
required_vars = [], |
46444 | 408 |
arguments = fn _ => fn _ => fn extra_options => fn timeout => fn _ => |
46429 | 409 |
("-Isabelle=1 -TimeLimit=" ^ string_of_int (to_secs 1 timeout)) |
46444 | 410 |
|> extra_options <> "" ? prefix (extra_options ^ " "), |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
411 |
proof_delims = #proof_delims spass_old_config, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
412 |
known_failures = #known_failures spass_old_config, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
413 |
prem_kind = #prem_kind spass_old_config, |
46381 | 414 |
best_slices = fn _ => |
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
415 |
(* FUDGE *) |
46455 | 416 |
[(0.1667, (false, ((150, DFG DFG_Sorted, "mono_native", combsN, true), ""))), |
417 |
(0.1667, (false, ((500, DFG DFG_Sorted, "mono_native", liftingN, true), spass_new_H2SOS))), |
|
418 |
(0.1666, (false, ((50, DFG DFG_Sorted, "mono_native", liftingN, true), spass_new_H2))), |
|
419 |
(0.1000, (false, ((250, DFG DFG_Sorted, "mono_native", combsN, true), spass_new_H2NuVS0))), |
|
47149 | 420 |
(0.1000, (false, ((1000, DFG DFG_Sorted, "mono_native", liftingN, true), spass_new_H1SOS))), |
46455 | 421 |
(0.1000, (false, ((150, DFG DFG_Sorted, "poly_guards??", liftingN, false), spass_new_H2NuVS0Red2))), |
47931
406d1df3787e
minor slice tweaking (swapped two slices to move polymorphic encoding up a bit)
blanchet
parents:
47916
diff
changeset
|
422 |
(0.1000, (false, ((300, DFG DFG_Sorted, "mono_native", combsN, true), spass_new_H2SOS))), |
406d1df3787e
minor slice tweaking (swapped two slices to move polymorphic encoding up a bit)
blanchet
parents:
47916
diff
changeset
|
423 |
(0.1000, (false, ((100, DFG DFG_Sorted, "mono_native", combs_and_liftingN, true), spass_new_H2NuVS0)))]} |
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
424 |
|
47646 | 425 |
val spass_new = (spass_newN, fn () => spass_new_config) |
45301
866b075aa99b
added sorted DFG output for coming version of SPASS
blanchet
parents:
45300
diff
changeset
|
426 |
|
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
427 |
val spass = |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
428 |
(spassN, fn () => if is_new_spass_version () then spass_new_config |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
429 |
else spass_old_config) |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
430 |
|
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
431 |
(* Vampire *) |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
432 |
|
44507
e08158671ef4
disable TFF for Vampire 1.8 until they've fixed the soundness issues and it's back on SystemOnTPTP
blanchet
parents:
44503
diff
changeset
|
433 |
(* Vampire 1.8 has TFF support, but it's buggy and therefore disabled on |
e08158671ef4
disable TFF for Vampire 1.8 until they've fixed the soundness issues and it's back on SystemOnTPTP
blanchet
parents:
44503
diff
changeset
|
434 |
SystemOnTPTP. *) |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
435 |
fun is_new_vampire_version () = |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
436 |
string_ord (getenv "VAMPIRE_VERSION", "1.8") = GREATER |
44420 | 437 |
|
44754 | 438 |
val vampire_tff0 = TFF (TPTP_Monomorphic, TPTP_Implicit) |
44589
0a1dfc6365e9
first step towards polymorphic TFF + changed defaults for Vampire
blanchet
parents:
44586
diff
changeset
|
439 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
440 |
val vampire_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
441 |
{exec = (["VAMPIRE_HOME"], "vampire"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
442 |
required_vars = [], |
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43567
diff
changeset
|
443 |
arguments = fn _ => fn _ => fn sos => fn timeout => fn _ => |
44417 | 444 |
"--mode casc -t " ^ string_of_int (to_secs 1 timeout) ^ |
45234
5509362b924b
disable Vampire's BDD optimization, which sometimes yields so huge proofs that this causes problems for reconstruction
blanchet
parents:
45207
diff
changeset
|
445 |
" --proof tptp --output_axiom_names on\ |
5509362b924b
disable Vampire's BDD optimization, which sometimes yields so huge proofs that this causes problems for reconstruction
blanchet
parents:
45207
diff
changeset
|
446 |
\ --forced_options propositional_to_bdd=off\ |
44417 | 447 |
\ --thanks \"Andrei and Krystof\" --input_file" |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
448 |
|> sos = sosN ? prefix "--sos on ", |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
449 |
proof_delims = |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
450 |
[("=========== Refutation ==========", |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
451 |
"======= End of refutation ======="), |
38033 | 452 |
("% SZS output start Refutation", "% SZS output end Refutation"), |
453 |
("% 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
|
454 |
known_failures = |
45203 | 455 |
known_szs_status_failures @ |
43050
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
42999
diff
changeset
|
456 |
[(GaveUp, "UNPROVABLE"), |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
42999
diff
changeset
|
457 |
(GaveUp, "CANNOT PROVE"), |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
458 |
(Unprovable, "Satisfiability detected"), |
38647
5500241da479
play with fudge factor + parse one more Vampire error
blanchet
parents:
38646
diff
changeset
|
459 |
(Unprovable, "Termination reason: Satisfiable"), |
39263
e2a3c435334b
more precise error messages when Vampire is interrupted or SPASS runs into an internal bug
blanchet
parents:
39262
diff
changeset
|
460 |
(Interrupted, "Aborted by signal SIGINT")], |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
461 |
prem_kind = Conjecture, |
42725
64dea91bbe0e
added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
blanchet
parents:
42723
diff
changeset
|
462 |
best_slices = fn ctxt => |
42723 | 463 |
(* FUDGE *) |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
464 |
(if is_new_vampire_version () then |
47948 | 465 |
[(0.333, (false, ((500, vampire_tff0, "mono_native", combs_or_liftingN, false), sosN))), |
466 |
(0.333, (false, ((150, vampire_tff0, "poly_guards??", combs_or_liftingN, false), sosN))), |
|
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
467 |
(0.334, (true, ((50, vampire_tff0, "mono_native", combs_or_liftingN, false), no_sosN)))] |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
468 |
else |
46449 | 469 |
[(0.333, (false, ((150, FOF, "poly_guards??", combs_or_liftingN, false), sosN))), |
470 |
(0.333, (false, ((500, FOF, "mono_tags??", combs_or_liftingN, false), sosN))), |
|
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
471 |
(0.334, (true, ((50, FOF, "mono_guards??", combs_or_liftingN, false), no_sosN)))]) |
44099 | 472 |
|> (if Config.get ctxt force_sos then hd #> apfst (K 1.0) #> single |
42725
64dea91bbe0e
added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
blanchet
parents:
42723
diff
changeset
|
473 |
else I)} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
474 |
|
47646 | 475 |
val vampire = (vampireN, fn () => vampire_config) |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
476 |
|
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
477 |
|
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
478 |
(* Z3 with TPTP syntax *) |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
479 |
|
44754 | 480 |
val z3_tff0 = TFF (TPTP_Monomorphic, TPTP_Implicit) |
44589
0a1dfc6365e9
first step towards polymorphic TFF + changed defaults for Vampire
blanchet
parents:
44586
diff
changeset
|
481 |
|
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
482 |
val z3_tptp_config : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
483 |
{exec = (["Z3_HOME"], "z3"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
484 |
required_vars = [], |
43354
396aaa15dd8b
pass --trim option to "eproof" script to speed up proof reconstruction
blanchet
parents:
43288
diff
changeset
|
485 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn _ => |
44420 | 486 |
"MBQI=true -tptp -t:" ^ string_of_int (to_secs 1 timeout), |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
487 |
proof_delims = [], |
45203 | 488 |
known_failures = known_szs_status_failures, |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
489 |
prem_kind = Hypothesis, |
42723 | 490 |
best_slices = |
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
491 |
(* FUDGE *) |
46435 | 492 |
K [(0.5, (false, ((250, z3_tff0, "mono_native", combsN, false), ""))), |
493 |
(0.25, (false, ((125, z3_tff0, "mono_native", combsN, false), ""))), |
|
494 |
(0.125, (false, ((62, z3_tff0, "mono_native", combsN, false), ""))), |
|
495 |
(0.125, (false, ((31, z3_tff0, "mono_native", combsN, false), "")))]} |
|
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
496 |
|
47646 | 497 |
val z3_tptp = (z3_tptpN, fn () => z3_tptp_config) |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
498 |
|
44590 | 499 |
|
44754 | 500 |
(* Not really a prover: Experimental Polymorphic TFF and THF output *) |
44590 | 501 |
|
44754 | 502 |
fun dummy_config format type_enc : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
503 |
{exec = (["ISABELLE_ATP"], "scripts/dummy_atp"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
504 |
required_vars = [], |
44590 | 505 |
arguments = K (K (K (K (K "")))), |
506 |
proof_delims = [], |
|
45203 | 507 |
known_failures = known_szs_status_failures, |
44590 | 508 |
prem_kind = Hypothesis, |
45521 | 509 |
best_slices = |
46407
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
510 |
K [(1.0, (false, ((200, format, type_enc, |
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
511 |
if is_format_higher_order format then keep_lamsN |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
512 |
else combsN, false), "")))]} |
44590 | 513 |
|
45365 | 514 |
val dummy_thf_format = THF (TPTP_Polymorphic, TPTP_Explicit, THF_With_Choice) |
46435 | 515 |
val dummy_thf_config = dummy_config dummy_thf_format "poly_native_higher" |
47646 | 516 |
val dummy_thf = (dummy_thfN, fn () => dummy_thf_config) |
44754 | 517 |
|
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
518 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
519 |
(* Remote ATP invocation via SystemOnTPTP *) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
520 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
521 |
val systems = Synchronized.var "atp_systems" ([] : string list) |
31835 | 522 |
|
523 |
fun get_systems () = |
|
44589
0a1dfc6365e9
first step towards polymorphic TFF + changed defaults for Vampire
blanchet
parents:
44586
diff
changeset
|
524 |
case Isabelle_System.bash_output |
0a1dfc6365e9
first step towards polymorphic TFF + changed defaults for Vampire
blanchet
parents:
44586
diff
changeset
|
525 |
"\"$ISABELLE_ATP/scripts/remote_atp\" -w 2>&1" of |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
526 |
(output, 0) => split_lines output |
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
527 |
| (output, _) => |
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
528 |
error (case extract_known_failure known_perl_failures output of |
41744 | 529 |
SOME failure => string_for_failure failure |
47499
4b0daca2bf88
redirect bash stderr to Isabelle warning as appropriate -- avoid raw process error output which may either get ignored or overload PIDE syslog in extreme cases;
wenzelm
parents:
47149
diff
changeset
|
530 |
| NONE => trim_line output ^ ".") |
31835 | 531 |
|
42537
25ceb855a18b
improve version handling -- prefer versions of ToFoF, SInE, and SNARK that are known to work
blanchet
parents:
42535
diff
changeset
|
532 |
fun find_system name [] systems = |
25ceb855a18b
improve version handling -- prefer versions of ToFoF, SInE, and SNARK that are known to work
blanchet
parents:
42535
diff
changeset
|
533 |
find_first (String.isPrefix (name ^ "---")) 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
|
534 |
| 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
|
535 |
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
|
536 |
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
|
537 |
| 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
|
538 |
|
38a926e033ad
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
blanchet
parents:
38685
diff
changeset
|
539 |
fun get_system name versions = |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
540 |
Synchronized.change_result systems |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38588
diff
changeset
|
541 |
(fn systems => (if null systems then get_systems () else systems) |
42955 | 542 |
|> `(`(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
|
543 |
|
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
|
544 |
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
|
545 |
case get_system name versions of |
42955 | 546 |
(SOME sys, _) => sys |
46480 | 547 |
| (NONE, []) => error ("SystemOnTPTP is not available.") |
42955 | 548 |
| (NONE, syss) => |
46480 | 549 |
case syss |> filter_out (String.isPrefix "%") |
550 |
|> filter_out (curry (op =) "") of |
|
551 |
[] => error ("SystemOnTPTP is not available.") |
|
552 |
| [msg] => error ("SystemOnTPTP is not available: " ^ msg ^ ".") |
|
553 |
| syss => |
|
554 |
error ("System " ^ quote name ^ " is not available at SystemOnTPTP.\n" ^ |
|
555 |
"(Available systems: " ^ commas_quote syss ^ ".)") |
|
31835 | 556 |
|
41148 | 557 |
val max_remote_secs = 240 (* give Geoff Sutcliffe's servers a break *) |
558 |
||
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
|
559 |
fun remote_config system_name system_versions proof_delims known_failures |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
560 |
prem_kind best_slice : atp_config = |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
561 |
{exec = (["ISABELLE_ATP"], "scripts/remote_atp"), |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
562 |
required_vars = [], |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
563 |
arguments = fn _ => fn _ => fn command => fn timeout => fn _ => |
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
564 |
(if command <> "" then "-c " ^ quote command ^ " " else "") ^ |
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
565 |
"-s " ^ the_system system_name system_versions ^ " " ^ |
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
566 |
"-t " ^ string_of_int (Int.min (max_remote_secs, to_secs 1 timeout)), |
42962
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
blanchet
parents:
42955
diff
changeset
|
567 |
proof_delims = union (op =) tstp_proof_delims proof_delims, |
45203 | 568 |
known_failures = known_failures @ known_perl_failures @ known_says_failures, |
42709
e7af132d48fe
allow each prover to specify its own formula kind for symbols occurring in the conjecture
blanchet
parents:
42708
diff
changeset
|
569 |
prem_kind = prem_kind, |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
570 |
best_slices = fn ctxt => [(1.0, (false, best_slice ctxt))]} |
42443
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42332
diff
changeset
|
571 |
|
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
572 |
fun remotify_config system_name system_versions best_slice |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
573 |
({proof_delims, known_failures, prem_kind, ...} : atp_config) |
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
574 |
: atp_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
|
575 |
remote_config system_name system_versions proof_delims known_failures |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
576 |
prem_kind best_slice |
38023 | 577 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
578 |
fun remote_atp name system_name system_versions proof_delims known_failures |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
579 |
prem_kind best_slice = |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
580 |
(remote_prefix ^ name, |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
581 |
fn () => remote_config system_name system_versions proof_delims |
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
582 |
known_failures prem_kind best_slice) |
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
583 |
fun remotify_atp (name, config) system_name system_versions best_slice = |
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
584 |
(remote_prefix ^ name, |
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
585 |
remotify_config system_name system_versions best_slice o config) |
28592 | 586 |
|
44754 | 587 |
val explicit_tff0 = TFF (TPTP_Monomorphic, TPTP_Explicit) |
44589
0a1dfc6365e9
first step towards polymorphic TFF + changed defaults for Vampire
blanchet
parents:
44586
diff
changeset
|
588 |
|
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
589 |
val remote_e = |
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
590 |
remotify_atp e "EP" ["1.0", "1.1", "1.2"] |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
591 |
(K ((750, FOF, "mono_tags??", combsN, false), "") (* FUDGE *)) |
44099 | 592 |
val remote_leo2 = |
593 |
remotify_atp leo2 "LEO-II" ["1.2.8", "1.2.6"] |
|
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
594 |
(K ((100, leo2_thf0, "mono_native_higher", liftingN, false), "") (* FUDGE *)) |
44099 | 595 |
val remote_satallax = |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
596 |
remotify_atp satallax "Satallax" ["2.3", "2.2", "2"] |
47076
f4838ce57772
removed Satallax option, now that this is the default
blanchet
parents:
47074
diff
changeset
|
597 |
(K ((100, satallax_thf0, "mono_native_higher", keep_lamsN, false), "") (* FUDGE *)) |
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
598 |
val remote_vampire = |
44499 | 599 |
remotify_atp vampire "Vampire" ["1.8"] |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
600 |
(K ((250, vampire_tff0, "mono_native", combs_or_liftingN, false), "") (* FUDGE *)) |
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
601 |
val remote_z3_tptp = |
44754 | 602 |
remotify_atp z3_tptp "Z3" ["3.0"] |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
603 |
(K ((250, z3_tff0, "mono_native", combsN, false), "") (* FUDGE *)) |
44092
bf489e54d7f8
renamed E wrappers for consistency with CASC conventions
blanchet
parents:
43989
diff
changeset
|
604 |
val remote_e_sine = |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
605 |
remote_atp e_sineN "SInE" ["0.4"] [] (#known_failures e_config) Conjecture |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
606 |
(K ((500, FOF, "mono_guards??", combsN, false), "") (* FUDGE *)) |
45338 | 607 |
val remote_iprover = |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
608 |
remote_atp iproverN "iProver" [] [] [] Conjecture |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
609 |
(K ((150, FOF, "mono_guards??", liftingN, false), "") (* FUDGE *)) |
45338 | 610 |
val remote_iprover_eq = |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
611 |
remote_atp iprover_eqN "iProver-Eq" [] [] [] Conjecture |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
612 |
(K ((150, FOF, "mono_guards??", liftingN, false), "") (* FUDGE *)) |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
613 |
val remote_snark = |
42939 | 614 |
remote_atp snarkN "SNARK" ["20080805r029", "20080805r024"] |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
615 |
[("refutation.", "end_refutation.")] [] Hypothesis |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
616 |
(K ((100, explicit_tff0, "mono_native", liftingN, false), "") (* FUDGE *)) |
44092
bf489e54d7f8
renamed E wrappers for consistency with CASC conventions
blanchet
parents:
43989
diff
changeset
|
617 |
val remote_e_tofof = |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
618 |
remote_atp e_tofofN "ToFoF" ["0.1"] [] (#known_failures e_config) Hypothesis |
47074
101976132929
improve "remote_satallax" by exploiting unsat core
blanchet
parents:
47073
diff
changeset
|
619 |
(K ((150, explicit_tff0, "mono_native", liftingN, false), "") (* FUDGE *)) |
42938 | 620 |
val remote_waldmeister = |
621 |
remote_atp waldmeisterN "Waldmeister" ["710"] |
|
45521 | 622 |
[("#START OF PROOF", "Proved Goals:")] |
623 |
[(OutOfResources, "Too many function symbols"), |
|
47506 | 624 |
(Inappropriate, "**** Unexpected end of file."), |
45521 | 625 |
(Crashed, "Unrecoverable Segmentation Fault")] |
47912
12de57c5eee5
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
blanchet
parents:
47900
diff
changeset
|
626 |
Hypothesis |
47898
6213900d6d5f
use raw monomorphic encoding with Waldmeister, to avoid overloading it with too many function symbols (as would be the case using mangled monomorphic encodings)
blanchet
parents:
47787
diff
changeset
|
627 |
(K ((50, CNF_UEQ, "raw_mono_tags??", combsN, false), "") (* FUDGE *)) |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
628 |
|
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
629 |
(* Setup *) |
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
630 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
631 |
fun add_atp (name, config) thy = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
632 |
Data.map (Symtab.update_new (name, (config, stamp ()))) thy |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
633 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name ^ ".") |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
634 |
|
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
635 |
fun get_atp thy name = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
636 |
the (Symtab.lookup (Data.get thy) name) |> fst |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
637 |
handle Option.Option => error ("Unknown ATP: " ^ name ^ ".") |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
638 |
|
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41725
diff
changeset
|
639 |
val supported_atps = Symtab.keys o Data.get |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
640 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
641 |
fun is_atp_installed thy name = |
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
642 |
let val {exec, required_vars, ...} = get_atp thy name () in |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
643 |
forall (exists (fn var => getenv var <> "")) (fst exec :: required_vars) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
644 |
end |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
645 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
646 |
fun refresh_systems_on_tptp () = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
647 |
Synchronized.change systems (fn _ => get_systems ()) |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
648 |
|
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
649 |
fun effective_term_order ctxt atp = |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
650 |
let val ord = Config.get ctxt term_order in |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
651 |
if ord = smartN then |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
652 |
if atp = spass_newN orelse |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
653 |
(atp = spassN andalso is_new_spass_version ()) then |
47073
c73f7b0c7ebc
generate weights and precedences for predicates as well
blanchet
parents:
47055
diff
changeset
|
654 |
{is_lpo = false, gen_weights = true, gen_prec = true, gen_simp = false} |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
655 |
else |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
656 |
{is_lpo = false, gen_weights = false, gen_prec = false, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
657 |
gen_simp = false} |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
658 |
else |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
659 |
let val is_lpo = String.isSubstring lpoN ord in |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
660 |
{is_lpo = is_lpo, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
661 |
gen_weights = not is_lpo andalso String.isSubstring xweightsN ord, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
662 |
gen_prec = String.isSubstring xprecN ord, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
663 |
gen_simp = String.isSubstring xsimpN ord} |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
664 |
end |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
665 |
end |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
666 |
|
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
667 |
val atps= |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
668 |
[alt_ergo, e, leo2, dummy_thf, satallax, spass_old, spass_new, spass, |
47055
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
669 |
vampire, z3_tptp, remote_e, remote_e_sine, remote_e_tofof, remote_iprover, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
670 |
remote_iprover_eq, remote_leo2, remote_satallax, remote_vampire, |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
671 |
remote_z3_tptp, remote_snark, remote_waldmeister] |
16e2633f3b4b
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
blanchet
parents:
47053
diff
changeset
|
672 |
|
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
673 |
val setup = fold add_atp atps |
35867 | 674 |
|
28592 | 675 |
end; |