Update complexHarmonic.lean

This commit is contained in:
Stefan Kebekus 2024-05-08 08:32:06 +02:00
parent 5ce2b83c20
commit 69a35228ee
1 changed files with 8 additions and 0 deletions

View File

@ -46,9 +46,14 @@ theorem holomorphic_is_harmonic {f : } (h : Differentiable f) :
unfold Complex.laplace
rw [CauchyRiemann₄ h]
-- This lemma says that partial derivatives commute with complex scalar
-- multiplication. This is a consequence of partialDeriv_compContLin once we
-- note that complex scalar multiplication is continuous -linear.
have : ∀ v, ∀ s : , ∀ g : , Differentiable g → Real.partialDeriv v (s • g) = s • (Real.partialDeriv v g) := by
intro v s g hg
-- Present scalar multiplication as a continuous -linear map. This is
-- horrible, there must be better ways to do that.
let sMuls : →L[] :=
{
toFun := fun x ↦ s * x
@ -61,8 +66,11 @@ theorem holomorphic_is_harmonic {f : } (h : Differentiable f) :
ring
}
-- Bring the goal into a form that is recognized by
-- partialDeriv_compContLin.
have : s • g = sMuls ∘ g := by rfl
rw [this]
rw [partialDeriv_compContLin hg]
rfl