Conformal maps between complex vector spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We prove the sufficient and necessary conditions for a real-linear map between complex vector spaces to be conformal.
Main results #
is_conformal_map_complex_linear
: a nonzero complex linear map into an arbitrary complex normed space is conformal.is_conformal_map_complex_linear_conj
: the composition of a nonzero complex linear map withconj
is complex linear.is_conformal_map_iff_is_complex_or_conj_linear
: a real linear map between the complex plane is conformal iff it's complex linear or the composition of some complex linear map andconj
.
Warning #
Antiholomorphic functions such as the complex conjugate are considered as conformal functions in this file.
theorem
is_conformal_map_complex_linear
{E : Type u_1}
[normed_add_comm_group E]
[normed_space ℝ E]
[normed_space ℂ E]
{map : ℂ →L[ℂ] E}
(nonzero : map ≠ 0) :
theorem
is_conformal_map_complex_linear_conj
{E : Type u_1}
[normed_add_comm_group E]
[normed_space ℝ E]
[normed_space ℂ E]
{map : ℂ →L[ℂ] E}
(nonzero : map ≠ 0) :