src/HOLCF/Cont.thy
changeset 3842 b55686a7b22c
parent 3323 194ae2e0c193
child 4721 c8a8482a8124
--- a/src/HOLCF/Cont.thy	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOLCF/Cont.thy	Fri Oct 10 19:02:28 1997 +0200
@@ -28,10 +28,10 @@
 monofun         "monofun(f) == ! x y. x << y --> f(x) << f(y)"
 
 contlub         "contlub(f) == ! Y. is_chain(Y) --> 
-                                f(lub(range(Y))) = lub(range(% i.f(Y(i))))"
+                                f(lub(range(Y))) = lub(range(% i. f(Y(i))))"
 
 cont            "cont(f)   == ! Y. is_chain(Y) --> 
-                                range(% i.f(Y(i))) <<| f(lub(range(Y)))"
+                                range(% i. f(Y(i))) <<| f(lub(range(Y)))"
 
 (* ------------------------------------------------------------------------ *)
 (* the main purpose of cont.thy is to show:                                 *)