src/HOL/Tools/Sledgehammer/sledgehammer_util.ML
changeset 48318 325c8fd0d762
parent 48316 252f45c04042
child 48383 df75b2d7e26a
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_util.ML	Wed Jul 18 08:44:04 2012 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_util.ML	Wed Jul 18 08:44:04 2012 +0200
@@ -9,6 +9,7 @@
   val plural_s : int -> string
   val serial_commas : string -> string list -> string list
   val simplify_spaces : string -> string
+  val time_mult : real -> Time.time -> Time.time
   val parse_bool_option : bool -> string -> string -> bool option
   val parse_time_option : string -> string -> Time.time option
   val subgoal_count : Proof.state -> int
@@ -26,6 +27,9 @@
 val serial_commas = Try.serial_commas
 val simplify_spaces = strip_spaces false (K true)
 
+fun time_mult k t =
+  Time.fromMilliseconds (Real.ceil (k * Real.fromInt (Time.toMilliseconds t)))
+
 fun parse_bool_option option name s =
   (case s of
      "smart" => if option then NONE else raise Option