aboutsummaryrefslogtreecommitdiff
path: root/src/Spec/MxDH.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Spec/MxDH.v')
-rw-r--r--src/Spec/MxDH.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Spec/MxDH.v b/src/Spec/MxDH.v
index 27f5f9a7f..d70521581 100644
--- a/src/Spec/MxDH.v
+++ b/src/Spec/MxDH.v
@@ -1,9 +1,9 @@
-Require Crypto.Algebra.
+Require Crypto.Algebra.Hierarchy.
Require Import Crypto.Util.Notations.
Module MxDH. (* from RFC7748 *)
Section MontgomeryLadderKeyExchange.
- Context {F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {field:@Algebra.field F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {Feq_dec:Decidable.DecidableRel Feq}.
+ Context {F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {field:@Algebra.Hierarchy.field F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {Feq_dec:Decidable.DecidableRel Feq}.
Local Infix "=" := Feq : type_scope. Local Notation "a <> b" := (not (a = b)) : type_scope.
Local Infix "+" := Fadd. Local Infix "*" := Fmul.
Local Infix "-" := Fsub. Local Infix "/" := Fdiv.