| author | bulwahn |
| Thu, 29 Mar 2012 17:40:44 +0200 | |
| changeset 47197 | ed681ca1188a |
| parent 46324 | e4bccf5ec61e |
| child 47557 | 32f35b3d9e42 |
| 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 |
|
8 |
imports Complex_Main |
|
9 |
uses ("atp_problem_import.ML")
|
|
10 |
begin |
|
11 |
||
12 |
typedecl iota (* for TPTP *) |
|
13 |
||
14 |
use "atp_problem_import.ML" |
|
15 |
||
16 |
end |