src/HOLCF/Adm.thy
changeset 27413 3154f3765cc7
parent 27290 784620cccb80
child 27419 ff2a2b8fcd09
equal deleted inserted replaced
27412:e93b937ca933 27413:3154f3765cc7
   165 
   165 
   166 lemma compactD: "compact k \<Longrightarrow> adm (\<lambda>x. \<not> k \<sqsubseteq> x)"
   166 lemma compactD: "compact k \<Longrightarrow> adm (\<lambda>x. \<not> k \<sqsubseteq> x)"
   167 unfolding compact_def .
   167 unfolding compact_def .
   168 
   168 
   169 lemma compactI2:
   169 lemma compactI2:
   170   "(\<And>Y. \<lbrakk>chain Y; x \<sqsubseteq> lub (range Y)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i) \<Longrightarrow> compact x"
   170   "(\<And>Y. \<lbrakk>chain Y; x \<sqsubseteq> (\<Squnion>i. Y i)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i) \<Longrightarrow> compact x"
   171 unfolding compact_def adm_def by fast
   171 unfolding compact_def adm_def by fast
   172 
   172 
   173 lemma compactD2:
   173 lemma compactD2:
   174   "\<lbrakk>compact x; chain Y; x \<sqsubseteq> lub (range Y)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i"
   174   "\<lbrakk>compact x; chain Y; x \<sqsubseteq> (\<Squnion>i. Y i)\<rbrakk> \<Longrightarrow> \<exists>i. x \<sqsubseteq> Y i"
   175 unfolding compact_def adm_def by fast
   175 unfolding compact_def adm_def by fast
   176 
   176 
   177 lemma compact_chfin [simp]: "compact (x::'a::chfin)"
   177 lemma compact_chfin [simp]: "compact (x::'a::chfin)"
   178 by (rule compactI [OF adm_chfin])
   178 by (rule compactI [OF adm_chfin])
   179 
   179