src/HOL/TPTP/MaSh_Eval.thy
changeset 48333 2250197977dc
parent 48322 8a8d71e34297
child 48891 c0eafbd55de3
--- a/src/HOL/TPTP/MaSh_Eval.thy	Wed Jul 18 08:44:05 2012 +0200
+++ b/src/HOL/TPTP/MaSh_Eval.thy	Wed Jul 18 08:44:05 2012 +0200
@@ -5,7 +5,7 @@
 header {* MaSh Evaluation Driver *}
 
 theory MaSh_Eval
-imports (* ### Complex_Main *) "~~/src/HOL/Sledgehammer2d"
+imports Complex_Main
 uses "mash_eval.ML"
 begin
 
@@ -20,14 +20,14 @@
 *}
 
 ML {*
-val do_it = false (* switch to "true" to generate the files *);
-val thy = @{theory Nat};
+val do_it = false (* switch to "true" to generate the files *)
+val thy = @{theory Nat}
 val params = Sledgehammer_Isar.default_params @{context} []
 *}
 
 ML {*
 if do_it then
-  evaluate_mash_suggestions @{context} params thy "/Users/blanchet/tum/mash/mash/results/natNB200ATP-15.pred"
+  evaluate_mash_suggestions @{context} params thy "/tmp/mash_suggestions"
 else
   ()
 *}