src/Tools/try.ML
changeset 52651 5adb5c69af97
parent 52648 b1ae4306f29f
child 52652 ebdbd5c79a13
--- a/src/Tools/try.ML	Sat Jul 13 18:13:09 2013 +0200
+++ b/src/Tools/try.ML	Sat Jul 13 18:33:33 2013 +0200
@@ -119,18 +119,22 @@
   Command.print_function name
     (fn {command_name} =>
       if Keyword.is_theory_goal command_name andalso Options.default_bool auto then
-        SOME {pri = ~ weight, persistent = true, print_fn = fn _ => fn st =>
-          let
-            val state = Toplevel.proof_of st
-            val auto_time_limit = Options.default_real @{option auto_time_limit}
-          in
-            if auto_time_limit > 0.0 then
-              (case TimeLimit.timeLimit (seconds auto_time_limit) (fn () => tool true state) () of
-                (true, (_, state')) =>
-                  List.app Pretty.writeln (Proof.pretty_goal_messages state')
-              | _ => ())
-            else ()
-          end handle exn => if Exn.is_interrupt exn then reraise exn else ()}
+        SOME
+         {delay = seconds (Options.default_real @{option auto_time_start}),
+          pri = ~ weight,
+          persistent = true,
+          print_fn = fn _ => fn st =>
+            let
+              val state = Toplevel.proof_of st
+              val auto_time_limit = Options.default_real @{option auto_time_limit}
+            in
+              if auto_time_limit > 0.0 then
+                (case TimeLimit.timeLimit (seconds auto_time_limit) (fn () => tool true state) () of
+                  (true, (_, state')) =>
+                    List.app Pretty.writeln (Proof.pretty_goal_messages state')
+                | _ => ())
+              else ()
+            end handle exn => if Exn.is_interrupt exn then reraise exn else ()}
       else NONE)