aboutsummaryrefslogtreecommitdiff
path: root/src/PushButtonSynthesis/MontgomeryReduction.v
diff options
context:
space:
mode:
authorGravatar jadep <jadep@mit.edu>2019-03-14 16:32:51 -0400
committerGravatar jadephilipoom <jade.philipoom@gmail.com>2019-04-03 23:34:53 +0100
commit299206fc77217802c4431ccda1a7c0cb372f0b87 (patch)
tree80975ef89fbbac45cd9c61277eae73b1c3c6eb1a /src/PushButtonSynthesis/MontgomeryReduction.v
parenta189b8ad9943cec026ea2797789d8dc72a6d3336 (diff)
fix imports and qualifiers so everything builds
Diffstat (limited to 'src/PushButtonSynthesis/MontgomeryReduction.v')
-rw-r--r--src/PushButtonSynthesis/MontgomeryReduction.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/PushButtonSynthesis/MontgomeryReduction.v b/src/PushButtonSynthesis/MontgomeryReduction.v
index f61ece27c..d784ebc3c 100644
--- a/src/PushButtonSynthesis/MontgomeryReduction.v
+++ b/src/PushButtonSynthesis/MontgomeryReduction.v
@@ -15,7 +15,7 @@ Require Import Crypto.Util.ZUtil.Tactics.RewriteModSmall.
Require Import Crypto.Language.
Require Import Crypto.CStringification.
Require Import Crypto.Arithmetic.Core.
-Require Import Crypto.Arithmetic.FancyMongomeryReduction.
+Require Import Crypto.Arithmetic.MongomeryReduction.
Require Import Crypto.BoundsPipeline.
Require Import Crypto.COperationSpecifications.
Require Import Crypto.Fancy.Compiler.