src/HOLCF/Adm.thy
changeset 27413 3154f3765cc7
parent 27290 784620cccb80
child 27419 ff2a2b8fcd09
--- a/src/HOLCF/Adm.thy	Tue Jul 01 01:28:44 2008 +0200
+++ b/src/HOLCF/Adm.thy	Tue Jul 01 02:19:53 2008 +0200
@@ -167,11 +167,11 @@
 unfolding compact_def .
 
 lemma compactI2:
-  "(\<And>Y. \<lbrakk>chain Y; x \<sqsubseteq> lub (range Y)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i) \<Longrightarrow> compact x"
+  "(\<And>Y. \<lbrakk>chain Y; x \<sqsubseteq> (\<Squnion>i. Y i)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i) \<Longrightarrow> compact x"
 unfolding compact_def adm_def by fast
 
 lemma compactD2:
-  "\<lbrakk>compact x; chain Y; x \<sqsubseteq> lub (range Y)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i"
+  "\<lbrakk>compact x; chain Y; x \<sqsubseteq> (\<Squnion>i. Y i)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i"
 unfolding compact_def adm_def by fast
 
 lemma compact_chfin [simp]: "compact (x::'a::chfin)"