src/HOL/Library/Predicate_Compile_Quickcheck.thy
changeset 45450 dc2236b19a3d
parent 43886 bf068e758783
child 48891 c0eafbd55de3
--- a/src/HOL/Library/Predicate_Compile_Quickcheck.thy	Fri Nov 11 08:32:44 2011 +0100
+++ b/src/HOL/Library/Predicate_Compile_Quickcheck.thy	Fri Nov 11 08:32:45 2011 +0100
@@ -9,12 +9,4 @@
 
 setup {* Predicate_Compile_Quickcheck.setup *}
 
-(*setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_wo_ff", Predicate_Compile_Quickcheck.quickcheck_compile_term
-  Predicate_Compile_Aux.New_Pos_Random_DSeq false true 4)) *}
-setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_ff_fs",
-  Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true true 4)) *}
-setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_ff_nofs",
-  Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true false 4)) *}
-*)
-
 end
\ No newline at end of file