highest priority for proofs with unknown / very short timing -- recover original scheduling with parallel_proofs_reuse_timing = false;
--- a/src/Pure/Isar/toplevel.ML Wed Feb 20 19:57:17 2013 +0100
+++ b/src/Pure/Isar/toplevel.ML Thu Feb 21 10:52:14 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 =>