src/HOLCF/Cont.thy
changeset 1150 66512c9e6bd6
parent 243 c22b85994e17
child 1168 74be52691d62
--- a/src/HOLCF/Cont.thy	Wed Jun 21 15:01:07 1995 +0200
+++ b/src/HOLCF/Cont.thy	Wed Jun 21 15:14:58 1995 +0200
@@ -27,11 +27,11 @@
 
 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))))"
+contlub		"contlub(f) == ! Y. is_chain(Y) --> 
+				f(lub(range(Y))) = lub(range(% i.f(Y(i))))"
 
-contX		"contX(f)   == ! Y. is_chain(Y) --> \
-\				range(% i.f(Y(i))) <<| f(lub(range(Y)))"
+contX		"contX(f)   == ! Y. is_chain(Y) --> 
+				range(% i.f(Y(i))) <<| f(lub(range(Y)))"
 
 (* ------------------------------------------------------------------------ *)
 (* the main purpose of cont.thy is to show:                                 *)