aboutsummaryrefslogtreecommitdiff
path: root/src/Util/NumTheoryUtil.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/Util/NumTheoryUtil.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/Util/NumTheoryUtil.v')
-rw-r--r--src/Util/NumTheoryUtil.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Util/NumTheoryUtil.v b/src/Util/NumTheoryUtil.v
index 5acef8b75..10ce148b0 100644
--- a/src/Util/NumTheoryUtil.v
+++ b/src/Util/NumTheoryUtil.v
@@ -1,8 +1,8 @@
-Require Import Zpower Znumtheory ZArith.ZArith ZArith.Zdiv.
-Require Import Omega NPeano Arith.
+Require Import Coq.ZArith.Zpower Coq.ZArith.Znumtheory Coq.ZArith.ZArith Coq.ZArith.Zdiv.
+Require Import Coq.omega.Omega Coq.Numbers.Natural.Peano.NPeano Coq.Arith.Arith.
Require Import Crypto.Util.NatUtil Crypto.Util.ZUtil.
Require Import Coqprime.Zp.
-Require Import VerdiTactics.
+Require Import Crypto.Tactics.VerdiTactics.
Local Open Scope Z.
(* TODO: move somewhere else for lemmas about Coqprime? *)