src/HOL/Mutabelle/MutabelleExtra.thy
changeset 40931 061b8257ab9f
parent 40653 d921c97bdbd8
child 43018 121aa59b4d17
--- a/src/HOL/Mutabelle/MutabelleExtra.thy	Fri Dec 03 08:40:47 2010 +0100
+++ b/src/HOL/Mutabelle/MutabelleExtra.thy	Fri Dec 03 09:55:45 2010 +0100
@@ -26,7 +26,7 @@
 nitpick_params [timeout = 5, sat_solver = MiniSat, no_overlord, verbose, card = 1-5, iter = 1,2,4,8,12]
 refute_params [maxtime = 10, minsize = 1, maxsize = 5, satsolver = jerusat]
 *)
-ML {* Auto_Tools.time_limit := 10 *}
+ML {* Auto_Tools.time_limit := 10.0 *}
 
 ML {* val mtds = [
   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "random",