src/HOL/Library/Predicate_Compile_Quickcheck.thy
changeset 43886 bf068e758783
parent 39252 8f176e575a49
child 45450 dc2236b19a3d
--- a/src/HOL/Library/Predicate_Compile_Quickcheck.thy	Mon Jul 18 10:34:21 2011 +0200
+++ b/src/HOL/Library/Predicate_Compile_Quickcheck.thy	Mon Jul 18 10:34:21 2011 +0200
@@ -7,11 +7,14 @@
 uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
 begin
 
-setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_wo_ff", Predicate_Compile_Quickcheck.quickcheck_compile_term
+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