author | blanchet |
Fri, 25 Oct 2019 15:59:25 +0200 | |
changeset 70940 | ce3a05ad07b7 |
parent 70939 | 3218999b3715 |
child 70941 | d4ef7617e31e |
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 |
53586
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
12 |
type atp_formula_role = ATP_Problem.atp_formula_role |
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
13 |
type atp_failure = ATP_Proof.atp_failure |
38023 | 14 |
|
51011 | 15 |
type slice_spec = (int * string) * 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 = |
57671
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
17 |
{exec : bool -> string list * string list, |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
18 |
arguments : Proof.context -> bool -> string -> Time.time -> string -> |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
19 |
term_order * (unit -> (string * int) list) * (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
|
20 |
proof_delims : (string * string) list, |
53586
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
21 |
known_failures : (atp_failure * string) list, |
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
22 |
prem_role : atp_formula_role, |
48716
1d2a12bb0640
stop distinguishing between complete and incomplete slices, since this is very fragile and has hardly any useful semantics to users
blanchet
parents:
48715
diff
changeset
|
23 |
best_slices : Proof.context -> (real * (slice_spec * string)) list, |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
24 |
best_max_mono_iters : int, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
25 |
best_max_new_mono_instances : int} |
38023 | 26 |
|
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
27 |
val default_max_mono_iters : int |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
28 |
val default_max_new_mono_instances : int |
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 |
50950 | 42 |
val spass_H1SOS : string |
43 |
val spass_H2 : string |
|
44 |
val spass_H2LR0LT0 : string |
|
45 |
val spass_H2NuVS0 : string |
|
46 |
val spass_H2NuVS0Red2 : string |
|
47 |
val spass_H2SOS : string |
|
48 |
val spass_extra_options : string Config.T |
|
68563 | 49 |
val is_vampire_noncommercial_license_accepted : unit -> bool option |
57671
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
50 |
val remote_atp : string -> string -> string list -> (string * string) list -> |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
51 |
(atp_failure * string) list -> atp_formula_role -> (Proof.context -> slice_spec * string) -> |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
52 |
string * (unit -> atp_config) |
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
53 |
val add_atp : string * (unit -> atp_config) -> theory -> theory |
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
54 |
val get_atp : theory -> string -> (unit -> atp_config) |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41725
diff
changeset
|
55 |
val supported_atps : theory -> string list |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
56 |
val is_atp_installed : theory -> string -> bool |
35867 | 57 |
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
|
58 |
val effective_term_order : Proof.context -> string -> term_order |
28592 | 59 |
end; |
60 |
||
36376 | 61 |
structure ATP_Systems : ATP_SYSTEMS = |
28592 | 62 |
struct |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
63 |
|
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
|
64 |
open ATP_Problem |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
65 |
open ATP_Proof |
46320 | 66 |
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
|
67 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
68 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
69 |
(* ATP configuration *) |
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
70 |
|
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
71 |
val default_max_mono_iters = 3 (* FUDGE *) |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
72 |
val default_max_new_mono_instances = 100 (* FUDGE *) |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
73 |
|
51011 | 74 |
type slice_spec = (int * string) * atp_format * string * string * bool |
46409
d4754183ccce
made option available to users (mostly for experiments)
blanchet
parents:
46407
diff
changeset
|
75 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
76 |
type atp_config = |
57671
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
77 |
{exec : bool -> string list * string list, |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
78 |
arguments : Proof.context -> bool -> string -> Time.time -> string -> |
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
79 |
term_order * (unit -> (string * int) list) * (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
|
80 |
proof_delims : (string * string) list, |
53586
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
81 |
known_failures : (atp_failure * string) list, |
bd5fa6425993
prefixed types and some functions with "atp_" for disambiguation
blanchet
parents:
53515
diff
changeset
|
82 |
prem_role : atp_formula_role, |
48716
1d2a12bb0640
stop distinguishing between complete and incomplete slices, since this is very fragile and has hardly any useful semantics to users
blanchet
parents:
48715
diff
changeset
|
83 |
best_slices : Proof.context -> (real * (slice_spec * string)) list, |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
84 |
best_max_mono_iters : int, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
85 |
best_max_new_mono_instances : int} |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
86 |
|
42723 | 87 |
(* "best_slices" must be found empirically, taking a wholistic approach since |
51011 | 88 |
the ATPs are run in parallel. Each slice has the format |
89 |
||
90 |
(time_frac, ((max_facts, fact_filter), format, type_enc, |
|
91 |
lam_trans, uncurried_aliases), extra) |
|
92 |
||
93 |
where |
|
94 |
||
95 |
time_frac = faction of the time available given to the slice (which should |
|
96 |
add up to 1.0) |
|
97 |
||
98 |
extra = extra information to the prover (e.g., SOS or no SOS). |
|
42723 | 99 |
|
100 |
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
|
101 |
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
|
102 |
slicing is disabled (e.g., by the minimizer). *) |
42710
84fcce345b5d
further improved type system setup based on Judgment Days
blanchet
parents:
42709
diff
changeset
|
103 |
|
51011 | 104 |
val mepoN = "mepo" |
105 |
val mashN = "mash" |
|
106 |
val meshN = "mesh" |
|
107 |
||
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
108 |
val tstp_proof_delims = |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
109 |
[("% SZS output start CNFRefutation", "% SZS output end CNFRefutation"), |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
110 |
("% SZS output start Refutation", "% SZS output end Refutation"), |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
111 |
("% SZS output start Proof", "% SZS output end Proof")] |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
112 |
|
38061
685d1f0f75b3
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents:
38049
diff
changeset
|
113 |
val known_perl_failures = |
38094 | 114 |
[(CantConnect, "HTTP error"), |
115 |
(NoPerl, "env: perl"), |
|
38065 | 116 |
(NoLibwwwPerl, "Can't locate HTTP")] |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
117 |
|
45203 | 118 |
fun known_szs_failures wrap = |
119 |
[(Unprovable, wrap "CounterSatisfiable"), |
|
120 |
(Unprovable, wrap "Satisfiable"), |
|
121 |
(GaveUp, wrap "GaveUp"), |
|
122 |
(GaveUp, wrap "Unknown"), |
|
123 |
(GaveUp, wrap "Incomplete"), |
|
124 |
(ProofMissing, wrap "Theorem"), |
|
125 |
(ProofMissing, wrap "Unsatisfiable"), |
|
126 |
(TimedOut, wrap "Timeout"), |
|
127 |
(Inappropriate, wrap "Inappropriate"), |
|
128 |
(OutOfResources, wrap "ResourceOut"), |
|
129 |
(OutOfResources, wrap "MemoryOut"), |
|
130 |
(Interrupted, wrap "Forced"), |
|
131 |
(Interrupted, wrap "User")] |
|
132 |
||
133 |
val known_szs_status_failures = known_szs_failures (prefix "SZS status ") |
|
134 |
val known_says_failures = known_szs_failures (prefix " says ") |
|
135 |
||
38023 | 136 |
structure Data = Theory_Data |
137 |
( |
|
47606
06dde48a1503
true delayed evaluation of "SPASS_VERSION" environment variable
blanchet
parents:
47506
diff
changeset
|
138 |
type T = ((unit -> atp_config) * stamp) Symtab.table |
38023 | 139 |
val empty = Symtab.empty |
140 |
val extend = I |
|
46407
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
141 |
fun merge data : T = |
30e9720cc0b9
optimization: slice caching in case two consecutive slices are nearly identical
blanchet
parents:
46402
diff
changeset
|
142 |
Symtab.merge (eq_snd (op =)) data |
63692 | 143 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name) |
38023 | 144 |
) |
38017
3ad3e3ca2451
move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
blanchet
parents:
38015
diff
changeset
|
145 |
|
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
|
146 |
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
|
147 |
|
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
148 |
val sosN = "sos" |
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
149 |
val no_sosN = "no_sos" |
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
150 |
|
69593 | 151 |
val force_sos = Attrib.setup_config_bool \<^binding>\<open>atp_force_sos\<close> (K false) |
44099 | 152 |
|
47032 | 153 |
val smartN = "smart" |
47073
c73f7b0c7ebc
generate weights and precedences for predicates as well
blanchet
parents:
47055
diff
changeset
|
154 |
(* val kboN = "kbo" *) |
47032 | 155 |
val lpoN = "lpo" |
47034
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
156 |
val xweightsN = "_weights" |
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
157 |
val xprecN = "_prec" |
77da780ddd6b
implement term order attribute (for experiments)
blanchet
parents:
47033
diff
changeset
|
158 |
val xsimpN = "_simp" (* SPASS-specific *) |
47032 | 159 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
160 |
(* Possible values for "atp_term_order": |
47049 | 161 |
"smart", "(kbo|lpo)(_weights)?(_prec|_simp)?" *) |
47032 | 162 |
val term_order = |
69593 | 163 |
Attrib.setup_config_string \<^binding>\<open>atp_term_order\<close> (K smartN) |
47032 | 164 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
165 |
|
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
166 |
(* agsyHOL *) |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
167 |
|
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
168 |
val agsyhol_config : atp_config = |
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
169 |
{exec = K (["AGSYHOL_HOME"], ["agsyHOL"]), |
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
170 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
68563 | 171 |
"--proof --time-out " ^ string_of_int (to_secs 1 timeout) ^ " " ^ file_name, |
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
172 |
proof_delims = tstp_proof_delims, |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
173 |
known_failures = known_szs_status_failures, |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
174 |
prem_role = Hypothesis, |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
175 |
best_slices = |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
176 |
(* FUDGE *) |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
177 |
K [(1.0, (((60, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), ""))], |
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
178 |
best_max_mono_iters = default_max_mono_iters - 1 (* FUDGE *), |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
179 |
best_max_new_mono_instances = default_max_new_mono_instances} |
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
180 |
|
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
181 |
val agsyhol = (agsyholN, fn () => agsyhol_config) |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
182 |
|
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
183 |
|
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
184 |
(* Alt-Ergo *) |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
185 |
|
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
186 |
val alt_ergo_config : atp_config = |
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
187 |
{exec = K (["WHY3_HOME"], ["why3"]), |
50927 | 188 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
68563 | 189 |
"--format tptp --prover 'Alt-Ergo,0.95.2,' --timelimit " ^ string_of_int (to_secs 1 timeout) ^ |
190 |
" " ^ file_name, |
|
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
191 |
proof_delims = [], |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
192 |
known_failures = |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
193 |
[(ProofMissing, ": Valid"), |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
194 |
(TimedOut, ": Timeout"), |
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
195 |
(GaveUp, ": Unknown")], |
47976 | 196 |
prem_role = Hypothesis, |
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
197 |
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
|
198 |
(* FUDGE *) |
57547
677b07d777c3
don't generate TPTP THF 'Definition's, because they complicate reconstruction for AgsyHOL and Satallax
blanchet
parents:
57293
diff
changeset
|
199 |
[(1.0, (((100, ""), TFF Polymorphic, "poly_native", liftingN, false), ""))], |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
200 |
best_max_mono_iters = default_max_mono_iters, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
201 |
best_max_new_mono_instances = default_max_new_mono_instances} |
46643
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
202 |
|
47646 | 203 |
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
|
204 |
|
a88bccd2b567
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
blanchet
parents:
46481
diff
changeset
|
205 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
206 |
(* E *) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
207 |
|
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
208 |
val e_smartN = "smart" |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
209 |
val e_autoN = "auto" |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
210 |
val e_fun_weightN = "fun_weight" |
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
211 |
val e_sym_offset_weightN = "sym_offset_weight" |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
212 |
|
47032 | 213 |
val e_selection_heuristic = |
69593 | 214 |
Attrib.setup_config_string \<^binding>\<open>atp_e_selection_heuristic\<close> (K e_smartN) |
41770 | 215 |
(* FUDGE *) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
216 |
val e_default_fun_weight = |
69593 | 217 |
Attrib.setup_config_real \<^binding>\<open>atp_e_default_fun_weight\<close> (K 20.0) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
218 |
val e_fun_weight_base = |
69593 | 219 |
Attrib.setup_config_real \<^binding>\<open>atp_e_fun_weight_base\<close> (K 0.0) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
220 |
val e_fun_weight_span = |
69593 | 221 |
Attrib.setup_config_real \<^binding>\<open>atp_e_fun_weight_span\<close> (K 40.0) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
222 |
val e_default_sym_offs_weight = |
69593 | 223 |
Attrib.setup_config_real \<^binding>\<open>atp_e_default_sym_offs_weight\<close> (K 1.0) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
224 |
val e_sym_offs_weight_base = |
69593 | 225 |
Attrib.setup_config_real \<^binding>\<open>atp_e_sym_offs_weight_base\<close> (K ~20.0) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
226 |
val e_sym_offs_weight_span = |
69593 | 227 |
Attrib.setup_config_real \<^binding>\<open>atp_e_sym_offs_weight_span\<close> (K 60.0) |
41725
7cca2de89296
added support for bleeding-edge E weighting function "SymOffsetsWeight"
blanchet
parents:
41335
diff
changeset
|
228 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
229 |
fun e_selection_heuristic_case heuristic fw sow = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
230 |
if heuristic = e_fun_weightN then fw |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
231 |
else if heuristic = e_sym_offset_weightN then sow |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
232 |
else raise Fail ("unexpected " ^ quote heuristic) |
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 scaled_e_selection_weight ctxt heuristic w = |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
235 |
w * Config.get ctxt (e_selection_heuristic_case heuristic |
47029 | 236 |
e_fun_weight_span e_sym_offs_weight_span) |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
237 |
+ Config.get ctxt (e_selection_heuristic_case heuristic |
47029 | 238 |
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
|
239 |
|> 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
|
240 |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
241 |
fun e_selection_weight_arguments ctxt heuristic sel_weights = |
51631 | 242 |
if heuristic = e_fun_weightN orelse heuristic = e_sym_offset_weightN then |
43622 | 243 |
(* supplied by Stephan Schulz *) |
41314
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
244 |
"--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
|
245 |
\--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
|
246 |
\--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
|
247 |
\--delete-bad-limit=150000000 -WSelectMaxLComplexAvoidPosPred -H'(4*" ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
248 |
e_selection_heuristic_case heuristic "FunWeight" "SymOffsetWeight" ^ |
48376
416e4123baf3
use "eproof_ram" script if available (plug-in replacement for "eproof", but faster)
blanchet
parents:
48232
diff
changeset
|
249 |
"(SimulateSOS," ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
250 |
(e_selection_heuristic_case heuristic |
47029 | 251 |
e_default_fun_weight e_default_sym_offs_weight |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
252 |
|> 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
|
253 |
",20,1.5,1.5,1" ^ |
47030 | 254 |
(sel_weights () |
47029 | 255 |
|> map (fn (s, w) => "," ^ s ^ ":" ^ |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
256 |
scaled_e_selection_weight ctxt heuristic w) |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
257 |
|> implode) ^ |
41314
2dc1dfc1bc69
use the options provided by Stephan Schulz -- much better
blanchet
parents:
41313
diff
changeset
|
258 |
"),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
|
259 |
\1.5,1.5,1),1*Clauseweight(PreferProcessed,1,1,1),1*\ |
57672 | 260 |
\FIFOWeight(PreferProcessed))' " |
51631 | 261 |
else |
57672 | 262 |
"-xAuto " |
41313
a96ac4d180b7
optionally supply constant weights to E -- turned off by default until properly parameterized
blanchet
parents:
41269
diff
changeset
|
263 |
|
70939
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
264 |
val e_ord_weights = map (fn (s, w) => s ^ ":" ^ string_of_int w) #> space_implode "," |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
265 |
fun e_ord_precedence [_] = "" |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
266 |
| e_ord_precedence info = info |> map fst |> space_implode "<" |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
267 |
|
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
|
268 |
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
|
269 |
| e_term_order_info_arguments gen_weights gen_prec ord_info = |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
270 |
let val ord_info = ord_info () in |
57672 | 271 |
(if gen_weights then "--order-weights='" ^ e_ord_weights ord_info ^ "' " else "") ^ |
272 |
(if gen_prec then "--precedence='" ^ e_ord_precedence ord_info ^ "' " else "") |
|
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
273 |
end |
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
274 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
275 |
val e_config : atp_config = |
66363 | 276 |
{exec = fn _ => (["E_HOME"], ["eprover"]), |
277 |
arguments = fn ctxt => fn _ => fn heuristic => fn timeout => fn file_name => |
|
57008 | 278 |
fn ({is_lpo, gen_weights, gen_prec, ...}, ord_info, sel_weights) => |
66363 | 279 |
"--auto-schedule --tstp-in --tstp-out --silent " ^ |
57672 | 280 |
e_selection_weight_arguments ctxt heuristic sel_weights ^ |
281 |
e_term_order_info_arguments gen_weights gen_prec ord_info ^ |
|
57636
3ab503b04bdb
stick to external proofs when invoking E, because they are more detailed and do not merge steps
blanchet
parents:
57547
diff
changeset
|
282 |
"--term-ordering=" ^ (if is_lpo then "LPO4" else "KBO6") ^ " " ^ |
48651 | 283 |
"--cpu-limit=" ^ string_of_int (to_secs 2 timeout) ^ |
66363 | 284 |
" --proof-object=1 " ^ |
285 |
file_name, |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
286 |
proof_delims = |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
287 |
[("# SZS output start CNFRefutation", "# SZS output end CNFRefutation")] @ |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
288 |
tstp_proof_delims, |
36265
41c9e755e552
distinguish between the different ATP errors in the user interface;
blanchet
parents:
36264
diff
changeset
|
289 |
known_failures = |
45203 | 290 |
[(TimedOut, "Failure: Resource limit exceeded (time)"), |
47972 | 291 |
(TimedOut, "time limit exceeded")] @ |
292 |
known_szs_status_failures, |
|
47976 | 293 |
prem_role = Conjecture, |
42646
4781fcd53572
replaced some Unsynchronized.refs with Config.Ts
blanchet
parents:
42643
diff
changeset
|
294 |
best_slices = fn ctxt => |
70939
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
295 |
let |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
296 |
val heuristic = Config.get ctxt e_selection_heuristic |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
297 |
val ehoh = string_ord (getenv "E_VERSION", "2.3") <> LESS |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
298 |
val (format, enc) = |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
299 |
if ehoh then (THF (Monomorphic, THF_Predicate_Free), "mono_native_higher") |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
300 |
else (TFF Monomorphic, "mono_native") |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
301 |
in |
43474
423cd1ecf714
optimized E's time slicing, based on latest exhaustive Judgment Day results
blanchet
parents:
43473
diff
changeset
|
302 |
(* FUDGE *) |
47038
2409b484e1cc
continued implementation of term ordering attributes
blanchet
parents:
47034
diff
changeset
|
303 |
if heuristic = e_smartN then |
70939
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
304 |
[(0.15, (((128, meshN), format, enc, combsN, false), e_fun_weightN)), |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
305 |
(0.15, (((128, mashN), format, enc, combsN, false), e_sym_offset_weightN)), |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
306 |
(0.15, (((91, mepoN), format, enc, combsN, false), e_autoN)), |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
307 |
(0.15, (((1000, meshN), format, "poly_guards??", combsN, false), e_sym_offset_weightN)), |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
308 |
(0.15, (((256, mepoN), format, enc, liftingN, false), e_fun_weightN)), |
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
309 |
(0.25, (((64, mashN), format, enc, combsN, false), e_fun_weightN))] |
43473
fb2713b803e6
deal with ATP time slices in a more flexible/robust fashion
blanchet
parents:
43467
diff
changeset
|
310 |
else |
70939
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
311 |
[(1.0, (((500, ""), format, enc, combsN, false), heuristic))] |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
312 |
end, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
313 |
best_max_mono_iters = default_max_mono_iters, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
314 |
best_max_new_mono_instances = default_max_new_mono_instances} |
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 |
|
70938 | 319 |
(* E-Par *) |
48651 | 320 |
|
70938 | 321 |
val e_par_config : atp_config = |
322 |
{exec = K (["E_HOME"], ["runepar.pl"]), |
|
50927 | 323 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
70938 | 324 |
string_of_int (to_secs 1 timeout) ^ " 1 " (* SInE *) ^ file_name ^ " 2" (* proofs *), |
48651 | 325 |
proof_delims = tstp_proof_delims, |
326 |
known_failures = #known_failures e_config, |
|
327 |
prem_role = Conjecture, |
|
328 |
best_slices = |
|
329 |
(* FUDGE *) |
|
51018 | 330 |
K [(0.25, (((500, meshN), FOF, "mono_guards??", combs_or_liftingN, false), "")), |
331 |
(0.25, (((150, meshN), FOF, "poly_tags??", combs_or_liftingN, false), "")), |
|
332 |
(0.25, (((50, meshN), FOF, "mono_tags??", combs_or_liftingN, false), "")), |
|
333 |
(0.25, (((1000, meshN), FOF, "poly_guards??", combsN, false), ""))], |
|
48651 | 334 |
best_max_mono_iters = default_max_mono_iters, |
335 |
best_max_new_mono_instances = default_max_new_mono_instances} |
|
336 |
||
50927 | 337 |
val e_par = (e_parN, fn () => e_par_config) |
338 |
||
339 |
||
48700 | 340 |
(* iProver *) |
341 |
||
342 |
val iprover_config : atp_config = |
|
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
343 |
{exec = K (["IPROVER_HOME"], ["iproveropt", "iprover"]), |
50927 | 344 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
345 |
"--clausifier \"$E_HOME\"/eprover " ^ |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
346 |
"--clausifier_options \"--tstp-format --silent --cnf\" " ^ |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
347 |
"--time_out_real " ^ string_of_real (Time.toReal timeout) ^ " " ^ file_name, |
48700 | 348 |
proof_delims = tstp_proof_delims, |
349 |
known_failures = |
|
350 |
[(ProofIncomplete, "% SZS output start CNFRefutation")] @ |
|
351 |
known_szs_status_failures, |
|
352 |
prem_role = Hypothesis, |
|
353 |
best_slices = |
|
354 |
(* FUDGE *) |
|
51011 | 355 |
K [(1.0, (((150, ""), FOF, "mono_guards??", liftingN, false), ""))], |
48700 | 356 |
best_max_mono_iters = default_max_mono_iters, |
357 |
best_max_new_mono_instances = default_max_new_mono_instances} |
|
358 |
||
359 |
val iprover = (iproverN, fn () => iprover_config) |
|
360 |
||
361 |
||
44099 | 362 |
(* LEO-II *) |
363 |
||
364 |
val leo2_config : atp_config = |
|
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
365 |
{exec = K (["LEO2_HOME"], ["leo.opt", "leo"]), |
57759 | 366 |
arguments = fn _ => fn full_proofs => fn _ => fn timeout => fn file_name => fn _ => |
367 |
"--foatp e --atp e=\"$E_HOME\"/eprover \ |
|
368 |
\--atp epclextract=\"$E_HOME\"/epclextract \ |
|
369 |
\--proofoutput 1 --timeout " ^ string_of_int (to_secs 1 timeout) ^ " " ^ |
|
370 |
(if full_proofs then "--notReplLeibnizEQ --notReplAndrewsEQ --notUseExtCnfCmbd " else "") ^ |
|
371 |
file_name, |
|
44099 | 372 |
proof_delims = tstp_proof_delims, |
45207 | 373 |
known_failures = |
47974
08d2dcc2dab9
improved LEO-II definition handling -- still hoping for a fix directly in LEO-II
blanchet
parents:
47972
diff
changeset
|
374 |
[(TimedOut, "CPU time limit exceeded, terminating"), |
47972 | 375 |
(GaveUp, "No.of.Axioms")] @ |
376 |
known_szs_status_failures, |
|
47976 | 377 |
prem_role = 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
|
378 |
best_slices = |
44099 | 379 |
(* FUDGE *) |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
380 |
K [(1.0, (((40, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), ""))], |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
381 |
best_max_mono_iters = default_max_mono_iters - 1 (* FUDGE *), |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
382 |
best_max_new_mono_instances = default_max_new_mono_instances} |
39491
2416666e6f94
refactoring: move ATP proof and error extraction code to "ATP_Proof" module
blanchet
parents:
39375
diff
changeset
|
383 |
|
47646 | 384 |
val leo2 = (leo2N, fn () => leo2_config) |
44099 | 385 |
|
386 |
||
67021
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
387 |
(* Leo-III *) |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
388 |
|
69717 | 389 |
(* Include choice? Disabled now since it's disabled for Satallax as well. *) |
67021
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
390 |
val leo3_config : atp_config = |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
391 |
{exec = K (["LEO3_HOME"], ["leo3"]), |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
392 |
arguments = fn _ => fn full_proofs => fn _ => fn timeout => fn file_name => fn _ => |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
393 |
file_name ^ " " ^ "--atp cvc=$CVC4_SOLVER --atp e=\"$E_HOME\"/eprover \ |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
394 |
\-p -t " ^ string_of_int (to_secs 1 timeout) ^ " " ^ |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
395 |
(if full_proofs then "--nleq --naeq " else ""), |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
396 |
proof_delims = tstp_proof_delims, |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
397 |
known_failures = known_szs_status_failures, |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
398 |
prem_role = Hypothesis, |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
399 |
best_slices = |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
400 |
(* FUDGE *) |
70940
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
401 |
K [(1.0, (((150, ""), THF (Polymorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), ""))], |
67021
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
402 |
best_max_mono_iters = default_max_mono_iters - 1 (* FUDGE *), |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
403 |
best_max_new_mono_instances = default_max_new_mono_instances} |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
404 |
|
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
405 |
val leo3 = (leo3N, fn () => leo3_config) |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
406 |
|
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
407 |
|
44099 | 408 |
(* Satallax *) |
409 |
||
52097 | 410 |
(* Choice is disabled until there is proper reconstruction for it. *) |
44099 | 411 |
val satallax_config : atp_config = |
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
412 |
{exec = K (["SATALLAX_HOME"], ["satallax.opt", "satallax"]), |
50927 | 413 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
70929 | 414 |
(case getenv "E_HOME" of |
415 |
"" => "" |
|
416 |
| home => "-E " ^ home ^ "/eprover ") ^ |
|
68563 | 417 |
"-p tstp -t " ^ string_of_int (to_secs 1 timeout) ^ " " ^ file_name, |
45162 | 418 |
proof_delims = |
57707
0242e9578828
imported patch satallax_proof_support_Sledgehammer
fleury
parents:
57672
diff
changeset
|
419 |
[("% SZS output start Proof", "% SZS output end Proof")], |
45203 | 420 |
known_failures = known_szs_status_failures, |
47981 | 421 |
prem_role = Hypothesis, |
44416
cabd06b69c18
added formats to the slice and use TFF for remote Vampire
blanchet
parents:
44391
diff
changeset
|
422 |
best_slices = |
44754 | 423 |
(* FUDGE *) |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
424 |
K [(1.0, (((150, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), ""))], |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
425 |
best_max_mono_iters = default_max_mono_iters - 1 (* FUDGE *), |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
426 |
best_max_new_mono_instances = default_max_new_mono_instances} |
44099 | 427 |
|
47646 | 428 |
val satallax = (satallaxN, fn () => satallax_config) |
44099 | 429 |
|
430 |
||
431 |
(* 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
|
432 |
|
48005
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
433 |
val spass_H1SOS = "-Heuristic=1 -SOS" |
50333
20c69b00e73c
tweak SPASS default a tiny bit, so that a more interesting heuristic is chosen when "slicing=false" (for experiments)
blanchet
parents:
49991
diff
changeset
|
434 |
val spass_H2 = "-Heuristic=2" |
48005
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
435 |
val spass_H2LR0LT0 = "-Heuristic=2 -LR=0 -LT=0" |
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
436 |
val spass_H2NuVS0 = "-Heuristic=2 -RNuV=1 -Sorts=0" |
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
437 |
val spass_H2NuVS0Red2 = "-Heuristic=2 -RNuV=1 -Sorts=0 -RFRew=2 -RBRew=2 -RTaut=2" |
50333
20c69b00e73c
tweak SPASS default a tiny bit, so that a more interesting heuristic is chosen when "slicing=false" (for experiments)
blanchet
parents:
49991
diff
changeset
|
438 |
val spass_H2SOS = "-Heuristic=2 -SOS" |
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
|
439 |
|
50950 | 440 |
val spass_extra_options = |
69593 | 441 |
Attrib.setup_config_string \<^binding>\<open>atp_spass_extra_options\<close> (K "") |
50950 | 442 |
|
48005
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
443 |
val spass_config : atp_config = |
66363 | 444 |
{exec = K (["SPASS_HOME"], ["SPASS"]), |
68563 | 445 |
arguments = fn _ => fn full_proofs => fn extra_options => fn timeout => fn file_name => fn _ => |
446 |
"-Isabelle=1 " ^ (if full_proofs then "-CNFRenaming=0 -Splits=0 " else "") ^ |
|
447 |
"-TimeLimit=" ^ string_of_int (to_secs 1 timeout) ^ " " ^ file_name |
|
448 |
|> extra_options <> "" ? prefix (extra_options ^ " "), |
|
36369
d2cd0d04b8e6
handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents:
36289
diff
changeset
|
449 |
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
|
450 |
known_failures = |
53225
16235bb41881
got rid of old error -- users who install SPASS manually are responsible for any version mismatches
blanchet
parents:
52995
diff
changeset
|
451 |
[(GaveUp, "SPASS beiseite: Completion found"), |
36370
a4f601daa175
centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents:
36369
diff
changeset
|
452 |
(TimedOut, "SPASS beiseite: Ran out of time"), |
36965 | 453 |
(OutOfResources, "SPASS beiseite: Maximal number of loops exceeded"), |
37413 | 454 |
(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
|
455 |
(MalformedInput, "Free Variable"), |
44391 | 456 |
(Unprovable, "No formulae and clauses found in input file"), |
47972 | 457 |
(InternalError, "Please report this error")] @ |
458 |
known_perl_failures, |
|
47976 | 459 |
prem_role = Conjecture, |
50950 | 460 |
best_slices = fn ctxt => |
42723 | 461 |
(* FUDGE *) |
51016 | 462 |
[(0.1667, (((150, meshN), DFG Monomorphic, "mono_native", combsN, true), "")), |
463 |
(0.1667, (((500, meshN), DFG Monomorphic, "mono_native", liftingN, true), spass_H2SOS)), |
|
464 |
(0.1666, (((50, meshN), DFG Monomorphic, "mono_native", liftingN, true), spass_H2LR0LT0)), |
|
465 |
(0.1000, (((250, meshN), DFG Monomorphic, "mono_native", combsN, true), spass_H2NuVS0)), |
|
466 |
(0.1000, (((1000, mepoN), DFG Monomorphic, "mono_native", liftingN, true), spass_H1SOS)), |
|
467 |
(0.1000, (((150, meshN), DFG Monomorphic, "poly_guards??", liftingN, false), spass_H2NuVS0Red2)), |
|
468 |
(0.1000, (((300, meshN), DFG Monomorphic, "mono_native", combsN, true), spass_H2SOS)), |
|
469 |
(0.1000, (((100, meshN), DFG Monomorphic, "mono_native", combs_and_liftingN, true), spass_H2))] |
|
50950 | 470 |
|> (case Config.get ctxt spass_extra_options of |
471 |
"" => I |
|
472 |
| opts => map (apsnd (apsnd (K opts)))), |
|
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
473 |
best_max_mono_iters = default_max_mono_iters, |
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
474 |
best_max_new_mono_instances = default_max_new_mono_instances} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
475 |
|
48005
eeede26f2721
killed SPASS 3.5/3.7 FLOTTER hack -- requires users to upgrade to SPASS 3.8
blanchet
parents:
48004
diff
changeset
|
476 |
val spass = (spassN, fn () => spass_config) |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
477 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
478 |
|
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
479 |
(* Vampire *) |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
480 |
|
68563 | 481 |
fun is_vampire_noncommercial_license_accepted () = |
482 |
let |
|
69593 | 483 |
val flag = Options.default_string \<^system_option>\<open>vampire_noncommercial\<close> |
68563 | 484 |
|> String.map Char.toLower |
485 |
in |
|
486 |
if flag = "yes" then |
|
487 |
SOME true |
|
488 |
else if flag = "no" then |
|
489 |
SOME false |
|
490 |
else |
|
491 |
NONE |
|
492 |
end |
|
493 |
||
494 |
fun check_vampire_noncommercial () = |
|
495 |
(case is_vampire_noncommercial_license_accepted () of |
|
496 |
SOME true => () |
|
497 |
| SOME false => |
|
498 |
error (Pretty.string_of (Pretty.para |
|
499 |
"The Vampire prover may be used only for noncommercial applications")) |
|
500 |
| NONE => |
|
501 |
error (Pretty.string_of (Pretty.para |
|
502 |
"The Vampire prover is not activated; to activate it, set the Isabelle system option \ |
|
503 |
\\"vampire_noncommercial\" to \"yes\" (e.g. via the Isabelle/jEdit menu Plugin Options \ |
|
504 |
\/ Isabelle / General)"))) |
|
44420 | 505 |
|
68563 | 506 |
val vampire_basic_options = "--proof tptp --output_axiom_names on $VAMPIRE_EXTRA_OPTIONS" |
58084 | 507 |
|
68224 | 508 |
(* cf. p. 20 of https://www.complang.tuwien.ac.at/lkovacs/Cade23_Tutorial_Slides/Session2_Slides.pdf *) |
58084 | 509 |
val vampire_full_proof_options = |
510 |
" --forced_options splitting=off:equality_proxy=off:general_splitting=off:inequality_splitting=0:\ |
|
511 |
\naming=0" |
|
512 |
||
513 |
val remote_vampire_full_proof_command = |
|
514 |
"vampire " ^ vampire_basic_options ^ " " ^ vampire_full_proof_options ^ " -t %d %s" |
|
515 |
||
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
516 |
val vampire_config : atp_config = |
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
517 |
{exec = K (["VAMPIRE_HOME"], ["vampire"]), |
58084 | 518 |
arguments = fn _ => fn full_proofs => fn sos => fn timeout => fn file_name => fn _ => |
68563 | 519 |
(check_vampire_noncommercial (); |
520 |
vampire_basic_options ^ (if full_proofs then " " ^ vampire_full_proof_options else "") ^ |
|
521 |
" -t " ^ string_of_int (to_secs 1 timeout) ^ " --input_file " ^ file_name |
|
522 |
|> 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
|
523 |
proof_delims = |
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
524 |
[("=========== Refutation ==========", |
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
525 |
"======= End of refutation =======")] @ |
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
526 |
tstp_proof_delims, |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
527 |
known_failures = |
43050
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
42999
diff
changeset
|
528 |
[(GaveUp, "UNPROVABLE"), |
59284a13abc4
support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
blanchet
parents:
42999
diff
changeset
|
529 |
(GaveUp, "CANNOT PROVE"), |
37509
f39464d971c4
factor out TPTP format output into file of its own, to facilitate further changes
blanchet
parents:
37506
diff
changeset
|
530 |
(Unprovable, "Satisfiability detected"), |
38647
5500241da479
play with fudge factor + parse one more Vampire error
blanchet
parents:
38646
diff
changeset
|
531 |
(Unprovable, "Termination reason: Satisfiable"), |
47972 | 532 |
(Interrupted, "Aborted by signal SIGINT")] @ |
533 |
known_szs_status_failures, |
|
63116 | 534 |
prem_role = Hypothesis, |
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
|
535 |
best_slices = fn ctxt => |
42723 | 536 |
(* FUDGE *) |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
537 |
[(0.333, (((500, meshN), TFF Monomorphic, "mono_native", combs_or_liftingN, false), sosN)), |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
538 |
(0.333, (((150, meshN), TFF Monomorphic, "poly_tags??", combs_or_liftingN, false), sosN)), |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
539 |
(0.334, (((50, meshN), TFF Monomorphic, "mono_native", combs_or_liftingN, false), no_sosN))] |
58084 | 540 |
|> Config.get ctxt force_sos ? (hd #> apfst (K 1.0) #> single), |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
541 |
best_max_mono_iters = default_max_mono_iters, |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
542 |
best_max_new_mono_instances = 2 * default_max_new_mono_instances (* FUDGE *)} |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
543 |
|
47646 | 544 |
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
|
545 |
|
68563 | 546 |
|
48803
ffa31bf5c662
tone down "z3_tptp", now that Z3 (starting with 4.1) no longer supports TPTP TFF0
blanchet
parents:
48801
diff
changeset
|
547 |
(* Z3 with TPTP syntax (half experimental, half legacy) *) |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
548 |
|
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
549 |
val z3_tptp_config : atp_config = |
56378 | 550 |
{exec = K (["Z3_TPTP_HOME"], ["z3_tptp"]), |
50927 | 551 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
57261 | 552 |
"-proof -t:" ^ string_of_int (to_secs 1 timeout) ^ " -file:" ^ file_name, |
56397 | 553 |
proof_delims = [("SZS status Theorem", "")], |
45203 | 554 |
known_failures = known_szs_status_failures, |
47976 | 555 |
prem_role = Hypothesis, |
42723 | 556 |
best_slices = |
44423
f74707e12d30
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet
parents:
44422
diff
changeset
|
557 |
(* FUDGE *) |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
558 |
K [(0.5, (((250, meshN), TFF Monomorphic, "mono_native", combsN, false), "")), |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
559 |
(0.25, (((125, mepoN), TFF Monomorphic, "mono_native", combsN, false), "")), |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
560 |
(0.125, (((62, mashN), TFF Monomorphic, "mono_native", combsN, false), "")), |
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
561 |
(0.125, (((31, meshN), TFF Monomorphic, "mono_native", combsN, false), ""))], |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
562 |
best_max_mono_iters = default_max_mono_iters, |
53515
f5b678b155f6
adjusted number of generated monomorphic instances for new monomorphizer based on new evaluation (E, SPASS, Vampire)
blanchet
parents:
53225
diff
changeset
|
563 |
best_max_new_mono_instances = 2 * default_max_new_mono_instances (* FUDGE *)} |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
564 |
|
47646 | 565 |
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
|
566 |
|
44590 | 567 |
|
69717 | 568 |
(* Zipperposition *) |
569 |
||
57154 | 570 |
val zipperposition_config : atp_config = |
571 |
{exec = K (["ZIPPERPOSITION_HOME"], ["zipperposition"]), |
|
572 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
|
68563 | 573 |
"-print none -proof tstp -print-types -timeout " ^ string_of_int (to_secs 1 timeout) ^ " " ^ |
574 |
file_name, |
|
57154 | 575 |
proof_delims = tstp_proof_delims, |
576 |
known_failures = known_szs_status_failures, |
|
577 |
prem_role = Hypothesis, |
|
578 |
best_slices = fn _ => |
|
579 |
(* FUDGE *) |
|
70940
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
580 |
[(1.0, (((250, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), ""))], |
57154 | 581 |
best_max_mono_iters = default_max_mono_iters, |
582 |
best_max_new_mono_instances = default_max_new_mono_instances} |
|
583 |
||
584 |
val zipperposition = (zipperpositionN, fn () => zipperposition_config) |
|
585 |
||
586 |
||
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
587 |
(* Remote Pirate invocation *) |
44590 | 588 |
|
59577 | 589 |
val remote_pirate_config : atp_config = |
590 |
{exec = K (["ISABELLE_ATP"], ["scripts/remote_pirate"]), |
|
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
591 |
arguments = fn _ => fn _ => fn _ => fn timeout => fn file_name => fn _ => |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
592 |
string_of_int (to_secs 1 timeout) ^ " " ^ file_name, |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
593 |
proof_delims = [("Involved clauses:", "Involved clauses:")], |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
594 |
known_failures = known_szs_status_failures, |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
595 |
prem_role = #prem_role spass_config, |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
596 |
best_slices = K [(1.0, (((200, ""), DFG Polymorphic, "tc_native", combsN, true), ""))], |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
597 |
best_max_mono_iters = default_max_mono_iters, |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
598 |
best_max_new_mono_instances = default_max_new_mono_instances} |
59577 | 599 |
val remote_pirate = (remote_prefix ^ pirateN, fn () => remote_pirate_config) |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
600 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
601 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
602 |
(* Remote ATP invocation via SystemOnTPTP *) |
28596
fcd463a6b6de
tuned interfaces -- plain prover function, without thread;
wenzelm
parents:
28592
diff
changeset
|
603 |
|
49984 | 604 |
val remote_systems = Synchronized.var "atp_remote_systems" ([] : string list) |
31835 | 605 |
|
49984 | 606 |
fun get_remote_systems () = |
62519 | 607 |
Timeout.apply (seconds 10.0) (fn () => |
58084 | 608 |
(case Isabelle_System.bash_output "\"$ISABELLE_ATP/scripts/remote_atp\" -w 2>&1" of |
609 |
(output, 0) => split_lines output |
|
610 |
| (output, _) => |
|
611 |
(warning |
|
612 |
(case extract_known_atp_failure known_perl_failures output of |
|
613 |
SOME failure => string_of_atp_failure failure |
|
63692 | 614 |
| NONE => trim_line output); []))) () |
62519 | 615 |
handle Timeout.TIMEOUT _ => [] |
31835 | 616 |
|
49984 | 617 |
fun find_remote_system name [] systems = |
42537
25ceb855a18b
improve version handling -- prefer versions of ToFoF, SInE, and SNARK that are known to work
blanchet
parents:
42535
diff
changeset
|
618 |
find_first (String.isPrefix (name ^ "---")) systems |
49984 | 619 |
| find_remote_system name (version :: versions) 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
|
620 |
case find_first (String.isPrefix (name ^ "---" ^ version)) systems of |
49984 | 621 |
NONE => find_remote_system name versions 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
|
622 |
| 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
|
623 |
|
49984 | 624 |
fun get_remote_system name versions = |
625 |
Synchronized.change_result remote_systems |
|
626 |
(fn systems => (if null systems then get_remote_systems () else systems) |
|
627 |
|> `(`(find_remote_system name versions))) |
|
32864
a226f29d4bdc
re-organized signature of AtpWrapper structure: records instead of unnamed parameters and return values,
boehmes
parents:
32740
diff
changeset
|
628 |
|
49984 | 629 |
fun the_remote_system name versions = |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
630 |
(case get_remote_system name versions of |
42955 | 631 |
(SOME sys, _) => sys |
63692 | 632 |
| (NONE, []) => error "SystemOnTPTP is currently not available" |
42955 | 633 |
| (NONE, syss) => |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
634 |
(case syss |> filter_out (String.isPrefix "%") |> filter_out (curry (op =) "") of |
63692 | 635 |
[] => error "SystemOnTPTP is currently not available" |
636 |
| [msg] => error ("SystemOnTPTP is currently not available: " ^ msg) |
|
46480 | 637 |
| syss => |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
638 |
error ("System " ^ quote name ^ " is not available at SystemOnTPTP.\n(Available systems: " ^ |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
639 |
commas_quote syss ^ ".)"))) |
31835 | 640 |
|
41148 | 641 |
val max_remote_secs = 240 (* give Geoff Sutcliffe's servers a break *) |
642 |
||
58084 | 643 |
fun remote_config system_name system_versions proof_delims known_failures prem_role best_slice = |
52754
d9d90d29860e
added support for E 1.8's internal proof objects (eliminating the need for "eproof_ram")
blanchet
parents:
52151
diff
changeset
|
644 |
{exec = K (["ISABELLE_ATP"], ["scripts/remote_atp"]), |
58084 | 645 |
arguments = fn _ => fn full_proofs => fn full_proof_command => fn timeout => fn file_name => fn _ => |
646 |
(if full_proofs andalso full_proof_command <> "" then "-c " ^ quote full_proof_command ^ " " |
|
647 |
else "") ^ |
|
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
648 |
"-s " ^ the_remote_system system_name system_versions ^ " " ^ |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
649 |
"-t " ^ string_of_int (Int.min (max_remote_secs, to_secs 1 timeout)) ^ |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
650 |
" " ^ file_name, |
42962
3b50fdeb6cfc
started adding support for THF output (but no lambdas)
blanchet
parents:
42955
diff
changeset
|
651 |
proof_delims = union (op =) tstp_proof_delims proof_delims, |
45203 | 652 |
known_failures = known_failures @ known_perl_failures @ known_says_failures, |
47976 | 653 |
prem_role = prem_role, |
48716
1d2a12bb0640
stop distinguishing between complete and incomplete slices, since this is very fragile and has hardly any useful semantics to users
blanchet
parents:
48715
diff
changeset
|
654 |
best_slices = fn ctxt => [(1.0, best_slice ctxt)], |
47962
137883567114
lower the monomorphization thresholds for less scalable provers
blanchet
parents:
47955
diff
changeset
|
655 |
best_max_mono_iters = default_max_mono_iters, |
58084 | 656 |
best_max_new_mono_instances = default_max_new_mono_instances} : atp_config |
42443
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42332
diff
changeset
|
657 |
|
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
658 |
fun remotify_config system_name system_versions best_slice |
58084 | 659 |
({proof_delims, known_failures, prem_role, ...} : atp_config) = |
660 |
remote_config system_name system_versions proof_delims known_failures prem_role best_slice |
|
38023 | 661 |
|
58084 | 662 |
fun remote_atp name system_name system_versions proof_delims known_failures prem_role best_slice = |
663 |
(remote_prefix ^ name, fn () => |
|
664 |
remote_config system_name system_versions proof_delims known_failures prem_role best_slice) |
|
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
665 |
fun remotify_atp (name, config) system_name system_versions best_slice = |
58084 | 666 |
(remote_prefix ^ name, remotify_config system_name system_versions best_slice o config) |
28592 | 667 |
|
57269
1df6f747f164
changed type encoding for new Waldmeister, to trigger filtering of 'dangerous' lemmas
blanchet
parents:
57265
diff
changeset
|
668 |
fun gen_remote_waldmeister name type_enc = |
57265 | 669 |
remote_atp name "Waldmeister" ["710"] tstp_proof_delims |
670 |
([(OutOfResources, "Too many function symbols"), |
|
671 |
(Inappropriate, "**** Unexpected end of file."), |
|
672 |
(Crashed, "Unrecoverable Segmentation Fault")] |
|
673 |
@ known_szs_status_failures) |
|
57264 | 674 |
Hypothesis |
57269
1df6f747f164
changed type encoding for new Waldmeister, to trigger filtering of 'dangerous' lemmas
blanchet
parents:
57265
diff
changeset
|
675 |
(K (((50, ""), CNF_UEQ, type_enc, combsN, false), "") (* FUDGE *)) |
57264 | 676 |
|
52094 | 677 |
val remote_agsyhol = |
678 |
remotify_atp agsyhol "agsyHOL" ["1.0", "1"] |
|
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
679 |
(K (((60, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", keep_lamsN, false), "") (* FUDGE *)) |
70937 | 680 |
val remote_alt_ergo = |
681 |
remotify_atp alt_ergo "Alt-Ergo" ["0.95.2"] |
|
682 |
(K (((250, ""), TFF Polymorphic, "poly_native", keep_lamsN, false), "") (* FUDGE *)) |
|
43500
4c357b7aa710
provide appropriate type system and number of fact defaults for remote ATPs
blanchet
parents:
43497
diff
changeset
|
683 |
val remote_e = |
63768 | 684 |
remotify_atp e "E" ["2.0", "1.9.1", "1.8"] |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
685 |
(K (((750, ""), TFF Monomorphic, "mono_native", combsN, false), "") (* FUDGE *)) |
48700 | 686 |
val remote_iprover = |
52094 | 687 |
remotify_atp iprover "iProver" ["0.99"] |
58084 | 688 |
(K (((150, ""), FOF, "mono_guards??", liftingN, false), "") (* FUDGE *)) |
44099 | 689 |
val remote_leo2 = |
52094 | 690 |
remotify_atp leo2 "LEO-II" ["1.5.0", "1.4", "1.3", "1.2", "1"] |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
691 |
(K (((40, ""), THF (Monomorphic, THF_Without_Choice), "mono_native_higher", liftingN, false), "") (* FUDGE *)) |
67021
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
692 |
val remote_leo3 = |
41f1f8c4259b
integrated Leo-III in Sledgehammer (thanks to Alexander Steen for the patch)
blanchet
parents:
66544
diff
changeset
|
693 |
remotify_atp leo3 "Leo-III" ["1.1"] |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
694 |
(K (((150, ""), THF (Polymorphic, THF_Without_Choice), "poly_native_higher", keep_lamsN, false), "") (* FUDGE *)) |
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
695 |
val remote_snark = |
52094 | 696 |
remote_atp snarkN "SNARK" ["20120808r022", "20080805r029", "20080805r024"] |
58084 | 697 |
[("refutation.", "end_refutation.")] [] Hypothesis |
70932
a35618d00d29
updated iProver setup and tuned other ATP setups
blanchet
parents:
70931
diff
changeset
|
698 |
(K (((100, ""), TFF Monomorphic, "mono_native", liftingN, false), "") (* FUDGE *)) |
70937 | 699 |
val remote_vampire = |
700 |
remotify_atp vampire "Vampire" ["4.2", "4.1", "4.0"] |
|
701 |
(K (((400, ""), TFF Monomorphic, "mono_native", combs_or_liftingN, false), remote_vampire_full_proof_command) (* FUDGE *)) |
|
57269
1df6f747f164
changed type encoding for new Waldmeister, to trigger filtering of 'dangerous' lemmas
blanchet
parents:
57265
diff
changeset
|
702 |
val remote_waldmeister = gen_remote_waldmeister waldmeisterN "raw_mono_tags??" |
70940
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
703 |
val remote_zipperposition = |
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
704 |
remotify_atp zipperposition "Zipperpin" ["1.5"] |
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
705 |
(K (((250, ""), THF (Monomorphic, THF_Without_Choice), "poly_native_higher", keep_lamsN, false), "") (* FUDGE *)) |
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
706 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
707 |
|
38454
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
708 |
(* Setup *) |
9043eefe8d71
detect old Vampire and give a nicer error message
blanchet
parents:
38433
diff
changeset
|
709 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
710 |
fun add_atp (name, config) thy = |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
711 |
Data.map (Symtab.update_new (name, (config, stamp ()))) thy |
63692 | 712 |
handle Symtab.DUP name => error ("Duplicate ATP: " ^ quote name) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
713 |
|
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
714 |
fun get_atp thy name = |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
715 |
fst (the (Symtab.lookup (Data.get thy) name)) |
63692 | 716 |
handle Option.Option => error ("Unknown ATP: " ^ name) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
717 |
|
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41725
diff
changeset
|
718 |
val supported_atps = Symtab.keys o Data.get |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
719 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
720 |
fun is_atp_installed thy name = |
48376
416e4123baf3
use "eproof_ram" script if available (plug-in replacement for "eproof", but faster)
blanchet
parents:
48232
diff
changeset
|
721 |
let val {exec, ...} = get_atp thy name () in |
57671
dc5e1b1db9ba
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
blanchet
parents:
57636
diff
changeset
|
722 |
exists (fn var => getenv var <> "") (fst (exec false)) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
723 |
end |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36370
diff
changeset
|
724 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
725 |
fun refresh_systems_on_tptp () = |
49984 | 726 |
Synchronized.change remote_systems (fn _ => get_remote_systems ()) |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39491
diff
changeset
|
727 |
|
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
|
728 |
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
|
729 |
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
|
730 |
if ord = smartN then |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
731 |
{is_lpo = false, gen_weights = (atp = spassN), gen_prec = (atp = spassN), |
59577 | 732 |
gen_simp = String.isSuffix pirateN atp} |
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
|
733 |
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
|
734 |
let val is_lpo = String.isSubstring lpoN ord in |
54788
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
735 |
{is_lpo = is_lpo, gen_weights = not is_lpo andalso String.isSubstring xweightsN ord, |
a898e15b522a
primitive support for SPASS-Pirate (Daniel Wand's polymorphic SPASS prototype)
blanchet
parents:
54197
diff
changeset
|
736 |
gen_prec = String.isSubstring xprecN ord, gen_simp = String.isSubstring xsimpN ord} |
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
|
737 |
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
|
738 |
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
|
739 |
|
52073
ccb292952774
started adding agsyHOL as an experimental prover
blanchet
parents:
51998
diff
changeset
|
740 |
val atps = |
70939
3218999b3715
folded experimental Ehoh into E now that E 2.3 has been released
blanchet
parents:
70938
diff
changeset
|
741 |
[agsyhol, alt_ergo, e, e_par, iprover, leo2, leo3, satallax, spass, vampire, z3_tptp, |
70938 | 742 |
zipperposition, remote_agsyhol, remote_alt_ergo, remote_e, remote_iprover, remote_leo2, |
70940
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
743 |
remote_leo3, remote_pirate, remote_snark, remote_vampire, remote_waldmeister, |
ce3a05ad07b7
added support for Zipperposition on SystemOnTPTP
blanchet
parents:
70939
diff
changeset
|
744 |
remote_zipperposition] |
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
|
745 |
|
57262 | 746 |
val _ = Theory.setup (fold add_atp atps) |
35867 | 747 |
|
28592 | 748 |
end; |