merged
authorwenzelm
Fri, 16 Nov 2012 18:49:46 +0100
changeset 50103 3d89c38408cd
parent 50101 a3bede207a04 (current diff)
parent 50102 5e01e32dadbe (diff)
child 50104 de19856feb54
merged
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Fri Nov 16 14:46:23 2012 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Fri Nov 16 18:49:46 2012 +0100
@@ -814,8 +814,8 @@
       end
     val sum_up_time =
       Vector.foldl
-        ((fn (SOME t, (b, s)) => (b, t + s)
-           | (NONE, (_, s)) => (true, preplay_timeout + s)) o apfst Lazy.force)
+        ((fn (SOME t, (b, s)) => (b, Time.+ (t, s))
+           | (NONE, (_, s)) => (true, Time.+ (preplay_timeout, s))) o apfst Lazy.force)
         (false, seconds 0.0)
 
     (* Metis Preplaying *)
@@ -858,7 +858,7 @@
           let
             val s12 = merge s1 s2
             val timeout =
-              t1 + t2 |> Time.toReal |> curry Real.* merge_timeout_slack
+              Time.+ (t1, t2) |> Time.toReal |> curry Real.* merge_timeout_slack
                       |> Time.fromReal
           in
             case try_metis timeout s12 () of