src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 40924 a9be7f26b4e6
parent 39800 17e29ddd538e
child 41956 c15ef1b85035
--- 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 *}