src/HOL/TPTP/ATP_Theory_Export.thy
changeset 48302 6cf5e58f1185
parent 48301 e5c5037a3104
child 48375 48628962976b
--- a/src/HOL/TPTP/ATP_Theory_Export.thy	Wed Jul 18 08:44:03 2012 +0200
+++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Wed Jul 18 08:44:03 2012 +0200
@@ -5,7 +5,7 @@
 header {* ATP Theory Exporter *}
 
 theory ATP_Theory_Export
-imports (* ### Complex_Main *) "~~/src/HOL/Sledgehammer2d"
+imports Complex_Main
 uses "atp_theory_export.ML"
 begin
 
@@ -15,7 +15,7 @@
 *}
 
 ML {*
-val do_it = true; (* switch to "true" to generate the files *)
+val do_it = false; (* switch to "true" to generate the files *)
 val thy = @{theory List};
 val ctxt = @{context}
 *}