src/HOL/ex/Random.thy
changeset 26042 e7a421d1f5c1
parent 26038 55a02586776d
child 26142 3d5df9a56537
--- a/src/HOL/ex/Random.thy	Wed Feb 06 08:34:32 2008 +0100
+++ b/src/HOL/ex/Random.thy	Wed Feb 06 08:34:51 2008 +0100
@@ -195,8 +195,8 @@
 
 subsection {* The @{text random} class *}
 
-class random = type +
-  fixes random :: "index \<Rightarrow> seed \<Rightarrow> 'a \<times> seed"
+class random =
+  fixes random :: "index \<Rightarrow> seed \<Rightarrow> 'a\<Colon>{} \<times> seed"
 
 -- {* FIXME dummy implementations *}
 
@@ -230,7 +230,7 @@
 
 end
 
-instantiation "+" :: (random, random) random
+instantiation "+" :: ("{type, random}", "{type, random}") random
 begin
 
 definition
@@ -250,7 +250,7 @@
 
 end
 
-instantiation "*" :: (random, random) random
+instantiation "*" :: ("{type, random}", "{type, random}") random
 begin
 
 definition
@@ -277,7 +277,7 @@
 
 end
 
-instantiation list :: (random) random
+instantiation list :: ("{type, random}") random
 begin
 
 primrec
@@ -429,7 +429,7 @@
 code_const "Eval.term_of :: ('a\<Colon>term_of \<Rightarrow> 'b\<Colon>term_of) \<Rightarrow> _"
   (SML "(fn '_ => Const (\"arbitrary\", dummyT))")
 
-instantiation "fun" :: (eq, random) random
+instantiation "fun" :: (eq, "{type, random}") random
 begin
 
 definition