src/HOL/Quickcheck_Random.thy
changeset 61076 bdc1e2f0a86a
parent 60758 d8d85a8172b5
child 61799 4cf66f21b764
--- a/src/HOL/Quickcheck_Random.thy	Tue Sep 01 17:25:36 2015 +0200
+++ b/src/HOL/Quickcheck_Random.thy	Tue Sep 01 22:32:58 2015 +0200
@@ -131,7 +131,7 @@
   \<Rightarrow> Random.seed \<Rightarrow> (('a \<Rightarrow> 'b) \<times> (unit \<Rightarrow> term)) \<times> Random.seed"
 
 definition random_fun_lift :: "(Random.seed \<Rightarrow> ('b \<times> (unit \<Rightarrow> term)) \<times> Random.seed)
-  \<Rightarrow> Random.seed \<Rightarrow> (('a\<Colon>term_of \<Rightarrow> 'b\<Colon>typerep) \<times> (unit \<Rightarrow> term)) \<times> Random.seed"
+  \<Rightarrow> Random.seed \<Rightarrow> (('a::term_of \<Rightarrow> 'b::typerep) \<times> (unit \<Rightarrow> term)) \<times> Random.seed"
 where
   "random_fun_lift f =
     random_fun_aux TYPEREP('a) TYPEREP('b) (op =) Code_Evaluation.term_of f Random.split_seed"