src/HOL/TPTP/MaSh_Export.thy
changeset 50349 b79803ee14f3
parent 50337 68555697f37e
child 50350 136d5318b1fe
--- a/src/HOL/TPTP/MaSh_Export.thy	Tue Dec 04 18:00:40 2012 +0100
+++ b/src/HOL/TPTP/MaSh_Export.thy	Tue Dec 04 18:12:29 2012 +0100
@@ -30,10 +30,11 @@
 
 ML {*
 val do_it = false (* switch to "true" to generate the files *)
-val thy = @{theory List}
+val thys = [@{theory Main}] (* [@{theory Fundamental_Theorem_Algebra}] *)
 val params as {provers, ...} = Sledgehammer_Isar.default_params @{context} []
 val prover = hd provers
-val prefix = "/tmp/" ^ Context.theory_name thy ^ "/"
+val dir = space_implode "__" (map Context.theory_name thys)
+val prefix = "/tmp/" ^ dir ^ "/"
 *}
 
 ML {*
@@ -42,42 +43,42 @@
 
 ML {*
 if do_it then
-  generate_accessibility @{context} thy false (prefix ^ "mash_accessibility")
+  generate_accessibility @{context} thys false (prefix ^ "mash_accessibility")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_features @{context} prover thy false (prefix ^ "mash_features")
+  generate_features @{context} prover thys false (prefix ^ "mash_features")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_isar_dependencies @{context} thy false (prefix ^ "mash_dependencies")
+  generate_isar_dependencies @{context} thys false (prefix ^ "mash_dependencies")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_commands @{context} params thy (prefix ^ "mash_commands")
+  generate_commands @{context} params thys (prefix ^ "mash_commands")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_mepo_suggestions @{context} params thy 1024 (prefix ^ "mash_mepo_suggestions")
+  generate_mepo_suggestions @{context} params thys 1024 (prefix ^ "mash_mepo_suggestions")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_atp_dependencies @{context} params thy false (prefix ^ "mash_atp_dependencies")
+  generate_atp_dependencies @{context} params thys false (prefix ^ "mash_atp_dependencies")
 else
   ()
 *}