src/HOL/TPTP/ATP_Theory_Export.thy
changeset 48375 48628962976b
parent 48302 6cf5e58f1185
child 48891 c0eafbd55de3
--- a/src/HOL/TPTP/ATP_Theory_Export.thy	Fri Jul 20 21:05:47 2012 +0200
+++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Fri Jul 20 22:19:45 2012 +0200
@@ -10,13 +10,13 @@
 begin
 
 ML {*
-open ATP_Problem;
-open ATP_Theory_Export;
+open ATP_Problem
+open ATP_Theory_Export
 *}
 
 ML {*
-val do_it = false; (* switch to "true" to generate the files *)
-val thy = @{theory List};
+val do_it = false (* switch to "true" to generate the files *)
+val thy = @{theory List}
 val ctxt = @{context}
 *}