src/HOLCF/Up.thy
changeset 27413 3154f3765cc7
parent 27310 d0229bc6c461
child 27414 95ec4bda5bb9
--- a/src/HOLCF/Up.thy	Tue Jul 01 01:28:44 2008 +0200
+++ b/src/HOLCF/Up.thy	Tue Jul 01 02:19:53 2008 +0200
@@ -154,7 +154,7 @@
 
 lemma up_chain_lemma:
   "chain Y \<Longrightarrow>
-   (\<exists>A. chain A \<and> lub (range Y) = Iup (lub (range A)) \<and>
+   (\<exists>A. chain A \<and> (\<Squnion>i. Y i) = Iup (\<Squnion>i. A i) \<and>
    (\<exists>j. \<forall>i. Y (i + j) = Iup (A i))) \<or> (Y = (\<lambda>i. Ibottom))"
 apply (rule disjCI)
 apply (simp add: expand_fun_eq)
@@ -168,7 +168,7 @@
 
 lemma cpo_up: "chain (Y::nat \<Rightarrow> 'a u) \<Longrightarrow> \<exists>x. range Y <<| x"
 apply (frule up_chain_lemma, safe)
-apply (rule_tac x="Iup (lub (range A))" in exI)
+apply (rule_tac x="Iup (\<Squnion>i. A i)" in exI)
 apply (erule_tac j="j" in is_lub_range_shift [THEN iffD1, standard])
 apply (simp add: is_lub_Iup cpo_lubI)
 apply (rule exI, rule lub_const)