Documentation

Mathlib.Data.ENat.Lattice

Extended natural numbers form a complete linear order #

This instance is not in Data.ENat.Basic to avoid dependency on Finsets.

We also restate some lemmas about WithTop for ENat to have versions that use Nat.cast instead of WithTop.some.

theorem ENat.iSup_coe_eq_top {ι : Sort u_1} {f : ι} :
⨆ (i : ι), (f i) = ¬BddAbove (Set.range f)
theorem ENat.iSup_coe_ne_top {ι : Sort u_1} {f : ι} :
⨆ (i : ι), (f i) BddAbove (Set.range f)
theorem ENat.iSup_coe_lt_top {ι : Sort u_1} {f : ι} :
⨆ (i : ι), (f i) < BddAbove (Set.range f)
theorem ENat.iInf_coe_eq_top {ι : Sort u_1} {f : ι} :
⨅ (i : ι), (f i) = IsEmpty ι
theorem ENat.iInf_coe_ne_top {ι : Sort u_1} {f : ι} :
⨅ (i : ι), (f i) Nonempty ι
theorem ENat.iInf_coe_lt_top {ι : Sort u_1} {f : ι} :
⨅ (i : ι), (f i) < Nonempty ι
theorem ENat.coe_sSup {s : Set } :
BddAbove s(sSup s) = ⨆ a ∈ s, a
theorem ENat.coe_sInf {s : Set } :
Set.Nonempty s(sInf s) = ⨅ a ∈ s, a
theorem ENat.coe_iSup {ι : Sort u_1} {f : ι} :
BddAbove (Set.range f)(⨆ (i : ι), f i) = ⨆ (i : ι), (f i)
theorem ENat.coe_iInf {ι : Sort u_1} {f : ι} [Nonempty ι] :
(⨅ (i : ι), f i) = ⨅ (i : ι), (f i)