src/HOL/New_Random_Sequence.thy
changeset 36176 3fe7e97ccca8
parent 36049 0ce5b7a5c2fd
child 40049 75d9f57123d6
equal deleted inserted replaced
36175:5cec4ca719d1 36176:3fe7e97ccca8
    89 *)
    89 *)
    90 definition neg_map :: "('a => 'b) => 'a neg_random_dseq => 'b neg_random_dseq"
    90 definition neg_map :: "('a => 'b) => 'a neg_random_dseq => 'b neg_random_dseq"
    91 where
    91 where
    92   "neg_map f P = neg_bind P (neg_single o f)"
    92   "neg_map f P = neg_bind P (neg_single o f)"
    93 (*
    93 (*
    94 hide const DSequence.empty DSequence.single DSequence.eval
    94 hide_const DSequence.empty DSequence.single DSequence.eval
    95   DSequence.map_seq DSequence.bind DSequence.union DSequence.if_seq DSequence.not_seq
    95   DSequence.map_seq DSequence.bind DSequence.union DSequence.if_seq DSequence.not_seq
    96   DSequence.map
    96   DSequence.map
    97 *)
    97 *)
    98 
    98 
    99 hide (open) const
    99 hide_const (open)
   100   pos_empty pos_single pos_bind pos_union pos_if_random_dseq pos_iterate_upto pos_not_random_dseq iter Random pos_map
   100   pos_empty pos_single pos_bind pos_union pos_if_random_dseq pos_iterate_upto pos_not_random_dseq iter Random pos_map
   101   neg_empty neg_single neg_bind neg_union neg_if_random_dseq neg_iterate_upto neg_not_random_dseq neg_map
   101   neg_empty neg_single neg_bind neg_union neg_if_random_dseq neg_iterate_upto neg_not_random_dseq neg_map
   102 hide type New_DSequence.pos_dseq New_DSequence.neg_dseq pos_random_dseq neg_random_dseq
   102 hide_type New_DSequence.pos_dseq New_DSequence.neg_dseq pos_random_dseq neg_random_dseq
   103 (* FIXME: hide facts *)
   103 (* FIXME: hide facts *)
   104 (*hide (open) fact empty_def single_def bind_def union_def if_random_dseq_def not_random_dseq_def Random.simps map_def*)
   104 (*hide_fact (open) empty_def single_def bind_def union_def if_random_dseq_def not_random_dseq_def Random.simps map_def*)
   105 
   105 
   106 end
   106 end