src/HOL/Quickcheck.thy
changeset 33583 b5e0909cd5ea
parent 33562 b1e2830ee31a
child 34968 ceeffca32eb0
--- a/src/HOL/Quickcheck.thy	Tue Nov 10 13:17:50 2009 +0100
+++ b/src/HOL/Quickcheck.thy	Tue Nov 10 13:54:00 2009 +0100
@@ -126,6 +126,8 @@
   shows "random_aux k = rhs k"
   using assms by (rule code_numeral.induct)
 
+setup {* Quickcheck.setup *}
+
 subsection {* the Random-Predicate Monad *} 
 
 types 'a randompred = "Random.seed \<Rightarrow> ('a Predicate.pred \<times> Random.seed)"