src/HOL/Mutabelle/MutabelleExtra.thy
changeset 43018 121aa59b4d17
parent 40931 061b8257ab9f
child 46453 9e83b7c24b05
--- a/src/HOL/Mutabelle/MutabelleExtra.thy	Fri May 27 10:30:08 2011 +0200
+++ b/src/HOL/Mutabelle/MutabelleExtra.thy	Fri May 27 10:30:08 2011 +0200
@@ -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.0 *}
+ML {* Try.auto_time_limit := 10.0 *}
 
 ML {* val mtds = [
   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "random",