From ecd6954da5768ca3d38c7c52c6ac40b2b24d41a6 Mon Sep 17 00:00:00 2001 From: Andres Erbsen Date: Tue, 23 Aug 2016 18:34:01 -0400 Subject: remove eq_dec from Monoid --- src/CompleteEdwardsCurve/Pre.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'src/CompleteEdwardsCurve/Pre.v') 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. -- cgit v1.2.3