src/HOL/Tools/Sledgehammer/sledgehammer_util.ML
changeset 36170 0cdb76723c88
parent 36169 27b1cc58715e
child 36183 f723348b2231
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_util.ML	Fri Apr 16 14:48:34 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_util.ML	Fri Apr 16 15:49:13 2010 +0200
@@ -10,13 +10,14 @@
   val serial_commas : string -> string list -> string list
   val replace_all : string -> string -> string -> string
   val remove_all : string -> string -> string
+  val timestamp : unit -> string
   val parse_bool_option : bool -> string -> string -> bool option
   val parse_time_option : string -> string -> Time.time option
   val hashw : word * word -> word
   val hashw_char : Char.char * word -> word
   val hashw_string : string * word -> word
 end;
-
+ 
 structure Sledgehammer_Util : SLEDGEHAMMER_UTIL =
 struct
 
@@ -40,6 +41,8 @@
 
 fun remove_all bef = replace_all bef ""
 
+val timestamp = Date.fmt "%Y-%m-%d %H:%M:%S" o Date.fromTimeLocal o Time.now
+
 fun parse_bool_option option name s =
   (case s of
      "smart" => if option then NONE else raise Option