src/HOL/TPTP/ATP_Theory_Export.thy
changeset 61323 99b3a17a7eab
parent 58889 5b7a9633cfa8
child 63167 0909deb8059b
--- a/src/HOL/TPTP/ATP_Theory_Export.thy	Sun Oct 04 17:48:34 2015 +0200
+++ b/src/HOL/TPTP/ATP_Theory_Export.thy	Mon Oct 05 13:26:25 2015 +0200
@@ -18,8 +18,17 @@
 ML {*
 val do_it = false (* switch to "true" to generate the files *)
 val ctxt = @{context}
-val thy = @{theory List}
-val infer_policy = Unchecked_Inferences
+val thy = @{theory Complex_Main}
+val infer_policy = (* Unchecked_Inferences *) No_Inferences
+*}
+
+ML {*
+if do_it then
+  "/tmp/isa_filter"
+  |> generate_casc_lbt_isa_files_for_theory ctxt thy (THF (Polymorphic, THF_Without_Choice))
+         infer_policy "poly_native_higher"
+else
+  ()
 *}
 
 ML {*