src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy
changeset 41231 2e901158675e
parent 40924 a9be7f26b4e6
child 41413 64cd30d6b0b8
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy	Fri Dec 17 08:37:35 2010 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy	Fri Dec 17 12:14:18 2010 +0100
@@ -50,7 +50,7 @@
 
 lemma
   "hotel s ==> feels_safe s r ==> g \<in> isin s r ==> owns s r = Some g"
-quickcheck[tester = small_generators_depth_14, finite_types = false, iterations = 1, size = 1, timeout = 60.0, expect = no_counterexample, timeout = 60]
+(*quickcheck[tester = small_generators_depth_14, finite_types = false, iterations = 1, size = 1, timeout = 60.0, expect = no_counterexample, timeout = 60]*)
 quickcheck[tester = small_generators_depth_15, finite_types = false, iterations = 1, size = 1, timeout = 60.0, expect = counterexample, timeout = 60]
 oops