working...

This commit is contained in:
Stefan Kebekus 2024-11-12 16:58:07 +01:00
parent c6caffc53d
commit 15fa18c52f
3 changed files with 11 additions and 26 deletions

View File

@ -63,5 +63,7 @@ theorem MeromorphicOn.decompose
sorry
have t₁ : ∀ᶠ x in 𝓝[≠] z, AnalyticAt (fun z => ∏ᶠ (p : ), (z - p) ^ h₁f.divisor p * g z) x := by
sorry
apply Filter.EventuallyEq.eq_of_nhds
apply StronglyMeromorphicAt.localIdentity
sorry

View File

@ -169,6 +169,7 @@ theorem StronglyMeromorphicAt.order_eq_zero_iff
exact nhdsWithin_le_nhds
exact this
theorem StronglyMeromorphicAt.localIdentity
{f g : }
{z₀ : }

View File

@ -45,32 +45,6 @@ theorem AnalyticOn.stronglyMeromorphicOn
exact h₁f z hz
/- Strongly meromorphic functions on compact, preconnected sets are quotients of analytic functions -/
theorem StronglyMeromorphicOn_finite
{f : }
{U : Set }
(h₁U : IsCompact U)
(h₂U : IsPreconnected U)
(h₁f : StronglyMeromorphicOn f U)
(h₂f : ∃ z ∈ U, f z ≠ 0) :
Set.Finite {z ∈ U | f z = 0} := by
sorry
/- Strongly meromorphic functions on compact, preconnected sets are quotients of analytic functions -/
theorem StronglyMeromorphicOn_quotient
{f : }
{U : Set }
(h₁U : IsCompact U)
(h₂U : IsPreconnected U)
(h₁f : StronglyMeromorphicOn f U)
(h₂f : ∃ z ∈ U, f z ≠ 0) :
∃ a b : , (AnalyticOnNhd a U) ∧ (AnalyticOnNhd b U) ∧ (∀ z ∈ U, a z ≠ 0 b z ≠ 0) ∧ f = a / b := by
sorry
/- Make strongly MeromorphicAt -/
noncomputable def MeromorphicOn.makeStronglyMeromorphicOn
{f : }
@ -105,6 +79,14 @@ theorem makeStronglyMeromorphicOn_changeDiscrete
· simp [h₂v]
theorem StronglyMeromorphicOn_of_makeStronglyMeromorphic
{f : }
{z₀ : }
(hf : MeromorphicOn f U) :
StronglyMeromorphicOn hf.makeStronglyMeromorphicOn U := by
sorry
theorem makeStronglyMeromorphicOn_changeDiscrete'
{f : }
{U : Set }