Update holomorphic_zero.lean

This commit is contained in:
Stefan Kebekus 2024-08-16 09:20:42 +02:00
parent 4b25e0694c
commit 83b3e0da1e
1 changed files with 31 additions and 5 deletions

View File

@ -1,10 +1,36 @@
import Mathlib.Analysis.Analytic.IsolatedZeros
import Nevanlinna.holomorphic
def zeroDivisor
{f : }
{R : }
(h₁f : ∀ z ∈ Metric.closedBall z R, HolomorphicAt f z)
(h₂f : ∃ z ∈ Metric.closedBall z R, f z ≠ 0) :
noncomputable def zeroDivisor
(f : ) :
:= by
intro z
if hf : AnalyticAt f z then
exact hf.order.toNat
else
exact 0
theorem discreteZeros
{f : } :
DiscreteTopology (Function.support (zeroDivisor f)) := by
sorry
theorem zeroDivisor_finiteOnCompact
{f : }
{s : Set }
(hs : IsCompact s) :
Set.Finite (s ∩ Function.support (zeroDivisor f)) := by
sorry
theorem eliminatingZeros
{f : }
{z₀ : }
{R : }
(h₁f : ∀ z ∈ Metric.ball z₀ R, HolomorphicAt f z)
(h₂f : ∃ z ∈ Metric.ball z₀ R, f z ≠ 0) :
∃ F : , ∀ z ∈ Metric.ball z₀ R, (HolomorphicAt F z) ∧ (f z = (F z) * ∏ᶠ a ∈ Metric.ball z₀ R, (z - a) ^ (zeroDivisor f a) ) := by
sorry