remove unnecessary import of Ffun;
authorhuffman
Thu, 12 Jun 2008 22:14:07 +0200
changeset 27181 e1e9b210d699
parent 27180 51f3f3557ef4
child 27182 9e4475b9d58c
remove unnecessary import of Ffun; add lemma admD2
src/HOLCF/Adm.thy
--- a/src/HOLCF/Adm.thy	Thu Jun 12 22:12:27 2008 +0200
+++ b/src/HOLCF/Adm.thy	Thu Jun 12 22:14:07 2008 +0200
@@ -6,7 +6,7 @@
 header {* Admissibility and compactness *}
 
 theory Adm
-imports Ffun
+imports Cont
 begin
 
 defaultsort cpo
@@ -24,6 +24,9 @@
 lemma admD: "\<lbrakk>adm P; chain Y; \<And>i. P (Y i)\<rbrakk> \<Longrightarrow> P (\<Squnion>i. Y i)"
 unfolding adm_def by fast
 
+lemma admD2: "\<lbrakk>adm (\<lambda>x. \<not> P x); chain Y; P (\<Squnion>i. Y i)\<rbrakk> \<Longrightarrow> \<exists>i. P (Y i)"
+unfolding adm_def by fast
+
 lemma triv_admI: "\<forall>x. P x \<Longrightarrow> adm P"
 by (rule admI, erule spec)