src/HOL/New_Random_Sequence.thy
changeset 42163 392fd6c4669c
parent 40049 75d9f57123d6
child 50055 94041d602ecb
--- a/src/HOL/New_Random_Sequence.thy	Wed Mar 30 11:32:51 2011 +0200
+++ b/src/HOL/New_Random_Sequence.thy	Wed Mar 30 11:32:52 2011 +0200
@@ -5,8 +5,8 @@
 imports Quickcheck New_DSequence
 begin
 
-types 'a pos_random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> 'a New_DSequence.pos_dseq"
-types 'a neg_random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> 'a New_DSequence.neg_dseq"
+type_synonym 'a pos_random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> 'a New_DSequence.pos_dseq"
+type_synonym 'a neg_random_dseq = "code_numeral \<Rightarrow> code_numeral \<Rightarrow> Random.seed \<Rightarrow> 'a New_DSequence.neg_dseq"
 
 definition pos_empty :: "'a pos_random_dseq"
 where