aboutsummaryrefslogtreecommitdiff
path: root/src/Spec/WeierstrassCurve.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Spec/WeierstrassCurve.v')
-rw-r--r--src/Spec/WeierstrassCurve.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Spec/WeierstrassCurve.v b/src/Spec/WeierstrassCurve.v
index fc7c64198..9a3a9185d 100644
--- a/src/Spec/WeierstrassCurve.v
+++ b/src/Spec/WeierstrassCurve.v
@@ -41,7 +41,7 @@ Module W.
Program Definition zero : point := ∞.
Local Notation "0" := Fzero. Local Notation "1" := Fone.
- Local Notation "2" := (1+1). Local Notation "3" := (1+2).
+ Local Notation "2" := (1+1). Local Notation "3" := (1+2).
Program Definition add (P1 P2:point) : point :=
match coordinates P1, coordinates P2 return F*F+∞ with