Theory of complete lattices #
This file contains results on complete lattices that need more theory to develop.
Naming conventions #
In lemma names,
sSup
is calledsSup
sInf
is calledsInf
⨆ i, s i
is callediSup
⨅ i, s i
is callediInf
⨆ i j, s i j
is callediSup₂
. This is aniSup
inside aniSup
.⨅ i j, s i j
is callediInf₂
. This is aniInf
inside aniInf
.⨆ i ∈ s, t i
is calledbiSup
for "boundediSup
". This is the special case ofiSup₂
wherej : i ∈ s
.⨅ i ∈ s, t i
is calledbiInf
for "boundediInf
". This is the special case ofiInf₂
wherej : i ∈ s
.
Notation #
Instances #
This is a weaker version of sup_sInf_eq
This is a weaker version of inf_sSup_eq
This is a weaker version of sInf_sup_eq
This is a weaker version of sSup_inf_eq
theorem
disjoint_sSup_left
{α : Type u_1}
[CompleteLattice α]
{a : Set α}
{b : α}
(d : Disjoint (sSup a) b)
{i : α}
(hi : i ∈ a)
:
Disjoint i b
theorem
disjoint_sSup_right
{α : Type u_1}
[CompleteLattice α]
{a : Set α}
{b : α}
(d : Disjoint b (sSup a))
{i : α}
(hi : i ∈ a)
:
Disjoint b i
Equations
- ULift.supSet = { sSup := fun (s : Set (ULift.{?u.19, ?u.18} α)) => { down := sSup (ULift.up ⁻¹' s) } }
Equations
- ULift.infSet = { sInf := fun (s : Set (ULift.{?u.19, ?u.18} α)) => { down := sInf (ULift.up ⁻¹' s) } }
Equations
Equations
- One or more equations did not get rendered due to their size.