Power function on ℝ≥0
and ℝ≥0∞
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We construct the power functions x ^ y
where
x
is a nonnegative real number andy
is a real number;x
is a number from[0, +∞]
(a.k.a.ℝ≥0∞
) andy
is a real number.
We also prove basic properties of these functions.
The nonnegative real power function x^y
, defined for x : ℝ≥0
and y : ℝ
as the
restriction of the real power function. For x > 0
, it is equal to exp (y log x)
. For x = 0
,
one sets 0 ^ 0 = 1
and 0 ^ y = 0
for y ≠ 0
.
Equations
The real power function x^y
on extended nonnegative reals, defined for x : ℝ≥0∞
and
y : ℝ
as the restriction of the real power function if 0 < x < ⊤
, and with the natural values
for 0
and ⊤
(i.e., 0 ^ x = 0
for x > 0
, 1
for x = 0
and ⊤
for x < 0
, and
⊤ ^ x = 1 / 0 ^ x
).
Equations
- ennreal.rpow (option.some x) y = ite (x = 0 ∧ y < 0) ⊤ ↑(x ^ y)
- ennreal.rpow option.none y = ite (0 < y) ⊤ (ite (y = 0) 1 0)
Equations
Bundles λ x : ℝ≥0∞, x ^ y
into an order isomorphism when y : ℝ
is positive,
where the inverse is λ x : ℝ≥0∞, x ^ (1 / y)
.
Equations
- ennreal.order_iso_rpow y hy = strict_mono.order_iso_of_right_inverse (λ (x : ennreal), x ^ y) _ (λ (x : ennreal), x ^ (1 / y)) _