diff -r be80c93ac0a2 -r a9be7f26b4e6 src/HOL/Predicate_Compile_Examples/IMP_4.thy --- a/src/HOL/Predicate_Compile_Examples/IMP_4.thy Fri Dec 03 08:40:47 2010 +0100 +++ b/src/HOL/Predicate_Compile_Examples/IMP_4.thy Fri Dec 03 08:40:47 2010 +0100 @@ -31,7 +31,7 @@ lemma "exec c s s' ==> exec (Seq c c) s s'" nitpick (* nitpick fails here! *) - 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 end \ No newline at end of file