aboutsummaryrefslogtreecommitdiff
path: root/src/CompleteEdwardsCurve/Pre.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2016-08-23 18:34:01 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2016-08-23 18:44:17 -0400
commitecd6954da5768ca3d38c7c52c6ac40b2b24d41a6 (patch)
treeb5084f85ba3295efc0c9dc23e58a7557adacd643 /src/CompleteEdwardsCurve/Pre.v
parent103549c7a210da4c007802a310cf79d314d277da (diff)
remove eq_dec from Monoid
Diffstat (limited to 'src/CompleteEdwardsCurve/Pre.v')
-rw-r--r--src/CompleteEdwardsCurve/Pre.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/CompleteEdwardsCurve/Pre.v b/src/CompleteEdwardsCurve/Pre.v
index 705597e15..fe98f5dcc 100644
--- a/src/CompleteEdwardsCurve/Pre.v
+++ b/src/CompleteEdwardsCurve/Pre.v
@@ -5,7 +5,7 @@ Require Import Crypto.Util.Notations Crypto.Util.Decidable.
Generalizable All Variables.
Section Pre.
Context {F eq zero one opp add sub mul inv div}
- `{field F eq zero one opp add sub mul inv div}.
+ `{field F eq zero one opp add sub mul inv div} {eq_dec:DecidableRel eq}.
Local Infix "=" := eq. Local Notation "a <> b" := (not (a = b)).
Local Infix "=" := eq : type_scope. Local Notation "a <> b" := (not (a = b)) : type_scope.