src/Pure/Isar/obtain.ML
changeset 46728 85f8e3932712
parent 46219 426ed18eba43
child 47815 43f677b3ae91
--- a/src/Pure/Isar/obtain.ML	Tue Feb 28 14:24:37 2012 +0100
+++ b/src/Pure/Isar/obtain.ML	Tue Feb 28 16:43:32 2012 +0100
@@ -299,7 +299,7 @@
 
     val goal = Var (("guess", 0), propT);
     fun print_result ctxt' (k, [(s, [_, th])]) =
-      Proof_Display.print_results int ctxt' (k, [(s, [th])]);
+      Proof_Display.print_results Isabelle_Markup.state int ctxt' (k, [(s, [th])]);
     val before_qed = SOME (Method.primitive_text (Goal.conclude #> Raw_Simplifier.norm_hhf #>
         (fn th => Goal.protect (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th))));
     fun after_qed [[_, res]] =