Exponential in a Banach algebra #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we define exp π : πΈ β πΈ
, the exponential map in a topological algebra πΈ
over a
field π
.
While for most interesting results we need πΈ
to be normed algebra, we do not require this in the
definition in order to make exp
independent of a particular choice of norm. The definition also
does not require that πΈ
be complete, but we need to assume it for most results.
We then prove some basic results, but we avoid importing derivatives here to minimize dependencies.
Results involving derivatives and comparisons with real.exp
and complex.exp
can be found in
analysis/special_functions/exponential
.
Main results #
We prove most result for an arbitrary field π
, and then specialize to π = β
or π = β
.
General case #
exp_add_of_commute_of_mem_ball
: ifπ
has characteristic zero, then given two commuting elementsx
andy
in the disk of convergence, we haveexp π (x+y) = (exp π x) * (exp π y)
exp_add_of_mem_ball
: ifπ
has characteristic zero andπΈ
is commutative, then given two elementsx
andy
in the disk of convergence, we haveexp π (x+y) = (exp π x) * (exp π y)
exp_neg_of_mem_ball
: ifπ
has characteristic zero andπΈ
is a division ring, then given an elementx
in the disk of convergence, we haveexp π (-x) = (exp π x)β»ΒΉ
.
π = β
or π = β
#
exp_series_radius_eq_top
: theformal_multilinear_series
definingexp π
has infinite radius of convergenceexp_add_of_commute
: given two commuting elementsx
andy
, we haveexp π (x+y) = (exp π x) * (exp π y)
exp_add
: ifπΈ
is commutative, then we haveexp π (x+y) = (exp π x) * (exp π y)
for anyx
andy
exp_neg
: ifπΈ
is a division ring, then we haveexp π (-x) = (exp π x)β»ΒΉ
.exp_sum_of_commute
: the analogous result toexp_add_of_commute
forfinset.sum
.exp_sum
: the analogous result toexp_add
forfinset.sum
.exp_nsmul
: repeated addition in the domain corresponds to repeated multiplication in the codomain.exp_zsmul
: repeated addition in the domain corresponds to repeated multiplication in the codomain.
Other useful compatibility results #
exp_eq_exp
: ifπΈ
is a normed algebra over two fieldsπ
andπ'
, thenexp π = exp π' πΈ
exp_series π πΈ
is the formal_multilinear_series
whose n
-th term is the map
(xα΅’) : πΈβΏ β¦ (1/n! : π) β’ β xα΅’
. Its sum is the exponential map exp π : πΈ β πΈ
.
Equations
- exp_series π πΈ = Ξ» (n : β), (β(n.factorial))β»ΒΉ β’ continuous_multilinear_map.mk_pi_algebra_fin π n πΈ
exp π : πΈ β πΈ
is the exponential map determined by the action of π
on πΈ
.
It is defined as the sum of the formal_multilinear_series
exp_series π πΈ
.
Note that when πΈ = matrix n n π
, this is the Matrix Exponential; see
analysis.normed_space.matrix_exponential
for lemmas specific to that
case.
Equations
- exp π x = (exp_series π πΈ).sum x
In a Banach-algebra πΈ
over a normed field π
of characteristic zero, if x
and y
are
in the disk of convergence and commute, then exp π (x + y) = (exp π x) * (exp π y)
.
exp π x
has explicit two-sided inverse exp π (-x)
.
Equations
- invertible_exp_of_mem_ball hx = {inv_of := exp π (-x), inv_of_mul_self := _, mul_inv_of_self := _}
Any continuous ring homomorphism commutes with exp
.
In a commutative Banach-algebra πΈ
over a normed field π
of characteristic zero,
exp π (x+y) = (exp π x) * (exp π y)
for all x
, y
in the disk of convergence.
In a normed algebra πΈ
over π = β
or π = β
, the series defining the exponential map
has an infinite radius of convergence.
In a Banach-algebra πΈ
over π = β
or π = β
, if x
and y
commute, then
exp π (x+y) = (exp π x) * (exp π y)
.
exp π x
has explicit two-sided inverse exp π (-x)
.
Equations
- invertible_exp π x = invertible_exp_of_mem_ball _
In a Banach-algebra πΈ
over π = β
or π = β
, if a family of elements f i
mutually
commute then exp π (β i, f i) = β i, exp π (f i)
.
Any continuous ring homomorphism commutes with exp
.
In a commutative Banach-algebra πΈ
over π = β
or π = β
,
exp π (x+y) = (exp π x) * (exp π y)
.
A version of exp_sum_of_commute
for a commutative Banach-algebra.
If a normed ring πΈ
is a normed algebra over two fields, then they define the same
exp_series
on πΈ
.
If a normed ring πΈ
is a normed algebra over two fields, then they define the same
exponential function on πΈ
.
A version of complex.of_real_exp
for exp
instead of complex.exp