src/Pure/Pure.thy
changeset 63513 9f8d06f23c09
parent 63510 0fc8be2f8176
child 63579 73939a9b70a3
--- a/src/Pure/Pure.thy	Sat Jul 16 00:11:03 2016 +0200
+++ b/src/Pure/Pure.thy	Sat Jul 16 00:38:33 2016 +0200
@@ -902,7 +902,14 @@
 val _ =
   Outer_Syntax.command @{command_keyword proof} "backward proof step"
     (Scan.option Method.parse >> (fn m =>
-      (Option.map Method.report m; Toplevel.proof (Proof.proof m #> Seq.the_result ""))));
+      (Option.map Method.report m;
+       Toplevel.proof (fn state =>
+         let
+          val state' = state |> Proof.proof m |> Seq.the_result "";
+          val _ =
+            Output.information
+              (Proof_Context.print_cases_proof (Proof.context_of state) (Proof.context_of state'));
+        in state' end))))
 
 in end\<close>