src/HOL/TPTP/MaSh_Export.thy
changeset 50484 8ec31bdb9d36
parent 50434 960a3429615c
child 50513 cacf3cdb3276
--- a/src/HOL/TPTP/MaSh_Export.thy	Wed Dec 12 00:14:58 2012 +0100
+++ b/src/HOL/TPTP/MaSh_Export.thy	Wed Dec 12 00:24:06 2012 +0100
@@ -52,7 +52,8 @@
 
 ML {*
 if do_it then
-  generate_isar_dependencies @{context} thys false (prefix ^ "mash_dependencies")
+  generate_isar_dependencies @{context} thys false
+      (prefix ^ "mash_dependencies")
 else
   ()
 *}
@@ -66,21 +67,24 @@
 
 ML {*
 if do_it then
-  generate_mepo_suggestions @{context} params thys 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 thys false (prefix ^ "mash_atp_dependencies")
+  generate_prover_dependencies @{context} params thys false
+      (prefix ^ "mash_prover_dependencies")
 else
   ()
 *}
 
 ML {*
 if do_it then
-  generate_atp_commands @{context} params thys (prefix ^ "mash_atp_commands")
+  generate_prover_commands @{context} params thys
+      (prefix ^ "mash_prover_commands")
 else
   ()
 *}