src/Tools/try.ML
changeset 62519 a564458f94db
parent 62505 9e2a65912111
child 63690 48a2c88091d7
--- a/src/Tools/try.ML	Sat Mar 05 13:57:25 2016 +0100
+++ b/src/Tools/try.ML	Sat Mar 05 17:01:45 2016 +0100
@@ -110,7 +110,7 @@
               val auto_time_limit = Options.default_real @{system_option auto_time_limit}
             in
               if auto_time_limit > 0.0 then
-                (case TimeLimit.timeLimit (seconds auto_time_limit) (fn () => tool true state) () of
+                (case Timeout.apply (seconds auto_time_limit) (fn () => tool true state) () of
                   (true, (_, outcome)) => List.app Output.information outcome
                 | _ => ())
               else ()