diff -r d72ca5742f80 -r c0eafbd55de3 src/HOL/SAT.thy --- a/src/HOL/SAT.thy Wed Aug 22 22:47:16 2012 +0200 +++ b/src/HOL/SAT.thy Wed Aug 22 22:55:41 2012 +0200 @@ -9,10 +9,10 @@ theory SAT imports Refute -uses - "Tools/sat_funcs.ML" begin +ML_file "Tools/sat_funcs.ML" + ML {* structure sat = SATFunc(cnf) *} method_setup sat = {* Scan.succeed (SIMPLE_METHOD' o sat.sat_tac) *}