Skip to content

Commit 6620157

Browse files
committed
chore(AlgebraicGeometry/EllipticCurve/Projective/*): split projective files (#22549)
1 parent 6befc63 commit 6620157

File tree

6 files changed

+2089
-2028
lines changed

6 files changed

+2089
-2028
lines changed

Mathlib.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1063,7 +1063,9 @@ import Mathlib.AlgebraicGeometry.EllipticCurve.IsomOfJ
10631063
import Mathlib.AlgebraicGeometry.EllipticCurve.Jacobian
10641064
import Mathlib.AlgebraicGeometry.EllipticCurve.ModelsWithJ
10651065
import Mathlib.AlgebraicGeometry.EllipticCurve.NormalForms
1066-
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective
1066+
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective.Basic
1067+
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective.Formula
1068+
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective.Point
10671069
import Mathlib.AlgebraicGeometry.EllipticCurve.VariableChange
10681070
import Mathlib.AlgebraicGeometry.EllipticCurve.Weierstrass
10691071
import Mathlib.AlgebraicGeometry.Fiber

Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean

Lines changed: 2 additions & 29 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: David Kurniadi Angdinata
55
-/
66
import Mathlib.AlgebraicGeometry.EllipticCurve.Jacobian
7-
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective
87
import Mathlib.LinearAlgebra.FreeModule.Norm
98
import Mathlib.RingTheory.ClassGroup
109
import Mathlib.RingTheory.Polynomial.UniqueFactorization
@@ -13,9 +12,8 @@ import Mathlib.RingTheory.Polynomial.UniqueFactorization
1312
# Group law on Weierstrass curves
1413
1514
This file proves that the nonsingular rational points on a Weierstrass curve form an abelian group
16-
under the geometric group law defined in `Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean`, in
17-
`Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean`, and in
18-
`Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean`.
15+
under the geometric group law defined in `Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean` and
16+
in `Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean`.
1917
2018
## Mathematical background
2119
@@ -38,9 +36,6 @@ auxiliary lemmas in the proof of `WeierstrassCurve.Affine.Point.instAddCommGroup
3836
When `W` is given in Jacobian coordinates, `WeierstrassCurve.Jacobian.Point.toAffineAddEquiv` pulls
3937
back the group law on `WeierstrassCurve.Affine.Point` to `WeierstrassCurve.Jacobian.Point`.
4038
41-
When `W` is given in projective coordinates, `WeierstrassCurve.Projective.Point.toAffineAddEquiv`
42-
pulls back the group law on `WeierstrassCurve.Affine.Point` to `WeierstrassCurve.Projective.Point`.
43-
4439
## Main definitions
4540
4641
* `WeierstrassCurve.Affine.CoordinateRing`: the coordinate ring `F[W]` of a Weierstrass curve `W`.
@@ -56,8 +51,6 @@ pulls back the group law on `WeierstrassCurve.Affine.Point` to `WeierstrassCurve
5651
coordinates forms an abelian group under addition.
5752
* `WeierstrassCurve.Jacobian.Point.instAddCommGroup`: the type of nonsingular points on a
5853
Weierstrass curve in Jacobian coordinates forms an abelian group under addition.
59-
* `WeierstrassCurve.Projective.Point.instAddCommGroup`: the type of nonsingular points on a
60-
Weierstrass curve in projective coordinates forms an abelian group under addition.
6154
6255
## References
6356
@@ -565,26 +558,6 @@ end Point
565558

566559
end WeierstrassCurve.Affine
567560

568-
namespace WeierstrassCurve.Projective.Point
569-
570-
/-! ## Weierstrass curves in projective coordinates -/
571-
572-
variable {F : Type u} [Field F] {W : Projective F}
573-
574-
noncomputable instance : AddCommGroup W.Point where
575-
nsmul := nsmulRec
576-
zsmul := zsmulRec
577-
zero_add _ := (toAffineAddEquiv W).injective <| by
578-
simp only [map_add, toAffineAddEquiv_apply, toAffineLift_zero, zero_add]
579-
add_zero _ := (toAffineAddEquiv W).injective <| by
580-
simp only [map_add, toAffineAddEquiv_apply, toAffineLift_zero, add_zero]
581-
neg_add_cancel P := (toAffineAddEquiv W).injective <| by
582-
simp only [map_add, toAffineAddEquiv_apply, toAffineLift_neg, neg_add_cancel, toAffineLift_zero]
583-
add_comm _ _ := (toAffineAddEquiv W).injective <| by simp only [map_add, add_comm]
584-
add_assoc _ _ _ := (toAffineAddEquiv W).injective <| by simp only [map_add, add_assoc]
585-
586-
end WeierstrassCurve.Projective.Point
587-
588561
namespace WeierstrassCurve.Jacobian.Point
589562

590563
/-! ## Weierstrass curves in Jacobian coordinates -/

0 commit comments

Comments
 (0)