src/HOL/Predicate_Compile_Examples/List_Examples.thy
changeset 43937 768c70befd59
parent 41956 c15ef1b85035
child 45451 74515e8e6046
--- a/src/HOL/Predicate_Compile_Examples/List_Examples.thy	Wed Jul 20 23:47:27 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/List_Examples.thy	Thu Jul 21 08:31:35 2011 +0200
@@ -5,7 +5,7 @@
   "~~/src/HOL/Library/Code_Prolog"
 begin
 
-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,