author | Andreas Lochbihler |
Wed, 27 Feb 2013 13:48:15 +0100 | |
changeset 51292 | 8a635bf2c86c |
parent 49985 | 5b4b0e4e5205 |
child 52470 | dedd7952a62c |
permissions | -rw-r--r-- |
46324 | 1 |
(* Title: HOL/TPTP/ATP_Problem_Import.thy |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
3 |
*) |
|
4 |
||
5 |
header {* ATP Problem Importer *} |
|
47812 | 6 |
|
46324 | 7 |
theory ATP_Problem_Import |
49985
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
blanchet
parents:
48891
diff
changeset
|
8 |
imports |
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
blanchet
parents:
48891
diff
changeset
|
9 |
Complex_Main |
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
blanchet
parents:
48891
diff
changeset
|
10 |
TPTP_Interpret |
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
blanchet
parents:
48891
diff
changeset
|
11 |
"~~/src/HOL/Library/Refute" |
46324 | 12 |
begin |
13 |
||
48891 | 14 |
ML_file "sledgehammer_tactics.ML" |
15 |
||
47765 | 16 |
ML {* Proofterm.proofs := 0 *} |
17 |
||
47670 | 18 |
declare [[show_consts]] (* for Refute *) |
47765 | 19 |
declare [[smt_oracle]] |
47670 | 20 |
|
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47790
diff
changeset
|
21 |
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
|
22 |
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
|
23 |
|
48891 | 24 |
ML_file "atp_problem_import.ML" |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47790
diff
changeset
|
25 |
|
47785 | 26 |
(* |
47794
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47790
diff
changeset
|
27 |
ML {* ATP_Problem_Import.isabelle_tptp_file @{theory} 50 |
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
blanchet
parents:
47790
diff
changeset
|
28 |
"$TPTP/Problems/PUZ/PUZ107^5.p" *} |
47785 | 29 |
*) |
30 |
||
46324 | 31 |
end |