src/HOL/Predicate_Compile_Examples/IMP_3.thy
changeset 43686 bc7d63c7fd6f
parent 42031 2de57cda5b24
child 45451 74515e8e6046
--- a/src/HOL/Predicate_Compile_Examples/IMP_3.thy	Sun Jul 03 09:59:25 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/IMP_3.thy	Wed Jul 06 13:52:42 2011 +0200
@@ -29,8 +29,8 @@
 
 lemma
   "exec c s s' ==> exec (Seq c c) s s'"
-  quickcheck[tester = predicate_compile_ff_nofs, size=2, iterations=10, quiet = false, expect = counterexample]
+  quickcheck[tester = predicate_compile_ff_nofs, size=2, iterations=100, quiet = false, expect = counterexample]
 oops
 
 
-end
\ No newline at end of file
+end