tuned whitespace;
authorwenzelm
Thu, 03 Nov 2011 23:32:31 +0100
changeset 45329 dd8208a3655a
parent 45328 e5b33eecbf6e
child 45330 93b8e30a5d1f
tuned whitespace;
src/Pure/Isar/element.ML
--- a/src/Pure/Isar/element.ML	Thu Nov 03 22:51:37 2011 +0100
+++ b/src/Pure/Isar/element.ML	Thu Nov 03 23:32:31 2011 +0100
@@ -294,9 +294,9 @@
   in proof after_qed' propss #> refine_witness #> Seq.hd end;
 
 fun proof_local cmd goal_ctxt int after_qed' propss =
-    Proof.map_context (K goal_ctxt)
-    #> Proof.local_goal (Proof_Display.print_results int) (K I) Proof_Context.bind_propp_i
-      cmd NONE after_qed' (map (pair Thm.empty_binding) propss);
+  Proof.map_context (K goal_ctxt) #>
+  Proof.local_goal (Proof_Display.print_results int) (K I) Proof_Context.bind_propp_i
+    cmd NONE after_qed' (map (pair Thm.empty_binding) propss);
 
 in