src/HOL/SAT.thy
changeset 32232 6c394343360f
parent 30549 d2d7874648bd
child 34120 f9920a3ddf50
--- a/src/HOL/SAT.thy	Mon Jul 27 20:45:40 2009 +0200
+++ b/src/HOL/SAT.thy	Mon Jul 27 23:17:40 2009 +0200
@@ -25,12 +25,12 @@
   maxtime=60,
   satsolver="auto"]
 
-ML {* structure sat = SATFunc(structure cnf = cnf); *}
+ML {* structure sat = SATFunc(cnf) *}
 
-method_setup sat = {* Scan.succeed (K (SIMPLE_METHOD' sat.sat_tac)) *}
+method_setup sat = {* Scan.succeed (SIMPLE_METHOD' o sat.sat_tac) *}
   "SAT solver"
 
-method_setup satx = {* Scan.succeed (K (SIMPLE_METHOD' sat.satx_tac)) *}
+method_setup satx = {* Scan.succeed (SIMPLE_METHOD' o sat.satx_tac) *}
   "SAT solver (with definitional CNF)"
 
 end