src/HOLCF/Pcpo.thy
changeset 5438 c89ee3a46a74
parent 4721 c8a8482a8124
child 12030 46d57d0290a2
--- a/src/HOLCF/Pcpo.thy	Tue Sep 08 17:07:39 1998 +0200
+++ b/src/HOLCF/Pcpo.thy	Wed Sep 09 16:13:35 1998 +0200
@@ -11,7 +11,7 @@
 (* ********************************************** *)
 axclass cpo < po
         (* class axiom: *)
-  cpo   "chain S ==> ? x. range(S) <<| (x::'a::po)" 
+  cpo   "chain S ==> ? x. range S <<| x" 
 
 (* The class pcpo of pointed cpos *)
 (* ****************************** *)