aboutsummaryrefslogtreecommitdiff
path: root/src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v
diff options
context:
space:
mode:
authorGravatar jadep <jadep@mit.edu>2019-04-01 06:57:19 -0400
committerGravatar jadephilipoom <jade.philipoom@gmail.com>2019-04-03 23:34:53 +0100
commitf40b3c81114a73c3ac259ca4cb5014464e779dd3 (patch)
treeceee31b6cab54a638cc9d0c94da1683e50b641b0 /src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v
parentc0fe35f49d61207d16c6db79936e38edf9661a49 (diff)
update import statements
Diffstat (limited to 'src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v')
-rw-r--r--src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v b/src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v
index 7a475a53a..84d5be615 100644
--- a/src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v
+++ b/src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v
@@ -7,6 +7,7 @@ Require Import Crypto.PushButtonSynthesis.ReificationCache.
Local Open Scope Z_scope.
Import Associational Positional.
+Import FancyMontgomeryReduction.MontgomeryReduction.
Local Set Keyed Unification. (* needed for making [autorewrite] fast, c.f. COQBUG(https://github.com/coq/coq/issues/9283) *)