src/HOL/TPTP/ATP_Theory_Export.thy
changeset 49317 6cf5e58f1185
parent 49316 e5c5037a3104
child 49390 48628962976b
     1.1 --- a/src/HOL/TPTP/ATP_Theory_Export.thy	Wed Jul 18 08:44:03 2012 +0200
     1.2 +++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Wed Jul 18 08:44:03 2012 +0200
     1.3 @@ -5,7 +5,7 @@
     1.4  header {* ATP Theory Exporter *}
     1.5  
     1.6  theory ATP_Theory_Export
     1.7 -imports (* ### Complex_Main *) "~~/src/HOL/Sledgehammer2d"
     1.8 +imports Complex_Main
     1.9  uses "atp_theory_export.ML"
    1.10  begin
    1.11  
    1.12 @@ -15,7 +15,7 @@
    1.13  *}
    1.14  
    1.15  ML {*
    1.16 -val do_it = true; (* switch to "true" to generate the files *)
    1.17 +val do_it = false; (* switch to "true" to generate the files *)
    1.18  val thy = @{theory List};
    1.19  val ctxt = @{context}
    1.20  *}