src/HOL/Library/Infinite_Set.thy
changeset 34113 dbc0fb6e7eae
parent 34112 ca842111d698
child 34941 156925dd67af
--- a/src/HOL/Library/Infinite_Set.thy	Thu Dec 17 09:33:30 2009 -0800
+++ b/src/HOL/Library/Infinite_Set.thy	Thu Dec 17 13:49:36 2009 -0800
@@ -433,6 +433,13 @@
   "MOST x. P x \<Longrightarrow> MOST x. Q x \<Longrightarrow> MOST x. P x \<and> Q x"
   by (simp add: MOST_conj_distrib)
 
+lemma INFM_conjI:
+  "INFM x. P x \<Longrightarrow> MOST x. Q x \<Longrightarrow> INFM x. P x \<and> Q x"
+  unfolding MOST_iff_cofinite INFM_iff_infinite
+  apply (drule (1) Diff_infinite_finite)
+  apply (simp add: Collect_conj_eq Collect_neg_eq)
+  done
+
 lemma MOST_rev_mp:
   assumes "\<forall>\<^sub>\<infinity>x. P x" and "\<forall>\<^sub>\<infinity>x. P x \<longrightarrow> Q x"
   shows "\<forall>\<^sub>\<infinity>x. Q x"