src/HOL/ex/RPred.thy
changeset 42463 f270e3e18be5
parent 36176 3fe7e97ccca8
child 44845 5e51075cbd97
equal deleted inserted replaced
42462:0fd80c27fdf5 42463:f270e3e18be5
     1 theory RPred
     1 theory RPred
     2 imports Quickcheck Random Predicate
     2 imports Quickcheck Random Predicate
     3 begin
     3 begin
     4 
     4 
     5 types 'a "rpred" = "Random.seed \<Rightarrow> ('a Predicate.pred \<times> Random.seed)"
     5 type_synonym 'a "rpred" = "Random.seed \<Rightarrow> ('a Predicate.pred \<times> Random.seed)"
     6 
     6 
     7 section {* The RandomPred Monad *}
     7 section {* The RandomPred Monad *}
     8 
     8 
     9 text {* A monad to combine the random state monad and the predicate monad *}
     9 text {* A monad to combine the random state monad and the predicate monad *}
    10 
    10