@@ -1743,11 +1743,13 @@ instance Pi.instCompleteLattice {α : Type*} {β : α → Type*} [∀ i, Complet
1743
1743
le_sInf _ _ hf := fun i => le_iInf fun g => hf g g.2 i
1744
1744
#align pi.complete_lattice Pi.instCompleteLattice
1745
1745
1746
+ @[simp]
1746
1747
theorem sSup_apply {α : Type *} {β : α → Type *} [∀ i, SupSet (β i)] {s : Set (∀ a, β a)} {a : α} :
1747
1748
(sSup s) a = ⨆ f : s, (f : ∀ a, β a) a :=
1748
1749
rfl
1749
1750
#align Sup_apply sSup_apply
1750
1751
1752
+ @[simp]
1751
1753
theorem sInf_apply {α : Type *} {β : α → Type *} [∀ i, InfSet (β i)] {s : Set (∀ a, β a)} {a : α} :
1752
1754
sInf s a = ⨅ f : s, (f : ∀ a, β a) a :=
1753
1755
rfl
@@ -1792,15 +1794,33 @@ theorem binary_relation_sInf_iff {α β : Type*} (s : Set (α → β → Prop))
1792
1794
1793
1795
section CompleteLattice
1794
1796
1795
- variable [Preorder α] [CompleteLattice β]
1797
+ variable {ι : Sort *} [Preorder α] [CompleteLattice β] {s : Set (α → β)} {f : ι → α → β}
1798
+
1799
+ protected lemma Monotone.sSup (hs : ∀ f ∈ s, Monotone f) : Monotone (sSup s) :=
1800
+ fun _ _ h ↦ iSup_mono fun f ↦ hs f f.2 h
1801
+ #align monotone_Sup_of_monotone Monotone.sSup
1802
+
1803
+ protected lemma Monotone.sInf (hs : ∀ f ∈ s, Monotone f) : Monotone (sInf s) :=
1804
+ fun _ _ h ↦ iInf_mono fun f ↦ hs f f.2 h
1805
+ #align monotone_Inf_of_monotone Monotone.sInf
1806
+
1807
+ protected lemma Antitone.sSup (hs : ∀ f ∈ s, Antitone f) : Antitone (sSup s) :=
1808
+ fun _ _ h ↦ iSup_mono fun f ↦ hs f f.2 h
1809
+
1810
+ protected lemma Antitone.sInf (hs : ∀ f ∈ s, Antitone f) : Antitone (sInf s) :=
1811
+ fun _ _ h ↦ iInf_mono fun f ↦ hs f f.2 h
1796
1812
1797
- theorem monotone_sSup_of_monotone {s : Set (α → β)} (m_s : ∀ f ∈ s, Monotone f) :
1798
- Monotone (sSup s) := fun _ _ h => iSup_mono fun f => m_s f f.2 h
1799
- #align monotone_Sup_of_monotone monotone_sSup_of_monotone
1813
+ @[deprecated (since := "2024-05-29")] alias monotone_sSup_of_monotone := Monotone.sSup
1814
+ @[deprecated (since := "2024-05-29")] alias monotone_sInf_of_monotone := Monotone.sInf
1800
1815
1801
- theorem monotone_sInf_of_monotone {s : Set (α → β)} (m_s : ∀ f ∈ s, Monotone f) :
1802
- Monotone (sInf s) := fun _ _ h => iInf_mono fun f => m_s f f.2 h
1803
- #align monotone_Inf_of_monotone monotone_sInf_of_monotone
1816
+ protected lemma Monotone.iSup (hf : ∀ i, Monotone (f i)) : Monotone (⨆ i, f i) :=
1817
+ Monotone.sSup (by simpa)
1818
+ protected lemma Monotone.iInf (hf : ∀ i, Monotone (f i)) : Monotone (⨅ i, f i) :=
1819
+ Monotone.sInf (by simpa)
1820
+ protected lemma Antitone.iSup (hf : ∀ i, Antitone (f i)) : Antitone (⨆ i, f i) :=
1821
+ Antitone.sSup (by simpa)
1822
+ protected lemma Antitone.iInf (hf : ∀ i, Antitone (f i)) : Antitone (⨅ i, f i) :=
1823
+ Antitone.sInf (by simpa)
1804
1824
1805
1825
end CompleteLattice
1806
1826
0 commit comments