tuned;
authorwenzelm
Tue, 28 Oct 2014 09:20:07 +0100
changeset 58795 492b64eccd10
parent 58794 e1a6a71b741d
child 58796 cc5a9a54d340
tuned;
src/Pure/Isar/toplevel.ML
--- a/src/Pure/Isar/toplevel.ML	Mon Oct 27 20:31:51 2014 +0100
+++ b/src/Pure/Isar/toplevel.ML	Tue Oct 28 09:20:07 2014 +0100
@@ -473,14 +473,13 @@
     let
       val (finish, prf) = init int gthy;
       val skip = Goal.skip_proofs_enabled ();
-      val (is_goal, no_skip) =
-        (true, Proof.schematic_goal prf) handle ERROR _ => (false, true);
+      val schematic_goal = try Proof.schematic_goal prf;
       val _ =
-        if is_goal andalso skip andalso no_skip then
+        if skip andalso schematic_goal = SOME true then
           warning "Cannot skip proof of schematic goal statement"
         else ();
     in
-      if skip andalso not no_skip then
+      if skip andalso schematic_goal = SOME false then
         Skipped_Proof (0, (finish (Proof.global_skip_proof true prf), gthy))
       else Proof (Proof_Node.init prf, (finish, gthy))
     end