| author | wenzelm | 
| Tue, 30 Jul 2019 11:41:39 +0200 | |
| changeset 70443 | a21a96eda033 | 
| parent 69605 | a96320074298 | 
| child 72001 | 3e08311ada8e | 
| permissions | -rw-r--r-- | 
| 46324 | 1  | 
(* Title: HOL/TPTP/ATP_Problem_Import.thy  | 
2  | 
Author: Jasmin Blanchette, TU Muenchen  | 
|
3  | 
*)  | 
|
4  | 
||
| 63167 | 5  | 
section \<open>ATP Problem Importer\<close>  | 
| 47812 | 6  | 
|
| 46324 | 7  | 
theory ATP_Problem_Import  | 
| 
66453
 
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
 
wenzelm 
parents: 
64561 
diff
changeset
 | 
8  | 
imports Complex_Main TPTP_Interpret "HOL-Library.Refute"  | 
| 46324 | 9  | 
begin  | 
10  | 
||
| 69605 | 11  | 
ML_file \<open>sledgehammer_tactics.ML\<close>  | 
| 48891 | 12  | 
|
| 63167 | 13  | 
ML \<open>Proofterm.proofs := 0\<close>  | 
| 47765 | 14  | 
|
| 47670 | 15  | 
declare [[show_consts]] (* for Refute *)  | 
| 47765 | 16  | 
declare [[smt_oracle]]  | 
| 47670 | 17  | 
|
| 
47794
 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 
blanchet 
parents: 
47790 
diff
changeset
 | 
18  | 
declare [[unify_search_bound = 60]]  | 
| 
 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 
blanchet 
parents: 
47790 
diff
changeset
 | 
19  | 
declare [[unify_trace_bound = 60]]  | 
| 
 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 
blanchet 
parents: 
47790 
diff
changeset
 | 
20  | 
|
| 69605 | 21  | 
ML_file \<open>atp_problem_import.ML\<close>  | 
| 
47794
 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 
blanchet 
parents: 
47790 
diff
changeset
 | 
22  | 
|
| 47785 | 23  | 
(*  | 
| 
57812
 
8dc9dc241973
make TPTP tools work on polymorphic (TFF1) problems as well
 
blanchet 
parents: 
52487 
diff
changeset
 | 
24  | 
ML {* ATP_Problem_Import.isabelle_tptp_file @{theory} 50 "$TPTP/Problems/PUZ/PUZ107^5.p" *}
 | 
| 64561 | 25  | 
ML {* ATP_Problem_Import.isabelle_hot_tptp_file @{theory} 20 "$TPTP/Problems/SYO/SYO304^5.p" *}
 | 
| 47785 | 26  | 
*)  | 
27  | 
||
| 46324 | 28  | 
end  |