src/HOL/Predicate_Compile_Examples/IMP_1.thy
changeset 39249 9c866b248cb1
parent 39186 475856793715
child 40924 a9be7f26b4e6
--- a/src/HOL/Predicate_Compile_Examples/IMP_1.thy	Thu Sep 09 09:11:13 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/IMP_1.thy	Thu Sep 09 11:10:44 2010 +0200
@@ -27,7 +27,7 @@
 
 lemma
   "exec c s s' ==> exec (Seq c c) s s'"
-quickcheck[generator = predicate_compile_wo_ff, size = 2, iterations = 1, expect = counterexample]
+quickcheck[generator = predicate_compile_wo_ff, size = 2, iterations = 10, expect = counterexample]
 oops