| changeset 46324 | e4bccf5ec61e |
| child 47557 | 32f35b3d9e42 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/TPTP/ATP_Problem_Import.thy Mon Jan 23 17:40:32 2012 +0100 @@ -0,0 +1,16 @@ +(* Title: HOL/TPTP/ATP_Problem_Import.thy + Author: Jasmin Blanchette, TU Muenchen +*) + +header {* ATP Problem Importer *} + +theory ATP_Problem_Import +imports Complex_Main +uses ("atp_problem_import.ML") +begin + +typedecl iota (* for TPTP *) + +use "atp_problem_import.ML" + +end