merged
authorwenzelm
Thu, 21 Feb 2013 16:00:48 +0100
changeset 51235 8333c10d1a6d
parent 51233 7b0c723562af (diff)
parent 51234 76c062c3323c (current diff)
child 51236 f301ad90c48b
merged
--- a/src/Pure/Isar/toplevel.ML	Thu Feb 21 15:35:09 2013 +0100
+++ b/src/Pure/Isar/toplevel.ML	Thu Feb 21 16:00:48 2013 +0100
@@ -718,9 +718,10 @@
         val (body_trs, end_tr) = split_last proof_trs;
         val finish = Context.Theory o Proof_Context.theory_of;
 
-        val timing_estimate = fold (curry Time.+ o get_timing) proof_trs Time.zeroTime;
-        val timing_order = Real.floor (Real.max (Math.log10 (Time.toReal timing_estimate), ~3.0));
-        val pri = Int.min (timing_order - 3, ~1);
+        val estimate = fold (curry Time.+ o get_timing) proof_trs Time.zeroTime;
+        val pri =
+          if estimate = Time.zeroTime then ~1
+	  else Int.min (Real.floor (Real.max (Math.log10 (Time.toReal estimate), ~3.0)) - 3, ~1);
 
         val future_proof = Proof.global_future_proof
           (fn prf =>