author | nipkow |
Wed, 18 Sep 2013 12:16:10 +0200 | |
changeset 53689 | 705f0b728b1b |
parent 52788 | da1fdbfebd39 |
child 54434 | e275d520f49d |
permissions | -rw-r--r-- |
46324 | 1 |
(* Title: HOL/TPTP/atp_problem_import.ML |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
3 |
Copyright 2012 |
|
4 |
||
5 |
Import TPTP problems as Isabelle terms or goals. |
|
6 |
*) |
|
7 |
||
8 |
signature ATP_PROBLEM_IMPORT = |
|
9 |
sig |
|
47845 | 10 |
val read_tptp_file : |
11 |
theory -> (term -> term) -> string |
|
12 |
-> term list * (term list * term list) * Proof.context |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
13 |
val nitpick_tptp_file : theory -> int -> string -> unit |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
14 |
val refute_tptp_file : theory -> int -> string -> unit |
47845 | 15 |
val can_tac : Proof.context -> tactic -> term -> bool |
16 |
val SOLVE_TIMEOUT : int -> string -> tactic -> tactic |
|
17 |
val atp_tac : |
|
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
18 |
Proof.context -> int -> (string * string) list -> int -> string -> int |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
19 |
-> tactic |
47845 | 20 |
val smt_solver_tac : string -> Proof.context -> int -> tactic |
21 |
val freeze_problem_consts : theory -> term -> term |
|
22 |
val make_conj : term list * term list -> term list -> term |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
23 |
val sledgehammer_tptp_file : theory -> int -> string -> unit |
48083
a4148c95134d
renamed TPTP commands to agree with Sutcliffe's terminology
blanchet
parents:
48082
diff
changeset
|
24 |
val isabelle_tptp_file : theory -> int -> string -> unit |
a4148c95134d
renamed TPTP commands to agree with Sutcliffe's terminology
blanchet
parents:
48082
diff
changeset
|
25 |
val isabelle_hot_tptp_file : theory -> int -> string -> unit |
46325 | 26 |
val translate_tptp_file : string -> string -> string -> unit |
46324 | 27 |
end; |
28 |
||
29 |
structure ATP_Problem_Import : ATP_PROBLEM_IMPORT = |
|
30 |
struct |
|
31 |
||
47643
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
32 |
open ATP_Util |
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
33 |
open ATP_Problem |
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
34 |
open ATP_Proof |
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
35 |
|
47776
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
36 |
val debug = false |
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
37 |
val overlord = false |
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
38 |
|
47643
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
39 |
|
47771 | 40 |
(** TPTP parsing **) |
47643
e33c2be488fe
reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
blanchet
parents:
47565
diff
changeset
|
41 |
|
47785 | 42 |
fun read_tptp_file thy postproc file_name = |
47644 | 43 |
let |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
44 |
fun has_role role (_, role', _, _) = (role' = role) |
47785 | 45 |
fun get_prop (_, _, P, _) = |
46 |
P |> Logic.varify_global |> close_form |> postproc |
|
47644 | 47 |
val path = |
48 |
Path.explode file_name |
|
49 |
|> (fn path => |
|
50 |
path |> not (Path.is_absolute path) |
|
51 |
? Path.append (Path.explode "$PWD")) |
|
47714 | 52 |
val ((_, _, problem), thy) = |
48829
6ed588c4f963
look in current directory first before looking up includes in the TPTP directory, as required by Geoff
blanchet
parents:
48143
diff
changeset
|
53 |
TPTP_Interpret.interpret_file true [Path.dir path, Path.explode "$TPTP"] |
6ed588c4f963
look in current directory first before looking up includes in the TPTP directory, as required by Geoff
blanchet
parents:
48143
diff
changeset
|
54 |
path [] [] thy |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
55 |
val (conjs, defs_and_nondefs) = |
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
56 |
problem |> List.partition (has_role TPTP_Syntax.Role_Conjecture) |
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
57 |
||> List.partition (has_role TPTP_Syntax.Role_Definition) |
47644 | 58 |
in |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
59 |
(map get_prop conjs, pairself (map get_prop) defs_and_nondefs, |
52788 | 60 |
thy |> Proof_Context.init_global) |
47557
32f35b3d9e42
started integrating Nik's parser into TPTP command-line tools
blanchet
parents:
46325
diff
changeset
|
61 |
end |
46325 | 62 |
|
47771 | 63 |
|
46324 | 64 |
(** Nitpick (alias Nitrox) **) |
65 |
||
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
66 |
fun aptrueprop f ((t0 as @{const Trueprop}) $ t1) = t0 $ f t1 |
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
67 |
| aptrueprop f t = f t |
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
68 |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
69 |
fun nitpick_tptp_file thy timeout file_name = |
46325 | 70 |
let |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
71 |
val (conjs, (defs, nondefs), ctxt) = read_tptp_file thy I file_name |
47771 | 72 |
val thy = Proof_Context.theory_of ctxt |
47991
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
73 |
val (defs, pseudo_defs) = |
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
74 |
defs |> map (ATP_Util.abs_extensionalize_term ctxt |
49985
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
blanchet
parents:
49983
diff
changeset
|
75 |
#> aptrueprop (hol_open_form I)) |
47991
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
76 |
|> List.partition (ATP_Util.is_legitimate_tptp_def |
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
77 |
o perhaps (try HOLogic.dest_Trueprop) |
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
78 |
o ATP_Util.unextensionalize_def) |
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
blanchet
parents:
47957
diff
changeset
|
79 |
val nondefs = pseudo_defs @ nondefs |
47714 | 80 |
val state = Proof.init ctxt |
46325 | 81 |
val params = |
47557
32f35b3d9e42
started integrating Nik's parser into TPTP command-line tools
blanchet
parents:
46325
diff
changeset
|
82 |
[("card", "1\<emdash>100"), |
46325 | 83 |
("box", "false"), |
84 |
("max_threads", "1"), |
|
47791 | 85 |
("batch_size", "5"), |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
86 |
("falsify", if null conjs then "false" else "true"), |
46325 | 87 |
("verbose", "true"), |
47776
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
88 |
("debug", if debug then "true" else "false"), |
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
89 |
("overlord", if overlord then "true" else "false"), |
46325 | 90 |
("show_consts", "true"), |
47755 | 91 |
("format", "1"), |
46325 | 92 |
("max_potential", "0"), |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
93 |
("timeout", string_of_int timeout), |
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
94 |
("tac_timeout", string_of_int ((timeout + 49) div 50))] |
47714 | 95 |
|> Nitpick_Isar.default_params thy |
46325 | 96 |
val i = 1 |
97 |
val n = 1 |
|
98 |
val step = 0 |
|
99 |
val subst = [] |
|
100 |
in |
|
47715
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
blanchet
parents:
47714
diff
changeset
|
101 |
Nitpick.pick_nits_in_term state params Nitpick.TPTP i n step subst |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
102 |
defs nondefs (case conjs of conj :: _ => conj | [] => @{prop True}); |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
103 |
() |
46325 | 104 |
end |
46324 | 105 |
|
106 |
||
107 |
(** Refute **) |
|
108 |
||
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
109 |
fun refute_tptp_file thy timeout file_name = |
46325 | 110 |
let |
52031
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents:
51717
diff
changeset
|
111 |
fun print_szs_of_outcome falsify s = |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
112 |
"% SZS status " ^ |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
113 |
(if s = "genuine" then |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
114 |
if falsify then "CounterSatisfiable" else "Satisfiable" |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
115 |
else |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
116 |
"Unknown") |
47788 | 117 |
|> Output.urgent_message |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
118 |
val (conjs, (defs, nondefs), ctxt) = read_tptp_file thy I file_name |
46325 | 119 |
val params = |
47714 | 120 |
[("maxtime", string_of_int timeout), |
121 |
("maxvars", "100000")] |
|
46325 | 122 |
in |
47718
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
blanchet
parents:
47715
diff
changeset
|
123 |
Refute.refute_term ctxt params (defs @ nondefs) |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
124 |
(case conjs of conj :: _ => conj | [] => @{prop True}) |
52031
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents:
51717
diff
changeset
|
125 |
|> print_szs_of_outcome (not (null conjs)) |
46325 | 126 |
end |
46324 | 127 |
|
128 |
||
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
129 |
(** Sledgehammer and Isabelle (combination of provers) **) |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
130 |
|
47785 | 131 |
fun can_tac ctxt tactic conj = can (Goal.prove ctxt [] [] conj) (K tactic) |
47771 | 132 |
|
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
133 |
fun SOLVE_TIMEOUT seconds name tac st = |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
134 |
let |
47788 | 135 |
val _ = Output.urgent_message ("running " ^ name ^ " for " ^ |
136 |
string_of_int seconds ^ " s") |
|
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
137 |
val result = |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
138 |
TimeLimit.timeLimit (Time.fromSeconds seconds) |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
139 |
(fn () => SINGLE (SOLVE tac) st) () |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
140 |
handle TimeLimit.TimeOut => NONE |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
141 |
| ERROR _ => NONE |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
142 |
in |
47785 | 143 |
case result of |
47788 | 144 |
NONE => (Output.urgent_message ("FAILURE: " ^ name); Seq.empty) |
145 |
| SOME st' => (Output.urgent_message ("SUCCESS: " ^ name); Seq.single st') |
|
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
146 |
end |
46324 | 147 |
|
47812 | 148 |
fun nitpick_finite_oracle_tac ctxt timeout i th = |
149 |
let |
|
150 |
fun is_safe (Type (@{type_name fun}, Ts)) = forall is_safe Ts |
|
151 |
| is_safe @{typ prop} = true |
|
152 |
| is_safe @{typ bool} = true |
|
153 |
| is_safe _ = false |
|
154 |
val conj = Thm.term_of (Thm.cprem_of th i) |
|
155 |
in |
|
156 |
if exists_type (not o is_safe) conj then |
|
157 |
Seq.empty |
|
158 |
else |
|
159 |
let |
|
160 |
val thy = Proof_Context.theory_of ctxt |
|
161 |
val state = Proof.init ctxt |
|
162 |
val params = |
|
163 |
[("box", "false"), |
|
164 |
("max_threads", "1"), |
|
165 |
("verbose", "true"), |
|
166 |
("debug", if debug then "true" else "false"), |
|
167 |
("overlord", if overlord then "true" else "false"), |
|
168 |
("max_potential", "0"), |
|
169 |
("timeout", string_of_int timeout)] |
|
170 |
|> Nitpick_Isar.default_params thy |
|
171 |
val i = 1 |
|
172 |
val n = 1 |
|
173 |
val step = 0 |
|
174 |
val subst = [] |
|
175 |
val (outcome, _) = |
|
176 |
Nitpick.pick_nits_in_term state params Nitpick.Normal i n step subst |
|
177 |
[] [] conj |
|
51552
c713c9505f68
clarified Skip_Proof.cheat_tac: more standard tactic;
wenzelm
parents:
49985
diff
changeset
|
178 |
in if outcome = "none" then ALLGOALS Skip_Proof.cheat_tac th else Seq.empty end |
47812 | 179 |
end |
180 |
||
48143 | 181 |
fun atp_tac ctxt completeness override_params timeout prover = |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
182 |
let |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
183 |
val ctxt = |
48143 | 184 |
ctxt |> Config.put Sledgehammer_Provers.completish (completeness > 0) |
52071 | 185 |
fun ref_of th = (Facts.named (Thm.derivation_name th), []) |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
186 |
in |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
187 |
Sledgehammer_Tactics.sledgehammer_as_oracle_tac ctxt |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
188 |
([("debug", if debug then "true" else "false"), |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
189 |
("overlord", if overlord then "true" else "false"), |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
190 |
("provers", prover), |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
191 |
("timeout", string_of_int timeout)] @ |
48143 | 192 |
(if completeness > 0 then |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
193 |
[("type_enc", |
52071 | 194 |
if completeness = 1 then "mono_native" else "poly_tags")] |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
195 |
else |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
196 |
[]) @ |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
197 |
override_params) |
52071 | 198 |
{add = map ref_of [ext, @{thm someI}], del = [], only = true} |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
199 |
end |
47765 | 200 |
|
47832 | 201 |
fun sledgehammer_tac demo ctxt timeout i = |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
202 |
let |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
203 |
val frac = if demo then 16 else 12 |
48143 | 204 |
fun slice mult completeness prover = |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
205 |
SOLVE_TIMEOUT (mult * timeout div frac) |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
206 |
(prover ^ |
48143 | 207 |
(if completeness > 0 then "(" ^ string_of_int completeness ^ ")" |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
208 |
else "")) |
48143 | 209 |
(atp_tac ctxt completeness [] (mult * timeout div frac) prover i) |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
210 |
in |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
211 |
slice 2 0 ATP_Systems.spassN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
212 |
ORELSE slice 2 0 ATP_Systems.vampireN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
213 |
ORELSE slice 2 0 ATP_Systems.eN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
214 |
ORELSE slice 2 0 ATP_Systems.z3_tptpN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
215 |
ORELSE slice 1 1 ATP_Systems.spassN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
216 |
ORELSE slice 1 2 ATP_Systems.eN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
217 |
ORELSE slice 1 1 ATP_Systems.vampireN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
218 |
ORELSE slice 1 2 ATP_Systems.vampireN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
219 |
ORELSE |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
220 |
(if demo then |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
221 |
slice 2 0 ATP_Systems.satallaxN |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
222 |
ORELSE slice 2 0 ATP_Systems.leo2N |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
223 |
else |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
224 |
no_tac) |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
225 |
end |
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
226 |
|
47832 | 227 |
fun smt_solver_tac solver ctxt = |
228 |
let |
|
229 |
val ctxt = ctxt |> Context.proof_map (SMT_Config.select_solver solver) |
|
230 |
in SMT_Solver.smt_tac ctxt [] end |
|
231 |
||
47785 | 232 |
fun auto_etc_tac ctxt timeout i = |
47812 | 233 |
SOLVE_TIMEOUT (timeout div 20) "nitpick" |
234 |
(nitpick_finite_oracle_tac ctxt (timeout div 20) i) |
|
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
235 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "simp" |
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
51552
diff
changeset
|
236 |
(asm_full_simp_tac ctxt i) |
47788 | 237 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "blast" (blast_tac ctxt i) |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
238 |
ORELSE SOLVE_TIMEOUT (timeout div 5) "auto+spass" |
47785 | 239 |
(auto_tac ctxt |
47946
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
240 |
THEN ALLGOALS (atp_tac ctxt 0 [] (timeout div 5) ATP_Systems.spassN)) |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
241 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "fast" (fast_tac ctxt i) |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
242 |
ORELSE SOLVE_TIMEOUT (timeout div 20) "z3" (smt_solver_tac "z3" ctxt i) |
33afcfad3f8d
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
blanchet
parents:
47845
diff
changeset
|
243 |
ORELSE SOLVE_TIMEOUT (timeout div 20) "cvc3" (smt_solver_tac "cvc3" ctxt i) |
47812 | 244 |
ORELSE SOLVE_TIMEOUT (timeout div 20) "best" (best_tac ctxt i) |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
245 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "force" (force_tac ctxt i) |
47832 | 246 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "meson" (Meson.meson_tac ctxt [] i) |
47812 | 247 |
ORELSE SOLVE_TIMEOUT (timeout div 10) "fastforce" (fast_force_tac ctxt i) |
47771 | 248 |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
249 |
fun problem_const_prefix thy = Context.theory_name thy ^ Long_Name.separator |
47785 | 250 |
|
251 |
(* Isabelle's standard automatic tactics ("auto", etc.) are more eager to |
|
252 |
unfold "definitions" of free variables than of constants (cf. PUZ107^5). *) |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
253 |
fun freeze_problem_consts thy = |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
254 |
let val is_problem_const = String.isPrefix (problem_const_prefix thy) in |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
255 |
map_aterms (fn t as Const (s, T) => |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
256 |
if is_problem_const s then Free (Long_Name.base_name s, T) |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
257 |
else t |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
258 |
| t => t) |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
259 |
end |
47785 | 260 |
|
47776
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
261 |
fun make_conj (defs, nondefs) conjs = |
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
262 |
Logic.list_implies (rev defs @ rev nondefs, |
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
263 |
case conjs of conj :: _ => conj | [] => @{prop False}) |
47771 | 264 |
|
52031
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents:
51717
diff
changeset
|
265 |
fun print_szs_of_success conjs success = |
47788 | 266 |
Output.urgent_message ("% SZS status " ^ |
267 |
(if success then |
|
268 |
if null conjs then "Unsatisfiable" else "Theorem" |
|
269 |
else |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
270 |
"Unknown")) |
47765 | 271 |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
272 |
fun sledgehammer_tptp_file thy timeout file_name = |
47771 | 273 |
let |
47785 | 274 |
val (conjs, assms, ctxt) = |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
275 |
read_tptp_file thy (freeze_problem_consts thy) file_name |
47776
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
276 |
val conj = make_conj assms conjs |
47771 | 277 |
in |
47832 | 278 |
can_tac ctxt (sledgehammer_tac true ctxt timeout 1) conj |
52031
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents:
51717
diff
changeset
|
279 |
|> print_szs_of_success conjs |
47771 | 280 |
end |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
281 |
|
48083
a4148c95134d
renamed TPTP commands to agree with Sutcliffe's terminology
blanchet
parents:
48082
diff
changeset
|
282 |
fun generic_isabelle_tptp_file demo thy timeout file_name = |
47771 | 283 |
let |
47785 | 284 |
val (conjs, assms, ctxt) = |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47793
diff
changeset
|
285 |
read_tptp_file thy (freeze_problem_consts thy) file_name |
47776
024cf0f7fb6d
further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
blanchet
parents:
47771
diff
changeset
|
286 |
val conj = make_conj assms conjs |
48143 | 287 |
val (last_hope_atp, last_hope_completeness) = |
48082 | 288 |
if demo then (ATP_Systems.satallaxN, 0) else (ATP_Systems.vampireN, 2) |
47771 | 289 |
in |
47811 | 290 |
(can_tac ctxt (auto_etc_tac ctxt (timeout div 2) 1) conj orelse |
47832 | 291 |
can_tac ctxt (sledgehammer_tac demo ctxt (timeout div 2) 1) conj orelse |
48082 | 292 |
can_tac ctxt (SOLVE_TIMEOUT timeout (last_hope_atp ^ "(*)") |
48143 | 293 |
(atp_tac ctxt last_hope_completeness [] timeout last_hope_atp 1)) conj) |
52031
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
blanchet
parents:
51717
diff
changeset
|
294 |
|> print_szs_of_success conjs |
47771 | 295 |
end |
46324 | 296 |
|
48083
a4148c95134d
renamed TPTP commands to agree with Sutcliffe's terminology
blanchet
parents:
48082
diff
changeset
|
297 |
val isabelle_tptp_file = generic_isabelle_tptp_file false |
a4148c95134d
renamed TPTP commands to agree with Sutcliffe's terminology
blanchet
parents:
48082
diff
changeset
|
298 |
val isabelle_hot_tptp_file = generic_isabelle_tptp_file true |
47832 | 299 |
|
300 |
||
46324 | 301 |
(** Translator between TPTP(-like) file formats **) |
302 |
||
46325 | 303 |
fun translate_tptp_file format in_file_name out_file_name = () |
46324 | 304 |
|
305 |
end; |