Power function on ℂ, ℝ, ℝ≥0, and ℝ≥0∞ #
We construct the power functions x ^ y where
xandyare complex numbers,- or
xandyare real numbers, - or
xis a nonnegative real number andyis a real number; - or
xis a number from[0, +∞](a.k.a.ℝ≥0∞) andyis a real number.
We also prove basic properties of these functions.
The complex power function x^y, given by x^y = exp(y log x) (where log is the principal
determination of the logarithm), unless x = 0 where one sets 0^0 = 1 and 0^y = 0 for
y ≠ 0.
Equations
- x.cpow y = ite (x = 0) (ite (y = 0) 1 0) (complex.exp ((complex.log x) * y))
Equations
The real power function x^y, defined as the real part of the complex 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.
For x < 0, the definition is somewhat arbitary as it depends on the choice of a complex
determination of the logarithm. With our conventions, it is equal to exp (y log x) cos (πy).
Equations
- real.has_pow = {pow := real.rpow}
For 0 ≤ x, the only problematic case in the equality x ^ y * x ^ z = x ^ (y + z) is for
x = 0 and y + z = 0, where the right hand side is 1 while the left hand side can vanish.
The inequality is always true, though, and given in this lemma.
The function x ^ y tends to +∞ at +∞ for any positive real y.
The function x ^ (-y) tends to 0 at +∞ for any positive real y.
The function x ^ (a / (b * x + c)) tends to 1 at +∞, for any real numbers a, b, and
c such that b is nonzero.
The function x ^ (1 / x) tends to 1 at +∞.
The function x ^ (-1 / x) tends to 1 at +∞.
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
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 : ℝ≥0∞), x ^ y) _ (λ (x : ℝ≥0∞), x ^ (1 / y)) _