src/HOLCF/Cprod.thy
changeset 27413 3154f3765cc7
parent 27310 d0229bc6c461
child 29138 661a8db7e647
--- a/src/HOLCF/Cprod.thy	Tue Jul 01 01:28:44 2008 +0200
+++ b/src/HOLCF/Cprod.thy	Tue Jul 01 02:19:53 2008 +0200
@@ -129,7 +129,7 @@
 
 lemma thelub_cprod:
   "chain (S::nat \<Rightarrow> 'a::cpo \<times> 'b::cpo)
-    \<Longrightarrow> lub (range S) = (\<Squnion>i. fst (S i), \<Squnion>i. snd (S i))"
+    \<Longrightarrow> (\<Squnion>i. S i) = (\<Squnion>i. fst (S i), \<Squnion>i. snd (S i))"
 by (rule lub_cprod [THEN thelubI])
 
 instance "*" :: (cpo, cpo) cpo
@@ -326,7 +326,7 @@
 done
 
 lemma thelub_cprod2:
-  "chain S \<Longrightarrow> lub (range S) = <\<Squnion>i. cfst\<cdot>(S i), \<Squnion>i. csnd\<cdot>(S i)>"
+  "chain S \<Longrightarrow> (\<Squnion>i. S i) = <\<Squnion>i. cfst\<cdot>(S i), \<Squnion>i. csnd\<cdot>(S i)>"
 by (rule lub_cprod2 [THEN thelubI])
 
 lemma csplit1 [simp]: "csplit\<cdot>f\<cdot>\<bottom> = f\<cdot>\<bottom>\<cdot>\<bottom>"