Lemmas about exp
on Quaternion
s #
This file contains results about exp
on Quaternion ℝ
.
Main results #
Quaternion.exp_eq
: the general expansion of the quaternion exponential in terms ofReal.cos
andReal.sin
.Quaternion.exp_of_re_eq_zero
: the special case when the quaternion has a zero real part.Quaternion.norm_exp
: the norm of the quaternion exponential is the norm of the exponential of the real part.
theorem
Quaternion.hasSum_expSeries_of_imaginary
{q : Quaternion ℝ}
(hq : q.re = 0)
{c : ℝ}
{s : ℝ}
(hc : HasSum (fun n => (-1) ^ n * ‖q‖ ^ (2 * n) / ↑(Nat.factorial (2 * n))) c)
(hs : HasSum (fun n => (-1) ^ n * ‖q‖ ^ (2 * n + 1) / ↑(Nat.factorial (2 * n + 1))) s)
:
Auxiliary result; if the power series corresponding to Real.cos
and Real.sin
evaluated
at ‖q‖
tend to c
and s
, then the exponential series tends to c + (s / ‖q‖)
.
The closed form for the quaternion exponential on arbitrary quaternions.
theorem
Quaternion.im_exp
(q : Quaternion ℝ)
:
Quaternion.im (exp ℝ q) = (exp ℝ q.re * (Real.sin ‖Quaternion.im q‖ / ‖Quaternion.im q‖)) • Quaternion.im q