Skip to content

Commit cea40eb

Browse files
urkudjcommelin
andcommitted
feat: port Order.Filter.AtTopBot (#1795)
Co-authored-by: Johan Commelin <johan@commelin.net>
1 parent fec4dbb commit cea40eb

File tree

3 files changed

+1973
-2
lines changed

3 files changed

+1973
-2
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -655,6 +655,7 @@ import Mathlib.Order.Cover
655655
import Mathlib.Order.Directed
656656
import Mathlib.Order.Disjoint
657657
import Mathlib.Order.Extension.Linear
658+
import Mathlib.Order.Filter.AtTopBot
658659
import Mathlib.Order.Filter.Bases
659660
import Mathlib.Order.Filter.Basic
660661
import Mathlib.Order.Filter.CountableInter

Mathlib/Order/ConditionallyCompleteLattice/Basic.lean

Lines changed: 9 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -828,10 +828,17 @@ theorem cinfᵢ_unique [Unique ι] {s : ι → α} : (⨅ i, s i) = s default :=
828828
@csupᵢ_unique αᵒᵈ _ _ _ _
829829
#align infi_unique cinfᵢ_unique
830830

831+
-- porting note: new lemma
832+
theorem csupᵢ_subsingleton [Subsingleton ι] (i : ι) (s : ι → α) : (⨆ i, s i) = s i :=
833+
@csupᵢ_unique α ι _ ⟨⟨i⟩, fun j => Subsingleton.elim j i⟩ _
834+
835+
-- porting note: new lemma
836+
theorem cinfᵢ_subsingleton [Subsingleton ι] (i : ι) (s : ι → α) : (⨅ i, s i) = s i :=
837+
@cinfᵢ_unique α ι _ ⟨⟨i⟩, fun j => Subsingleton.elim j i⟩ _
838+
831839
@[simp]
832840
theorem csupᵢ_pos {p : Prop} {f : p → α} (hp : p) : (⨆ h : p, f h) = f hp :=
833-
haveI := uniqueProp hp
834-
csupᵢ_unique
841+
csupᵢ_subsingleton hp f
835842
#align csupr_pos csupᵢ_pos
836843

837844
@[simp]

0 commit comments

Comments
 (0)