Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 86dd706

Browse files
committed
feat(set/lattice): two lemmas about when sInter is empty (#9033)
- Added sInter_eq_empty_iff - Added sInter_nonempty_iff
1 parent 98cbad7 commit 86dd706

File tree

1 file changed

+11
-0
lines changed

1 file changed

+11
-0
lines changed

src/data/set/lattice.lean

Lines changed: 11 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -742,6 +742,17 @@ lemma sUnion_eq_univ_iff {c : set (set α)} :
742742
⋃₀ c = univ ↔ ∀ a, ∃ b ∈ c, a ∈ b :=
743743
by simp only [eq_univ_iff_forall, mem_sUnion]
744744

745+
-- classical
746+
lemma sInter_eq_empty_iff {c : set (set α)} :
747+
⋂₀ c = ∅ ↔ ∀ a, ∃ b ∈ c, a ∉ b :=
748+
by simp [set.eq_empty_iff_forall_not_mem, mem_sInter]
749+
750+
-- classical
751+
@[simp] theorem sInter_nonempty_iff {c : set (set α)}:
752+
(⋂₀ c).nonempty ↔ ∃ a, ∀ b ∈ c, a ∈ b :=
753+
by simp [← ne_empty_iff_nonempty, sInter_eq_empty_iff]
754+
755+
-- classical
745756
theorem compl_sUnion (S : set (set α)) :
746757
(⋃₀ S)ᶜ = ⋂₀ (compl '' S) :=
747758
ext $ λ x, by simp

0 commit comments

Comments
 (0)