src/HOL/Complete_Lattices.thy
changeset 69020 4f94e262976d
parent 68980 5717fbc55521
child 69164 74f1b0f10b2b
--- a/src/HOL/Complete_Lattices.thy	Wed Sep 19 21:06:12 2018 +0200
+++ b/src/HOL/Complete_Lattices.thy	Thu Sep 20 14:17:58 2018 +0100
@@ -1180,6 +1180,10 @@
 lemma Int_Inter_image: "(\<Inter>x\<in>C. A x \<inter> B x) = \<Inter>(A ` C) \<inter> \<Inter>(B ` C)"  (* FIXME drop *)
   by (simp add: INT_Int_distrib)
 
+lemma Int_Inter_eq: "A \<inter> \<Inter>\<B> = (if \<B>={} then A else (\<Inter>B\<in>\<B>. A \<inter> B))"
+                    "\<Inter>\<B> \<inter> A = (if \<B>={} then A else (\<Inter>B\<in>\<B>. B \<inter> A))"
+  by auto
+
 lemma Un_Union_image: "(\<Union>x\<in>C. A x \<union> B x) = \<Union>(A ` C) \<union> \<Union>(B ` C)"  (* FIXME drop *)
   \<comment> \<open>Devlin, Fundamentals of Contemporary Set Theory, page 12, exercise 5:\<close>
   \<comment> \<open>Union of a family of unions\<close>