src/Pure/Isar/toplevel.ML
changeset 69882 a9e574e2cba5
parent 69878 ccc8e4c99520
child 69883 f8293bf510a0
--- a/src/Pure/Isar/toplevel.ML	Fri Mar 08 18:56:48 2019 +0000
+++ b/src/Pure/Isar/toplevel.ML	Sat Mar 09 10:31:20 2019 +0100
@@ -480,10 +480,10 @@
 
 local
 
-fun begin_proof init = transaction0 (fn int =>
+fun begin_proof init_proof = transaction0 (fn int =>
   (fn Theory gthy =>
     let
-      val (finish, prf) = init int gthy;
+      val (finish, prf) = init_proof int gthy;
       val document = Options.default_string "document";
       val skip = (document = "" orelse document = "false") andalso Goal.skip_proofs_enabled ();
       val schematic_goal = try Proof.schematic_goal prf;