src/HOL/TPTP/ATP_Theory_Export.thy
changeset 46321 484dc68c8c89
parent 45305 3e09961326ce
child 46435 e9c90516bc0d
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Mon Jan 23 17:40:32 2012 +0100
@@ -0,0 +1,63 @@
+(*  Title:      HOL/TPTP/ATP_Theory_Export.thy
+    Author:     Jasmin Blanchette, TU Muenchen
+*)
+
+header {* ATP Theory Exporter *}
+
+theory ATP_Theory_Export
+imports Complex_Main
+uses "atp_theory_export.ML"
+begin
+
+ML {*
+open ATP_Problem;
+open ATP_Theory_Export;
+*}
+
+ML {*
+val do_it = false; (* switch to "true" to generate the files *)
+val thy = @{theory Complex_Main};
+val ctxt = @{context}
+*}
+
+ML {*
+if do_it then
+  "/tmp/axs_mono_simple.dfg"
+  |> generate_tptp_inference_file_for_theory ctxt thy (DFG DFG_Sorted)
+         "mono_simple"
+else
+  ()
+*}
+
+ML {*
+if do_it then
+  "/tmp/infs_poly_guards.tptp"
+  |> generate_tptp_inference_file_for_theory ctxt thy FOF "poly_guards"
+else
+  ()
+*}
+
+ML {*
+if do_it then
+  "/tmp/infs_poly_tags.tptp"
+  |> generate_tptp_inference_file_for_theory ctxt thy FOF "poly_tags"
+else
+  ()
+*}
+
+ML {*
+if do_it then
+  "/tmp/infs_poly_tags_uniform.tptp"
+  |> generate_tptp_inference_file_for_theory ctxt thy FOF "poly_tags_uniform"
+else
+  ()
+*}
+
+ML {*
+if do_it then
+  "/tmp/graph.out" |> generate_tptp_graph_file_for_theory ctxt thy
+else
+  ()
+*}
+
+end