src/HOL/Mutabelle/MutabelleExtra.thy
changeset 43018 121aa59b4d17
parent 40931 061b8257ab9f
child 46453 9e83b7c24b05
equal deleted inserted replaced
43017:944b19ab6003 43018:121aa59b4d17
    24 
    24 
    25 (*
    25 (*
    26 nitpick_params [timeout = 5, sat_solver = MiniSat, no_overlord, verbose, card = 1-5, iter = 1,2,4,8,12]
    26 nitpick_params [timeout = 5, sat_solver = MiniSat, no_overlord, verbose, card = 1-5, iter = 1,2,4,8,12]
    27 refute_params [maxtime = 10, minsize = 1, maxsize = 5, satsolver = jerusat]
    27 refute_params [maxtime = 10, minsize = 1, maxsize = 5, satsolver = jerusat]
    28 *)
    28 *)
    29 ML {* Auto_Tools.time_limit := 10.0 *}
    29 ML {* Try.auto_time_limit := 10.0 *}
    30 
    30 
    31 ML {* val mtds = [
    31 ML {* val mtds = [
    32   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "random",
    32   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "random",
    33   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types true) "random",
    33   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types true) "random",
    34   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "small",
    34   MutabelleExtra.quickcheck_mtd (Config.put Quickcheck.finite_types false) "small",