aboutsummaryrefslogtreecommitdiff
path: root/src/Curves/Weierstrass/Jacobian/Precomputed.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Curves/Weierstrass/Jacobian/Precomputed.v')
-rw-r--r--src/Curves/Weierstrass/Jacobian/Precomputed.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/Curves/Weierstrass/Jacobian/Precomputed.v b/src/Curves/Weierstrass/Jacobian/Precomputed.v
index 75aa6bf53..dbb1ecddf 100644
--- a/src/Curves/Weierstrass/Jacobian/Precomputed.v
+++ b/src/Curves/Weierstrass/Jacobian/Precomputed.v
@@ -20,7 +20,8 @@ Module Jacobian.
Local Notation "x ^ 2" := (x*x). Local Notation "x ^ 3" := (x^2*x).
Local Notation Wpoint := (@W.point F Feq Fadd Fmul a b).
- (* TODO: move non-precomputation-related defintions to a different file *)
+ (* TODO: import Jacobian.Basic here *)
+ (* TODO: factor out common parts of the tactic *)
Definition point : Type := { P : F*F*F | let '(X,Y,Z) := P in
if dec (Z=0) then True else Y^2 = X^3 + a*X*(Z^2)^2 + b*(Z^3)^2 }.