src/HOL/Tools/sat_funcs.ML
changeset 32155 e2bf2f73b0c8
parent 32091 30e2ffbba718
child 32231 95b8afcbb0ed
--- a/src/HOL/Tools/sat_funcs.ML	Thu Jul 23 22:20:37 2009 +0200
+++ b/src/HOL/Tools/sat_funcs.ML	Thu Jul 23 23:12:21 2009 +0200
@@ -337,7 +337,7 @@
 		val _ = if !trace_sat then
 				tracing "'quick_and_dirty' is set: proof reconstruction skipped, using oracle instead."
 			else ()
-		val False_thm = SkipProof.make_thm (the_context ()) (HOLogic.Trueprop $ HOLogic.false_const)
+		val False_thm = SkipProof.make_thm @{theory} (HOLogic.Trueprop $ HOLogic.false_const)
 	in
 		(* 'fold Thm.weaken (rev sorted_clauses)' is linear, while 'fold    *)
 		(* Thm.weaken sorted_clauses' would be quadratic, since we sorted   *)
@@ -388,7 +388,7 @@
 			val msg = "SAT solver found a countermodel:\n"
 				^ (commas
 					o map (fn (term, idx) =>
-						Syntax.string_of_term_global (the_context ()) term ^ ": "
+						Syntax.string_of_term_global @{theory} term ^ ": "
 							^ (case assignment idx of NONE => "arbitrary" | SOME true => "true" | SOME false => "false")))
 					(Termtab.dest atom_table)
 		in