src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 43953 3b69f057ef2e
parent 41956 c15ef1b85035
child 43974 30f4d346b204
--- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy	Sat Jul 23 17:22:28 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy	Sat Jul 23 20:05:28 2011 +0200
@@ -98,7 +98,7 @@
 oops
 
 
-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,