diff -r 0869ce2006eb -r 13798dcbdca5 src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy --- a/src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy Mon Apr 18 16:33:45 2011 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy Mon Apr 18 17:07:47 2011 +0200 @@ -51,7 +51,7 @@ lemma "hotel s ==> feels_safe s r ==> g \ isin s r ==> owns s r = Some g" (*quickcheck[tester = small_generators_depth_14, finite_types = false, iterations = 1, size = 1, timeout = 1200.0, expect = no_counterexample]*) -quickcheck[tester = small_generators_depth_15, finite_types = false, iterations = 1, size = 1, timeout = 1200.0, expect = counterexample] +quickcheck[tester = small_generators_depth_15, finite_types = false, iterations = 1, size = 1, timeout = 2400.0, expect = counterexample] oops