src/HOLCF/Pcpo.thy
changeset 27413 3154f3765cc7
parent 26480 544cef16045b
child 27415 be852e06d546
--- a/src/HOLCF/Pcpo.thy	Tue Jul 01 01:28:44 2008 +0200
+++ b/src/HOLCF/Pcpo.thy	Tue Jul 01 02:19:53 2008 +0200
@@ -15,11 +15,11 @@
 
 axclass cpo < po
         -- {* class axiom: *}
-  cpo:   "chain S \<Longrightarrow> \<exists>x. range S <<| x" 
+  cpo:   "chain S \<Longrightarrow> \<exists>x. range S <<| x"
 
 text {* in cpo's everthing equal to THE lub has lub properties for every chain *}
 
-lemma cpo_lubI: "chain (S::nat \<Rightarrow> 'a::cpo) \<Longrightarrow> range S <<| lub (range S)"
+lemma cpo_lubI: "chain (S::nat \<Rightarrow> 'a::cpo) \<Longrightarrow> range S <<| (\<Squnion>i. S i)"
 by (fast dest: cpo elim: lubI)
 
 lemma thelubE: "\<lbrakk>chain S; (\<Squnion>i. S i) = (l::'a::cpo)\<rbrakk> \<Longrightarrow> range S <<| l"