src/HOL/TPTP/ATP_Theory_Export.thy
changeset 51646 005b7682178b
parent 51645 86e8c87e1f1b
child 51648 3e09226c3378
--- a/src/HOL/TPTP/ATP_Theory_Export.thy	Tue Apr 09 15:19:14 2013 +0200
+++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Tue Apr 09 15:19:14 2013 +0200
@@ -5,7 +5,7 @@
 header {* ATP Theory Exporter *}
 
 theory ATP_Theory_Export
-imports Complex_Main
+imports "~~/src/HOL/Sledgehammer2d"(*###*) Complex_Main
 begin
 
 ML_file "atp_theory_export.ML"
@@ -16,34 +16,25 @@
 *}
 
 ML {*
-val do_it = false (* switch to "true" to generate the files *)
-val thy = @{theory List}
+val do_it = true (* ### *)
+val thy = @{theory Orderings}
 val ctxt = @{context}
 *}
 
 ML {*
-if do_it then
-  "/tmp/axs_tc_native.dfg"
-  |> generate_atp_inference_file_for_theory ctxt thy (DFG Polymorphic)
-         "tc_native"
-else
-  ()
+"/tmp/casc_ltb_isa"
+|> generate_casc_lbt_isa_files_for_theory ctxt thy FOF Unchecked_Inferences
+        "poly_tags??"
 *}
 
+
+
+
 ML {*
-if do_it then
-  "/tmp/infs_poly_guards_query_query.tptp"
-  |> generate_atp_inference_file_for_theory ctxt thy FOF "poly_guards??"
-else
-  ()
+"/tmp/orderings.tptp"
+|> generate_atp_inference_file_for_theory ctxt thy FOF Unchecked_Inferences
+       "poly_tags??"
 *}
 
-ML {*
-if do_it then
-  "/tmp/infs_poly_tags_query_query.tptp"
-  |> generate_atp_inference_file_for_theory ctxt thy FOF "poly_tags??"
-else
-  ()
-*}
 
 end