Documentation

Mathlib.Analysis.NormedSpace.QuaternionExponential

Lemmas about exp on Quaternions #

This file contains results about exp on Quaternion.

Main results #

@[simp]
theorem Quaternion.exp_coe (r : ) :
exp r = ↑(exp r)
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) :
HasSum (fun n => ↑(expSeries (Quaternion ) n) fun x => q) (c + (s / q) q)

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 imaginary quaternions.

The closed form for the quaternion exponential on arbitrary quaternions.

theorem Quaternion.re_exp (q : Quaternion ) :
(exp q).re = exp q.re * Real.cos q - q.re
theorem Quaternion.normSq_exp (q : Quaternion ) :
Quaternion.normSq (exp q) = exp q.re ^ 2
@[simp]

Note that this implies that exponentials of pure imaginary quaternions are unit quaternions since in that case the RHS is 1 via exp_zero and norm_one.