Update complexHarmonic.lean

This commit is contained in:
Stefan Kebekus 2024-05-15 21:17:42 +02:00
parent 1c34aee7be
commit bfeade4095
1 changed files with 9 additions and 12 deletions

View File

@ -159,6 +159,7 @@ theorem logabs_of_holomorphic_is_harmonic
have : (2 : )⁻¹ • (Real.log ∘ Complex.normSq ∘ f) = (fun z ↦ (2 : )⁻¹ • ((Real.log ∘ ⇑Complex.normSq ∘ f) z)) := by have : (2 : )⁻¹ • (Real.log ∘ Complex.normSq ∘ f) = (fun z ↦ (2 : )⁻¹ • ((Real.log ∘ ⇑Complex.normSq ∘ f) z)) := by
simp simp
exact rfl
rw [this] rw [this]
apply contDiff_iff_contDiffAt.2 apply contDiff_iff_contDiffAt.2
@ -229,18 +230,18 @@ theorem logabs_of_holomorphic_is_harmonic
exact h₂ z exact h₂ z
rw [this] rw [this]
rw [laplace_add] rw [laplace_add]
have : Differentiable (Complex.log ∘ f) := by have : Differentiable (Complex.log ∘ f) := by
intro z intro z
apply DifferentiableAt.comp apply DifferentiableAt.comp
exact Complex.differentiableAt_log (h₃ z) exact Complex.differentiableAt_log (h₃ z)
exact h₁ z exact h₁ z
have : Complex.laplace (Complex.log ∘ f) = 0 := by have t₁: Complex.laplace (Complex.log ∘ f) = 0 := by
let A := holomorphic_is_harmonic this let A := holomorphic_is_harmonic this
funext z funext z
exact A.2 z exact A.2 z
rw [this] rw [t]
simp simp
have : Complex.log ∘ ⇑(starRingEnd ) ∘ f = ⇑(starRingEnd ) ∘ Complex.log ∘ f := by have : Complex.log ∘ ⇑(starRingEnd ) ∘ f = ⇑(starRingEnd ) ∘ Complex.log ∘ f := by
@ -253,13 +254,9 @@ theorem logabs_of_holomorphic_is_harmonic
have : ⇑(starRingEnd ) ∘ Complex.log ∘ f = Complex.conjCLE ∘ Complex.log ∘ f := by have : ⇑(starRingEnd ) ∘ Complex.log ∘ f = Complex.conjCLE ∘ Complex.log ∘ f := by
rfl rfl
rw [this] rw [this]
have : ContDiff 2 (Complex.log ∘ f) := by sorry rw [laplace_compCLE]
rw [t₁]
have : Complex.laplace (⇑Complex.conjCLE ∘ f) = ⇑Complex.conjCLE ∘ Complex.laplace (f) := by simp
sorry
sorry
sorry
sorry sorry
sorry sorry