src/HOL/TPTP/TPTP_Interpret.thy
changeset 48891 c0eafbd55de3
parent 47519 9c3acd90063a
child 57796 07521fed6071
--- a/src/HOL/TPTP/TPTP_Interpret.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/TPTP/TPTP_Interpret.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -8,9 +8,10 @@
 theory TPTP_Interpret
 imports Main TPTP_Parser
 keywords "import_tptp" :: thy_decl
-uses  ("TPTP_Parser/tptp_interpret.ML")
+begin
+
+typedecl "ind"
 
-begin
-typedecl "ind"
-use  "TPTP_Parser/tptp_interpret.ML"
+ML_file  "TPTP_Parser/tptp_interpret.ML"
+
 end
\ No newline at end of file