src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 36142 f5e15e9aae10
parent 36141 c31602d268be
child 36143 6490319b1703
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Wed Apr 14 17:10:16 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Wed Apr 14 18:23:51 2010 +0200
@@ -100,7 +100,10 @@
   |> fold (AList.default (op =))
           [("atps", [!atps]),
            ("full_types", [if !full_types then "true" else "false"]),
-           ("timeout", [string_of_int (!timeout) ^ " s"])]
+           ("timeout", let val timeout = !timeout in
+                         [if timeout <= 0 then "none"
+                          else string_of_int timeout ^ " s"]
+                       end)]
 
 val infinity_time_in_secs = 60 * 60 * 24 * 365
 val the_timeout = the_default (Time.fromSeconds infinity_time_in_secs)
@@ -181,7 +184,7 @@
       get_params thy
           [("atps", [atp]),
            ("minimize_timeout",
-            [string_of_int (Time.toSeconds timeout) ^ " s"])]
+            [string_of_int (Time.toMilliseconds timeout) ^ " ms"])]
     val prover =
       (case get_prover thy atp of
         SOME prover => prover