aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/IntegrationTestMontgomeryP256.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-06-17 23:51:38 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-06-17 23:51:38 -0400
commitec7aae22d2eef0787a529bb57a3530b18b3f02ad (patch)
tree6138e15afcdd9090cd659b6ac2027471eb22a36e /src/Specific/IntegrationTestMontgomeryP256.v
parent80d8ffbfb6bf3607cf7ef28033d13561bbadf2ba (diff)
Add 128-bit version of montgomery for testing
Diffstat (limited to 'src/Specific/IntegrationTestMontgomeryP256.v')
-rw-r--r--src/Specific/IntegrationTestMontgomeryP256.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Specific/IntegrationTestMontgomeryP256.v b/src/Specific/IntegrationTestMontgomeryP256.v
index 90aae7723..2fb08fb40 100644
--- a/src/Specific/IntegrationTestMontgomeryP256.v
+++ b/src/Specific/IntegrationTestMontgomeryP256.v
@@ -36,7 +36,7 @@ Section BoundedField25p5.
Definition mulmod_256 : { f:feBW -> feBW -> feBW
| forall A B,
BoundedWordToZ _ _ _ (f A B) =
- Saturated.drop_high (redc (r:=r)(R_numlimbs:=4) p256 (BoundedWordToZ _ _ _ A) (BoundedWordToZ _ _ _ B) 1)
+ Saturated.drop_high (redc (r:=r)(R_numlimbs:=sz) p256 (BoundedWordToZ _ _ _ A) (BoundedWordToZ _ _ _ B) 1)
}.
Proof.
(*Definition mulmod :