src/HOL/Predicate_Compile_Examples/IMP_2.thy
changeset 42397 13798dcbdca5
parent 42031 2de57cda5b24
child 43686 bc7d63c7fd6f
--- a/src/HOL/Predicate_Compile_Examples/IMP_2.thy	Mon Apr 18 16:33:45 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/IMP_2.thy	Mon Apr 18 17:07:47 2011 +0200
@@ -29,7 +29,7 @@
 
 lemma
   "exec c s s' ==> exec (Seq c c) s s'"
-quickcheck[tester = predicate_compile_wo_ff, size = 2, iterations = 10]
+quickcheck[tester = predicate_compile_wo_ff, size = 2, iterations = 10, timeout = 600.0, expect = counterexample]
 oops