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

Commit db18144

Browse files
committed
chore(order/bounded_lattice): add is_compl.inf_left_eq_bot_iff etc (#3460)
1 parent 1bb3d19 commit db18144

File tree

2 files changed

+13
-3
lines changed

2 files changed

+13
-3
lines changed

src/order/bounded_lattice.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1007,6 +1007,18 @@ lemma inf_sup {x' y'} (h : is_compl x y) (h' : is_compl x' y') :
10071007
is_compl (x ⊓ x') (y ⊔ y') :=
10081008
(h.symm.sup_inf h'.symm).symm
10091009

1010+
lemma inf_left_eq_bot_iff (h : is_compl y z) : x ⊓ y = ⊥ ↔ x ≤ z :=
1011+
inf_eq_bot_iff_le_compl h.sup_eq_top h.inf_eq_bot
1012+
1013+
lemma inf_right_eq_bot_iff (h : is_compl y z) : x ⊓ z = ⊥ ↔ x ≤ y :=
1014+
h.symm.inf_left_eq_bot_iff
1015+
1016+
lemma disjoint_left_iff (h : is_compl y z) : disjoint x y ↔ x ≤ z :=
1017+
disjoint_iff.trans h.inf_left_eq_bot_iff
1018+
1019+
lemma disjoint_right_iff (h : is_compl y z) : disjoint x z ↔ x ≤ y :=
1020+
h.symm.disjoint_left_iff
1021+
10101022
end is_compl
10111023

10121024
lemma is_compl_bot_top [bounded_lattice α] : is_compl (⊥ : α) ⊤ :=

src/topology/basic.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -654,9 +654,7 @@ lemma closure_eq_cluster_pts {s : set α} : closure s = {a | cluster_pt a (𝓟
654654
calc closure s = (interior sᶜ)ᶜ : closure_eq_compl_interior_compl
655655
... = {a | ¬ 𝓝 a ≤ 𝓟 sᶜ} : by rw [interior_eq_nhds]; refl
656656
... = {a | cluster_pt a (𝓟 s)} : set.ext $ assume a, not_congr
657-
(inf_eq_bot_iff_le_compl
658-
(show 𝓟 s ⊔ 𝓟 sᶜ = ⊤, by simp only [sup_principal, union_compl_self, principal_univ])
659-
(by simp only [inf_principal, inter_compl_self, principal_empty])).symm
657+
(is_compl_principal s).inf_left_eq_bot_iff.symm
660658

661659
theorem mem_closure_iff_cluster_pt {s : set α} {a : α} : a ∈ closure s ↔ cluster_pt a (𝓟 s) :=
662660
by simp only [closure_eq_cluster_pts, mem_set_of_eq]

0 commit comments

Comments
 (0)