src/HOL/TPTP/TPTP_Interpret_Test.thy
changeset 62519 a564458f94db
parent 62505 9e2a65912111
child 63167 0909deb8059b
--- a/src/HOL/TPTP/TPTP_Interpret_Test.thy	Sat Mar 05 13:57:25 2016 +0100
+++ b/src/HOL/TPTP/TPTP_Interpret_Test.thy	Sat Mar 05 17:01:45 2016 +0100
@@ -35,7 +35,7 @@
 ML {*
   (*default timeout is 1 min*)
   fun interpret timeout file thy =
-    TimeLimit.timeLimit (Time.fromSeconds (if timeout = 0 then 60 else timeout))
+    Timeout.apply (Time.fromSeconds (if timeout = 0 then 60 else timeout))
      (TPTP_Interpret.interpret_file
        false
        [Path.explode "$TPTP"]