src/HOL/TPTP/MaSh_Export.thy
changeset 48304 50e64af9c829
parent 48301 e5c5037a3104
child 48333 2250197977dc
--- a/src/HOL/TPTP/MaSh_Export.thy	Wed Jul 18 08:44:04 2012 +0200
+++ b/src/HOL/TPTP/MaSh_Export.thy	Wed Jul 18 08:44:04 2012 +0200
@@ -14,7 +14,6 @@
    lam_trans = combs_and_lifting, timeout = 5, dont_preplay, minimize]
 
 ML {*
-open Sledgehammer_Filter_MaSh
 open MaSh_Export
 *}
 
@@ -26,7 +25,7 @@
 
 ML {*
 if do_it then
-  generate_accessibility @{context} thy false "/tmp/mash_accessibility"
+  generate_accessibility thy false "/tmp/mash_accessibility"
 else
   ()
 *}
@@ -40,7 +39,7 @@
 
 ML {*
 if do_it then
-  generate_isa_dependencies @{context} thy false "/tmp/mash_isa_dependencies"
+  generate_isa_dependencies thy false "/tmp/mash_isa_dependencies"
 else
   ()
 *}