| author | blanchet |
| Tue, 24 Apr 2012 09:47:40 +0200 | |
| changeset 47714 | d6683fe037b1 |
| parent 47670 | 24babc4b1925 |
| child 47765 | 18f37b7aa6a6 |
| 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 |
| 46324 | 9 |
uses ("atp_problem_import.ML")
|
10 |
begin |
|
11 |
||
| 47670 | 12 |
declare [[show_consts]] (* for Refute *) |
13 |
||
| 46324 | 14 |
use "atp_problem_import.ML" |
15 |
||
16 |
end |