src/Provers/blast.ML
changeset 42012 2c3fe3cbebae
parent 41491 a2ad5b824051
child 42364 8c674b3b8e44
--- a/src/Provers/blast.ML	Sun Mar 20 21:20:07 2011 +0100
+++ b/src/Provers/blast.ML	Sun Mar 20 21:28:11 2011 +0100
@@ -914,7 +914,7 @@
 
 fun printStats (State {ntried, nclosed, ...}) (b, start, tacs) =
   if b then
-    writeln (#message (end_timing start) ^ " for search.  Closed: "
+    writeln (Timing.message (Timing.result start) ^ " for search.  Closed: "
              ^ string_of_int (!nclosed) ^
              " tried: " ^ string_of_int (!ntried) ^
              " tactics: " ^ string_of_int (length tacs))
@@ -1256,7 +1256,7 @@
       val hyps  = strip_imp_prems skoprem
       and concl = strip_imp_concl skoprem
       fun cont (tacs,_,choices) =
-          let val start = start_timing ()
+          let val start = Timing.start ()
           in
           case Seq.pull(EVERY' (rev tacs) i st) of
               NONE => (writeln ("PROOF FAILED for depth " ^
@@ -1265,7 +1265,7 @@
                        else ();
                        backtrack choices)
             | cell => (if (!trace orelse !stats)
-                       then writeln (#message (end_timing start) ^ " for reconstruction")
+                       then writeln (Timing.message (Timing.result start) ^ " for reconstruction")
                        else ();
                        Seq.make(fn()=> cell))
           end
@@ -1273,13 +1273,13 @@
   handle PROVE     => Seq.empty
 
 (*Public version with fixed depth*)
-fun depth_tac cs lim i st = timing_depth_tac (start_timing ()) cs lim i st;
+fun depth_tac cs lim i st = timing_depth_tac (Timing.start ()) cs lim i st;
 
 val (depth_limit, setup_depth_limit) = Attrib.config_int_global "blast_depth_limit" (K 20);
 
 fun blast_tac cs i st =
     ((DEEPEN (1, Config.get_global (Thm.theory_of_thm st) depth_limit)
-        (timing_depth_tac (start_timing ()) cs) 0) i
+        (timing_depth_tac (Timing.start ()) cs) 0) i
      THEN flexflex_tac) st
     handle TRANS s =>
       ((if !trace then warning ("blast: " ^ s) else ());
@@ -1299,7 +1299,7 @@
   let
     val state as State {fullTrace = ft, ...} = initialize thy;
     val res = timeap prove
-      (state, start_timing(), cs, [initBranch ([readGoal thy s], lim)], I);
+      (state, Timing.start (), cs, [initBranch ([readGoal thy s], lim)], I);
     val _ = fullTrace := !ft;
   in res end;