aboutsummaryrefslogtreecommitdiff
path: root/src/CompleteEdwardsCurve/Pre.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-03-10 13:49:01 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-03-10 13:49:01 -0500
commitbb6d1cb9e5dea833adf07689df0864178732a494 (patch)
tree2e6e1d7befc950131f217633af09d7ac27e9b04b /src/CompleteEdwardsCurve/Pre.v
parentdbe09dd5bfc2595cb9fd96725d87d9a729cd0247 (diff)
Finish absolutizing imports
The file coqprime/Coqprime/ListAux.v was importing List, which was confusing machines on which mathclasses was also installed. Using https://github.com/JasonGross/coq-tools ```bash make -kj10 cd src git ls-files "*.v" | xargs python ~/Documents/repos/coq-tools/absolutize-imports.py -i -R . Crypto ```
Diffstat (limited to 'src/CompleteEdwardsCurve/Pre.v')
-rw-r--r--src/CompleteEdwardsCurve/Pre.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/CompleteEdwardsCurve/Pre.v b/src/CompleteEdwardsCurve/Pre.v
index e4dc140e1..fea4a99b3 100644
--- a/src/CompleteEdwardsCurve/Pre.v
+++ b/src/CompleteEdwardsCurve/Pre.v
@@ -1,4 +1,4 @@
-Require Import BinInt Znumtheory VerdiTactics.
+Require Import Coq.ZArith.BinInt Coq.ZArith.Znumtheory Crypto.Tactics.VerdiTactics.
Require Import Crypto.Spec.ModularArithmetic.
Require Import Crypto.ModularArithmetic.PrimeFieldTheorems.