src/HOL/ex/SAT_Examples.thy
changeset 21588 cd0dc678a205
parent 21422 25ed0a4c7dc5
child 22054 4cb2fe751952
--- a/src/HOL/ex/SAT_Examples.thy	Wed Nov 29 15:44:46 2006 +0100
+++ b/src/HOL/ex/SAT_Examples.thy	Wed Nov 29 15:44:51 2006 +0100
@@ -82,7 +82,7 @@
 ML {* reset sat.trace_sat; *}
 ML {* reset quick_and_dirty; *}
 
-method_setup rawsat = {* Method.no_args (Method.SIMPLE_METHOD (sat.rawsat_tac 1)) *}
+method_setup rawsat = {* Method.no_args (Method.SIMPLE_METHOD' sat.rawsat_tac) *}
   "SAT solver (no preprocessing)"
 
 (* ML {* Toplevel.profiling := 1; *} *)