From f40b3c81114a73c3ac259ca4cb5014464e779dd3 Mon Sep 17 00:00:00 2001 From: jadep Date: Mon, 1 Apr 2019 06:57:19 -0400 Subject: update import statements --- src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v | 1 + 1 file changed, 1 insertion(+) (limited to 'src/PushButtonSynthesis/FancyMontgomeryReductionReificationCache.v') 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) *) -- cgit v1.2.3