Update Basic.lean
Some checks failed
Lean Action CI / build (push) Has been cancelled

This commit is contained in:
Stefan Kebekus
2025-11-26 16:54:46 +01:00
parent c6396e002d
commit c699823ad8

View File

@@ -1,20 +1,44 @@
import Mathlib.Analysis.Meromorphic.Basic
import Mathlib.Analysis.Meromorphic.Order
import Mathlib.Analysis.Calculus.Deriv.Mul
import Mathlib.Analysis.Calculus.Deriv.ZPow
import Mathlib.Analysis.Calculus.Deriv.Shift
open MeromorphicOn Metric Real Set Classical
variable
{𝕜 : Type*} [NontriviallyNormedField 𝕜] [CompleteSpace 𝕜]
{𝕜 : Type*} [NontriviallyNormedField 𝕜]
{E : Type*} [NormedAddCommGroup E] [NormedSpace 𝕜 E] [CompleteSpace E]
{U : Set 𝕜} {f g : 𝕜 E} {a : WithTop E} {a₀ : E}
/-- Derivatives of meromorphic functions are meromorphic. -/
theorem meromorphicAt_deriv_of_order_eq_top {f : 𝕜 𝕜} {x : 𝕜}
(h : MeromorphicAt f x) (h₁ : h.order ) :
@[fun_prop]
theorem meromorphicAt_deriv {f : 𝕜 E} {x : 𝕜} (h : MeromorphicAt f x) :
MeromorphicAt (deriv f) x := by
have := h.eventually_analyticAt
obtain n, hn := h
rw [MeromorphicAt.iff_eventuallyEq_zpow_smul_analyticAt] at h
obtain n, g, h₁g, h₂g := h
let g : 𝕜 𝕜 := sorry
rw [MeromorphicAt.meromorphicAt_congr]
have : deriv (fun z (z - x) ^ n g z)
=[nhdsWithin x {x}] fun z₀ (n * (z₀ - x) ^ (n - 1)) g z₀ + (z₀ - x) ^ n deriv g z₀ := by
have τ₀ : (y : 𝕜) in nhdsWithin x {x}, AnalyticAt 𝕜 g y := by
exact eventually_nhdsWithin_of_eventually_nhds h₁g.eventually_analyticAt
have τ₁ : (y : 𝕜) in nhdsWithin x {x}, y x := by
exact eventually_nhdsWithin_of_forall fun x_1 a a
filter_upwards [τ₀, τ₁] with z₀ h₁ h₂
rw [deriv_smul]
rw [add_comm]
congr
rw [deriv_comp_sub_const (f := fun z z ^ n)]
aesop
refine DifferentiableAt.zpow ?_ ?_
fun_prop
left
exact sub_ne_zero_of_ne h₂
fun_prop
sorry
have : deriv f =[nhdsWithin x {x}] (fun z (z - x) ^ n g z) := by
sorry
apply MeromorphicAt.congr _ this.symm
fun_prop