Documentation

Mathlib.AlgebraicGeometry.EllipticCurve.ModelsWithJ

Models of elliptic curves with prescribed j-invariant #

This file defines the Weierstrass equation over a field with prescribed j-invariant, proved that it is an elliptic curve, and that its j-invariant is equal to the given value. It is a modification of [Sil09], Chapter III, Proposition 1.4 (c).

Main definitions #

Main statements #

References #

Tags #

elliptic curve, weierstrass equation, j invariant

The Weierstrass curve $Y^2 + Y = X^3$. It is of j-invariant 0 if it is an elliptic curve.

Equations
Instances For

    The Weierstrass curve $Y^2 = X^3 + X$. It is of j-invariant 1728 if it is an elliptic curve.

    Equations
    Instances For

      The Weierstrass curve $Y^2 + (j - 1728)XY = X^3 - 36(j - 1728)^3X - (j - 1728)^5$. It is a modification of the curve in [Sil09], Chapter III, Proposition 1.4 (c) to avoid denominators. It is of j-invariant j if it is an elliptic curve.

      Equations
      Instances For
        theorem WeierstrassCurve.ofJNe0Or1728_c₄ {R : Type u_1} [CommRing R] (j : R) :
        (WeierstrassCurve.ofJNe0Or1728 j).c₄ = j * (j - 1728) ^ 3
        theorem WeierstrassCurve.ofJNe0Or1728_Δ {R : Type u_1} [CommRing R] (j : R) :
        (WeierstrassCurve.ofJNe0Or1728 j) = j ^ 2 * (j - 1728) ^ 9

        When 3 is a unit, $Y^2 + Y = X^3$ is an elliptic curve. It is of j-invariant 0 (see WeierstrassCurve.ofJ0_j).

        When 2 is a unit, $Y^2 = X^3 + X$ is an elliptic curve. It is of j-invariant 1728 (see WeierstrassCurve.ofJ1728_j).

        When j and j - 1728 are both units, $Y^2 + (j - 1728)XY = X^3 - 36(j - 1728)^3X - (j - 1728)^5$ is an elliptic curve. It is of j-invariant j (see WeierstrassCurve.ofJNe0Or1728_j).

        theorem WeierstrassCurve.ofJNe0Or1728_j {R : Type u_1} [CommRing R] (j : R) [Fact (IsUnit j)] [Fact (IsUnit (j - 1728))] :

        For any element j of a field $F$, there exists an elliptic curve over $F$ with j-invariant equal to j (see WeierstrassCurve.ofJ_j). Its coefficients are given explicitly (see WeierstrassCurve.ofJ0, WeierstrassCurve.ofJ1728 and WeierstrassCurve.ofJNe0Or1728).

        Equations
        Instances For
          theorem WeierstrassCurve.instIsEllipticOfJ {F : Type u_2} [Field F] (j : F) [DecidableEq F] :
          (WeierstrassCurve.ofJ j).IsElliptic
          theorem WeierstrassCurve.ofJ_j {F : Type u_2} [Field F] (j : F) [DecidableEq F] :
          Equations