src/HOL/Tools/sat.ML
changeset 56853 a265e41cc33b
parent 56851 35ff4ede3409
child 58839 ccda99401bc8
--- a/src/HOL/Tools/sat.ML	Sun May 04 19:01:36 2014 +0200
+++ b/src/HOL/Tools/sat.ML	Sun May 04 19:08:29 2014 +0200
@@ -202,7 +202,7 @@
 
 (* ------------------------------------------------------------------------- *)
 (* replay_proof: replays the resolution proof returned by the SAT solver;    *)
-(*      cf. SatSolver.proof for details of the proof format.  Updates the    *)
+(*      cf. SAT_Solver.proof for details of the proof format.  Updates the   *)
 (*      'clauses' array with derived clauses, and returns the derived clause *)
 (*      at index 'empty_id' (which should just be "False" if proof           *)
 (*      reconstruction was successful, with the used clauses as hyps).       *)
@@ -335,9 +335,9 @@
       let
         val the_solver = Config.get ctxt solver
         val _ = cond_tracing ctxt (fn () => "Invoking solver " ^ the_solver)
-      in SatSolver.invoke_solver the_solver fm end
+      in SAT_Solver.invoke_solver the_solver fm end
     of
-      SatSolver.UNSATISFIABLE (SOME (clause_table, empty_id)) =>
+      SAT_Solver.UNSATISFIABLE (SOME (clause_table, empty_id)) =>
        (cond_tracing ctxt (fn () =>
           "Proof trace from SAT solver:\n" ^
           "clauses: " ^ ML_Syntax.print_list
@@ -370,13 +370,13 @@
             (* [c_1, ..., c_n] |- False *)
             Thm.implies_elim (Thm.implies_intr cnf_cterm raw_thm) clauses_thm
           end)
-    | SatSolver.UNSATISFIABLE NONE =>
+    | SAT_Solver.UNSATISFIABLE NONE =>
         if Config.get ctxt quick_and_dirty then
          (warning "SAT solver claims the formula to be unsatisfiable, but did not provide a proof";
           make_quick_and_dirty_thm ())
         else
           raise THM ("SAT solver claims the formula to be unsatisfiable, but did not provide a proof", 0, [])
-    | SatSolver.SATISFIABLE assignment =>
+    | SAT_Solver.SATISFIABLE assignment =>
         let
           val msg =
             "SAT solver found a countermodel:\n" ^
@@ -388,7 +388,7 @@
         in
           raise THM (msg, 0, [])
         end
-    | SatSolver.UNKNOWN =>
+    | SAT_Solver.UNKNOWN =>
         raise THM ("SAT solver failed to decide the formula", 0, [])
   end;