aboutsummaryrefslogtreecommitdiff
path: root/src/BaseSystem.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/BaseSystem.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/BaseSystem.v')
-rw-r--r--src/BaseSystem.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/src/BaseSystem.v b/src/BaseSystem.v
index f0e0db077..4e07c4564 100644
--- a/src/BaseSystem.v
+++ b/src/BaseSystem.v
@@ -1,7 +1,7 @@
-Require Import List.
-Require Import Util.ListUtil Util.CaseUtil Util.ZUtil.
-Require Import ZArith.ZArith ZArith.Zdiv.
-Require Import Omega NPeano Arith.
+Require Import Coq.Lists.List.
+Require Import Crypto.Util.ListUtil Crypto.Util.CaseUtil Crypto.Util.ZUtil.
+Require Import Coq.ZArith.ZArith Coq.ZArith.Zdiv.
+Require Import Coq.omega.Omega Coq.Numbers.Natural.Peano.NPeano Coq.Arith.Arith.
Local Open Scope Z.