--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Fri Dec 03 08:40:47 2010 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Fri Dec 03 08:40:47 2010 +0100
@@ -92,7 +92,7 @@
lemma
"\<Gamma> \<turnstile> t : U \<Longrightarrow> t \<rightarrow>\<^sub>\<beta> t' \<Longrightarrow> \<Gamma> \<turnstile> t' : U"
-quickcheck[generator = prolog, iterations = 1, expect = counterexample]
+quickcheck[tester = prolog, iterations = 1, expect = counterexample]
oops
text {* Verifying that the found counterexample really is one by means of a proof *}