src/HOL/Random_Sequence.thy
changeset 50055 94041d602ecb
parent 42163 392fd6c4669c
child 51126 df86080de4cb
equal deleted inserted replaced
50054:6da283e4497b 50055:94041d602ecb
     1 
     1 
     2 (* Author: Lukas Bulwahn, TU Muenchen *)
     2 (* Author: Lukas Bulwahn, TU Muenchen *)
     3 
     3 
     4 theory Random_Sequence
     4 theory Random_Sequence
     5 imports Quickcheck DSequence
     5 imports Quickcheck
     6 begin
     6 begin
     7 
     7 
     8 type_synonym 'a random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> ('a DSequence.dseq \<times> Random.seed)"
     8 type_synonym 'a random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> ('a DSequence.dseq \<times> Random.seed)"
     9 
     9 
    10 definition empty :: "'a random_dseq"
    10 definition empty :: "'a random_dseq"