Weierstrass ℘ functions #
Main definitions #
PeriodPair.℘: The Weierstrass℘-function associated to a pair of periods.
tags #
Weierstrass p-functions, Weierstrass p functions
A pair of ℝ-linearly independent complex numbers.
They span the period lattice in lattice,
and are the periods of the elliptic functions we shall construct.
- ω₁ : ℂ
The first period in a
PeriodPair. - ω₂ : ℂ
The second period in a
PeriodPair.
Instances For
The ℝ-basis of ℂ determined by a pair of periods.
Instances For
The lattice spanned by a pair of periods.
Instances For
theorem
PeriodPair.isClosed_of_subset_lattice
(L : PeriodPair)
{s : Set ℂ}
(hs : s ⊆ ↑L.lattice)
:
IsClosed s
The ℤ-basis of the lattice determined by a pair of periods.
Equations
- L.latticeBasis = (Module.Basis.span ⋯).map (LinearEquiv.ofEq (Submodule.span ℤ (Set.range ![L.ω₁, L.ω₂])) L.lattice ⋯)
Instances For
The equivalence from the lattice generated by a pair of periods to ℤ × ℤ.
Equations
Instances For
theorem
PeriodPair.hasSumLocallyUniformly_aux
(L : PeriodPair)
(f : ↥L.lattice → ℂ → ℂ)
(u : ℝ → ↥L.lattice → ℝ)
(hu : ∀ r > 0, Summable (u r))
(hf : ∀ r > 0, ∀ᶠ (R : ℝ) in Filter.atTop, ∀ (x : ℂ), ‖x‖ < r → ∀ (l : ↥L.lattice), ‖↑l‖ = R → ‖f l x‖ ≤ u r l)
:
HasSumLocallyUniformly f fun (x : ℂ) => ∑' (j : ↥L.lattice), f j x
The Weierstrass ℘ function with the l₀-term missing.
This is mainly a tool for calculations where one would want to omit a diverging term.