aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/GF25519.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Assembly/GF25519.v')
-rw-r--r--src/Assembly/GF25519.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Assembly/GF25519.v b/src/Assembly/GF25519.v
index 081ddc008..84e692424 100644
--- a/src/Assembly/GF25519.v
+++ b/src/Assembly/GF25519.v
@@ -6,8 +6,8 @@ Require Import Crypto.Specific.GF25519.
Require Import Crypto.Util.Tuple.
Module GF25519.
- Definition bits: nat := 32.
- Definition width: Width bits := W32.
+ Definition bits: nat := 64.
+ Definition width: Width bits := W64.
Fixpoint makeBoundList {n} k (b: @WordRangeOpt n) :=
match k with