src/HOL/TPTP/MaSh_Eval.thy
changeset 50358 b7d3319409b7
parent 48891 c0eafbd55de3
child 50402 923f1e199f4f
--- a/src/HOL/TPTP/MaSh_Eval.thy	Tue Dec 04 23:43:24 2012 +0100
+++ b/src/HOL/TPTP/MaSh_Eval.thy	Tue Dec 04 23:50:36 2012 +0100
@@ -11,8 +11,8 @@
 ML_file "mash_eval.ML"
 
 sledgehammer_params
-  [provers = e, max_relevant = 40, strict, dont_slice, type_enc = poly_guards??,
-   lam_trans = combs_and_lifting, timeout = 5, dont_preplay, minimize]
+  [provers = spass, max_relevant = 40, strict, dont_slice, type_enc = mono_native,
+   lam_trans = combs_and_lifting, timeout = 15, dont_preplay, minimize]
 
 declare [[sledgehammer_instantiate_inducts]]
 
@@ -22,13 +22,12 @@
 
 ML {*
 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 "/tmp/mash_suggestions"
+  evaluate_mash_suggestions @{context} params "/tmp/mash_suggestions"
 else
   ()
 *}