src/HOL/Tools/Sledgehammer/sledgehammer_try0.ML
changeset 54765 b05b0ea06306
parent 54764 1c9ef5c834e8
child 54766 6ac273f176cd
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_try0.ML	Mon Dec 16 09:48:26 2013 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_try0.ML	Mon Dec 16 12:02:28 2013 +0100
@@ -21,7 +21,9 @@
 open Sledgehammer_Proof
 open Sledgehammer_Preplay
 
-val variant_methods = [SimpM, AutoM, ArithM, FastforceM, BlastM, ForceM, MetisM, MesonM]
+val variant_methods =
+  [Simp_Method, Auto_Method, Arith_Method, Fastforce_Method, Blast_Method, Force_Method,
+   Metis_Method, Meson_Method]
 
 fun variants_of_step (Let _) = raise Fail "Sledgehammer_Try0: variants_of_step"
   | variants_of_step (Prove (qs, xs, l, t, subproofs, (facts, meth))) =