src/HOL/Predicate_Compile_Examples/IMP_1.thy
changeset 40924 a9be7f26b4e6
parent 39249 9c866b248cb1
child 41413 64cd30d6b0b8
--- a/src/HOL/Predicate_Compile_Examples/IMP_1.thy	Fri Dec 03 08:40:47 2010 +0100
+++ b/src/HOL/Predicate_Compile_Examples/IMP_1.thy	Fri Dec 03 08:40:47 2010 +0100
@@ -27,7 +27,7 @@
 
 lemma
   "exec c s s' ==> exec (Seq c c) s s'"
-quickcheck[generator = predicate_compile_wo_ff, size = 2, iterations = 10, expect = counterexample]
+quickcheck[tester = predicate_compile_wo_ff, size = 2, iterations = 10, expect = counterexample]
 oops