Extended non-negative reals
Topology on ennreal
.
Note: this is different from the emetric_space
topology. The emetric_space
topology has
is_open {⊤}
, while this topology doesn't have singleton elements.
Equations
Equations
The set of finite ennreal
numbers is homeomorphic to nnreal
.
Equations
- ennreal.ne_top_homeomorph_nnreal = {to_equiv := {to_fun := λ (x : ↥{a : ennreal | a ≠ ⊤}), ↑x.to_nnreal, inv_fun := λ (x : nnreal), ⟨↑x, _⟩, left_inv := ennreal.ne_top_homeomorph_nnreal._proof_1, right_inv := ennreal.ne_top_homeomorph_nnreal._proof_2}, continuous_to_fun := ennreal.ne_top_homeomorph_nnreal._proof_3, continuous_inv_fun := ennreal.ne_top_homeomorph_nnreal._proof_4}
The set of finite ennreal
numbers is homeomorphic to nnreal
.
Equations
- ennreal.lt_top_homeomorph_nnreal = (homeomorph.set_congr ennreal.lt_top_homeomorph_nnreal._proof_1).trans ennreal.ne_top_homeomorph_nnreal
Characterization of neighborhoods for ennreal
numbers. See also tendsto_order
for a version with strict inequalities.
Equations
- ennreal.has_continuous_add = _
- _ = _
- _ = _
In an emetric ball, the distance between points is everywhere finite
Each ball in an extended metric space gives us a metric space, as the edist is everywhere finite.
Yet another metric characterization of Cauchy sequences on integers. This one is often the most efficient.
If edist (f n) (f (n+1))
is bounded above by a function d : ℕ → ennreal
,
then the distance from f n
to the limit is bounded by ∑'_{k=n}^∞ d k
.
If edist (f n) (f (n+1))
is bounded above by a function d : ℕ → ennreal
,
then the distance from f 0
to the limit is bounded by ∑'_{k=0}^∞ d k
.