Maps between real and extended non-negative real numbers #
This file focuses on the functions ENNReal.toReal : ℝ≥0∞ → ℝ
and ENNReal.ofReal : ℝ → ℝ≥0∞
which
were defined in Data.ENNReal.Basic
. It collects all the basic results of the interactions between
these functions and the algebraic and lattice operations, although a few may appear in earlier
files.
This file provides a positivity
extension for ENNReal.ofReal
.
Main theorems #
trichotomy (p : ℝ≥0∞) : p = 0 ∨ p = ∞ ∨ 0 < p.toReal
: often used forWithLp
andlp
dichotomy (p : ℝ≥0∞) [Fact (1 ≤ p)] : p = ∞ ∨ 1 ≤ p.toReal
: often used forWithLp
andlp
toNNReal_iInf
throughtoReal_sSup
: these declarations allow for easy conversions between indexed or set infima and suprema inℝ
,ℝ≥0
andℝ≥0∞
. This is especially useful becauseℝ≥0∞
is a complete lattice.
@[simp]
@[simp]
@[simp]
Alias of the reverse direction of ENNReal.ofReal_eq_zero
.
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
theorem
ENNReal.toReal_le_of_le_ofReal
{a : ENNReal}
{b : ℝ}
(hb : 0 ≤ b)
(h : a ≤ ENNReal.ofReal b)
:
ENNReal.toNNReal
as a MonoidHom
.
Equations
- ENNReal.toNNRealHom = { toFun := ENNReal.toNNReal, map_one' := ENNReal.toNNRealHom.proof_1, map_mul' := ⋯ }
Instances For
@[simp]
Extension for the positivity
tactic: ENNReal.ofReal
.