author | blanchet |
Fri, 27 Apr 2012 12:16:10 +0200 | |
changeset 47785 | d27bb852c430 |
parent 47770 | 53e30966b4b6 |
child 47788 | 44b33c1e702e |
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 *} |
|
6 |
||
7 |
theory ATP_Problem_Import |
|
47557
32f35b3d9e42
started integrating Nik's parser into TPTP command-line tools
blanchet
parents:
46324
diff
changeset
|
8 |
imports Complex_Main TPTP_Interpret |
47766
9f7cdd5fff7c
more work on TPTP Isabelle and Sledgehammer tactics
blanchet
parents:
47765
diff
changeset
|
9 |
uses "~~/src/HOL/ex/sledgehammer_tactics.ML" |
47770 | 10 |
"atp_problem_import.ML" |
46324 | 11 |
begin |
12 |
||
47765 | 13 |
ML {* Proofterm.proofs := 0 *} |
14 |
||
47670 | 15 |
declare [[show_consts]] (* for Refute *) |
47765 | 16 |
declare [[smt_oracle]] |
47670 | 17 |
|
47785 | 18 |
(* |
19 |
ML {* ATP_Problem_Import.isabelle_tptp_file 100 "$TPTP/Problems/PUZ/PUZ107^5.p" *} |
|
20 |
*) |
|
21 |
||
46324 | 22 |
end |