Documentation

Mathlib.Analysis.Calculus.Conformal.InnerProduct

Conformal maps between inner product spaces #

A function between inner product spaces which has a derivative at x is conformal at x iff the derivative preserves inner products up to a scalar multiple.

theorem conformalAt_iff' {E : Type u_1} {F : Type u_2} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {f : EF} {x : E} :
ConformalAt f x ∃ (c : ), 0 < c ∀ (u v : E), (fderiv f x) u, (fderiv f x) v⟫_ = c * u, v⟫_

A real differentiable map f is conformal at point x if and only if its differential fderiv ℝ f x at that point scales every inner product by a positive scalar.

theorem conformalAt_iff {E : Type u_1} {F : Type u_2} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {f : EF} {x : E} {f' : E →L[] F} (h : HasFDerivAt f f' x) :
ConformalAt f x ∃ (c : ), 0 < c ∀ (u v : E), f' u, f' v⟫_ = c * u, v⟫_

A real differentiable map f is conformal at point x if and only if its differential f' at that point scales every inner product by a positive scalar.

def conformalFactorAt {E : Type u_1} {F : Type u_2} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {f : EF} {x : E} (h : ConformalAt f x) :

The conformal factor of a conformal map at some point x. Some authors refer to this function as the characteristic function of the conformal map.

Equations
Instances For
    theorem conformalFactorAt_inner_eq_mul_inner' {E : Type u_1} {F : Type u_2} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {f : EF} {x : E} (h : ConformalAt f x) (u : E) (v : E) :
    (fderiv f x) u, (fderiv f x) v⟫_ = conformalFactorAt h * u, v⟫_
    theorem conformalFactorAt_inner_eq_mul_inner {E : Type u_1} {F : Type u_2} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {f : EF} {x : E} {f' : E →L[] F} (h : HasFDerivAt f f' x) (H : ConformalAt f x) (u : E) (v : E) :
    f' u, f' v⟫_ = conformalFactorAt H * u, v⟫_