Division polynomials of Weierstrass curves #
This file defines certain polynomials associated to division polynomials of Weierstrass curves.
These are defined in terms of the auxiliary sequences for normalised elliptic divisibility sequences
(EDS) as defined in Mathlib.NumberTheory.EllipticDivisibilitySequence
.
Mathematical background #
Let W
be a Weierstrass curve over a commutative ring R
. The sequence of n
-division polynomials
ψₙ ∈ R[X, Y]
of W
is the normalised EDS with initial values
ψ₀ := 0
,ψ₁ := 1
,ψ₂ := 2Y + a₁X + a₃
,ψ₃ := 3X⁴ + b₂X³ + 3b₄X² + 3b₆X + b₈
, andψ₄ := ψ₂ ⬝ (2X⁶ + b₂X⁵ + 5b₄X⁴ + 10b₆X³ + 10b₈X² + (b₂b₈ - b₄b₆)X + (b₄b₈ - b₆²))
.
Furthermore, define the associated sequences φₙ, ωₙ ∈ R[X, Y]
by
φₙ := Xψₙ² - ψₙ₊₁ ⬝ ψₙ₋₁
, andωₙ := (ψ₂ₙ / ψₙ - ψₙ ⬝ (a₁φₙ + a₃ψₙ²)) / 2
.
Note that ωₙ
is always well-defined as a polynomial in R[X, Y]
. As a start, it can be shown by
induction that ψₙ
always divides ψ₂ₙ
in R[X, Y]
, so that ψ₂ₙ / ψₙ
is always well-defined as
a polynomial, while division by 2
is well-defined when R
has characteristic different from 2
.
In general, it can be shown that 2
always divides the polynomial ψ₂ₙ / ψₙ - ψₙ ⬝ (a₁φₙ + a₃ψₙ²)
in the characteristic 0
universal ring 𝓡[X, Y] := ℤ[A₁, A₂, A₃, A₄, A₆][X, Y]
of W
, where the
Aᵢ
are indeterminates. Then ωₙ
can be equivalently defined as the image of this division under
the associated universal morphism 𝓡[X, Y] → R[X, Y]
mapping Aᵢ
to aᵢ
.
Now, in the coordinate ring R[W]
, note that ψ₂²
is congruent to the polynomial
Ψ₂Sq := 4X³ + b₂X² + 2b₄X + b₆ ∈ R[X]
. As such, the recurrences of a normalised EDS show that
ψₙ / ψ₂
are congruent to certain polynomials in R[W]
. In particular, define preΨₙ ∈ R[X]
as
the auxiliary sequence for a normalised EDS with extra parameter Ψ₂Sq²
and initial values
The corresponding normalised EDS Ψₙ ∈ R[X, Y]
is then given by
Ψₙ := preΨₙ ⬝ ψ₂
ifn
is even, andΨₙ := preΨₙ
ifn
is odd.
Furthermore, define the associated sequences ΨSqₙ, Φₙ ∈ R[X]
by
ΨSqₙ := preΨₙ² ⬝ Ψ₂Sq
ifn
is even,ΨSqₙ := preΨₙ²
ifn
is odd,Φₙ := XΨSqₙ - preΨₙ₊₁ ⬝ preΨₙ₋₁
ifn
is even, andΦₙ := XΨSqₙ - preΨₙ₊₁ ⬝ preΨₙ₋₁ ⬝ Ψ₂Sq
ifn
is odd.
With these definitions, ψₙ ∈ R[X, Y]
and φₙ ∈ R[X, Y]
are congruent in R[W]
to Ψₙ ∈ R[X, Y]
and Φₙ ∈ R[X]
respectively, which are defined in terms of Ψ₂Sq ∈ R[X]
and preΨₙ ∈ R[X]
.
Main definitions #
WeierstrassCurve.preΨ
: the univariate polynomialspreΨₙ
.WeierstrassCurve.ΨSq
: the univariate polynomialsΨSqₙ
.WeierstrassCurve.Ψ
: the bivariate polynomialsΨₙ
.WeierstrassCurve.Φ
: the univariate polynomialsΦₙ
.WeierstrassCurve.ψ
: the bivariaten
-division polynomialsψₙ
.WeierstrassCurve.φ
: the bivariate polynomialsφₙ
.- TODO: the bivariate polynomials
ωₙ
.
Implementation notes #
Analogously to Mathlib.NumberTheory.EllipticDivisibilitySequence
, the bivariate polynomials
Ψₙ
are defined in terms of the univariate polynomials preΨₙ
. This is done partially to avoid
ring division, but more crucially to allow the definition of ΨSqₙ
and Φₙ
as univariate
polynomials without needing to work under the coordinate ring, and to allow the computation of their
leading terms without ambiguity. Furthermore, evaluating these polynomials at a rational point on
W
recovers their original definition up to linear combinations of the Weierstrass equation of W
,
hence also avoiding the need to work in the coordinate ring.
TODO: implementation notes for the definition of ωₙ
.
References #
J Silverman, The Arithmetic of Elliptic Curves
Tags #
elliptic curve, division polynomial, torsion point
The 2
-division polynomial ψ₂ = Ψ₂
.
Equations
- W.ψ₂ = W.toAffine.polynomialY
Instances For
The univariate polynomial Ψ₂Sq
congruent to ψ₂²
.
Equations
Instances For
The univariate polynomials preΨₙ
for n ∈ ℕ
#
The 3
-division polynomial ψ₃ = Ψ₃
.
Equations
Instances For
The univariate polynomial preΨ₄
, which is auxiliary to the 4-division polynomial
ψ₄ = Ψ₄ = preΨ₄ψ₂
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The univariate polynomials preΨₙ
for n ∈ ℕ
, which are auxiliary to the bivariate polynomials
Ψₙ
congruent to the bivariate n
-division polynomials ψₙ
.
Equations
- W.preΨ' n = preNormEDS' (W.Ψ₂Sq ^ 2) W.Ψ₃ W.preΨ₄ n
Instances For
The univariate polynomials preΨₙ
for n ∈ ℤ
#
The univariate polynomials preΨₙ
for n ∈ ℤ
, which are auxiliary to the bivariate polynomials
Ψₙ
congruent to the bivariate n
-division polynomials ψₙ
.
Equations
- W.preΨ n = preNormEDS (W.Ψ₂Sq ^ 2) W.Ψ₃ W.preΨ₄ n
Instances For
The univariate polynomials ΨSqₙ
#
The univariate polynomials ΨSqₙ
congruent to ψₙ²
.
Instances For
The bivariate polynomials Ψₙ
#
The bivariate polynomials Ψₙ
congruent to the n
-division polynomials ψₙ
.
Instances For
The univariate polynomials Φₙ
#
The univariate polynomials Φₙ
congruent to φₙ
.
Equations
Instances For
The bivariate polynomials ψₙ
#
The bivariate n
-division polynomials ψₙ
.
Instances For
The bivariate polynomials φₙ
#
The bivariate polynomials φₙ
.