src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 43937 768c70befd59
parent 41956 c15ef1b85035
child 52666 391913d17d15
--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Wed Jul 20 23:47:27 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Thu Jul 21 08:31:35 2011 +0200
@@ -79,7 +79,7 @@
 
 section {* Manual setup to find counterexample *}
 
-setup {* Context.theory_map (Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck)) *}
+setup {* Context.theory_map (Quickcheck.add_tester ("prolog", (Code_Prolog.active, Code_Prolog.test_goals))) *}
 
 setup {* Code_Prolog.map_code_options (K 
   { ensure_groundness = true,