src/HOL/Quickcheck.thy
changeset 33254 d0c00b81db1d
parent 33250 5c2af18a3237
child 33562 b1e2830ee31a
equal deleted inserted replaced
33253:d9ca0c3bf680 33254:d0c00b81db1d
   175   for this reason we use a distinguished target @{text Quickcheck}
   175   for this reason we use a distinguished target @{text Quickcheck}
   176   not spoiling the regular trusted code generation *}
   176   not spoiling the regular trusted code generation *}
   177 
   177 
   178 code_reserved Quickcheck Quickcheck_Generators
   178 code_reserved Quickcheck Quickcheck_Generators
   179 
   179 
   180 
   180 hide (open) fact empty_def single_def bind_def union_def if_randompred_def not_randompred_def Random_def map_def
   181 hide (open) type randompred
   181 hide (open) type randompred
   182 hide (open) const random collapse beyond random_fun_aux random_fun_lift
   182 hide (open) const random collapse beyond random_fun_aux random_fun_lift
   183   empty single bind union if_randompred not_randompred Random map
   183   empty single bind union if_randompred not_randompred Random map
   184 
   184 
   185 no_notation fcomp (infixl "o>" 60)
   185 no_notation fcomp (infixl "o>" 60)