src/HOL/Quickcheck.thy
changeset 35028 108662d50512
parent 34968 ceeffca32eb0
child 35880 2623b23e41fc
equal deleted inserted replaced
35027:ed7d12bcf8f8 35028:108662d50512
   162 
   162 
   163 definition union :: "'a randompred \<Rightarrow> 'a randompred \<Rightarrow> 'a randompred"
   163 definition union :: "'a randompred \<Rightarrow> 'a randompred \<Rightarrow> 'a randompred"
   164 where
   164 where
   165   "union R1 R2 = (\<lambda>s. let
   165   "union R1 R2 = (\<lambda>s. let
   166      (P1, s') = R1 s; (P2, s'') = R2 s'
   166      (P1, s') = R1 s; (P2, s'') = R2 s'
   167    in (upper_semilattice_class.sup P1 P2, s''))"
   167    in (semilattice_sup_class.sup P1 P2, s''))"
   168 
   168 
   169 definition if_randompred :: "bool \<Rightarrow> unit randompred"
   169 definition if_randompred :: "bool \<Rightarrow> unit randompred"
   170 where
   170 where
   171   "if_randompred b = (if b then single () else empty)"
   171   "if_randompred b = (if b then single () else empty)"
   172 
   172