aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--Makefile.common2
-rw-r--r--theories/Numbers/Integer/TreeMod/ZTreeMod.v6
-rw-r--r--theories/Numbers/NatInt/Makefile4
3 files changed, 4 insertions, 8 deletions
diff --git a/Makefile.common b/Makefile.common
index cf0f234d7..e45d70b99 100644
--- a/Makefile.common
+++ b/Makefile.common
@@ -561,7 +561,7 @@ ZARITHVO:=\
theories/ZArith/ZOdiv_def.vo theories/ZArith/ZOdiv.vo
INTSVO:=\
- theories/Ints/Z/ZAux.vo \
+ theories/Ints/Zaux.vo \
theories/Ints/Basic_type.vo theories/Ints/Int31.vo \
theories/Ints/num/GenBase.vo theories/Ints/num/ZnZ.vo \
theories/Ints/num/GenAdd.vo theories/Ints/num/GenSub.vo \
diff --git a/theories/Numbers/Integer/TreeMod/ZTreeMod.v b/theories/Numbers/Integer/TreeMod/ZTreeMod.v
index e885d25bc..f81c71d72 100644
--- a/theories/Numbers/Integer/TreeMod/ZTreeMod.v
+++ b/theories/Numbers/Integer/TreeMod/ZTreeMod.v
@@ -8,13 +8,13 @@
(* Evgeny Makarov, INRIA, 2007 *)
(************************************************************************)
-(*i i*)
+(*i $Id:$ i*)
Require Export NZAxioms.
Require Import NMake. (* contains W0Type *)
Require Import ZnZ.
-Require Import Basic_type. (* contais base *)
-Require Import ZAux.
+Require Import Basic_type. (* contains base *)
+Require Import Zaux.
Module NZBigIntsAxiomsMod (Import BoundedIntsMod : W0Type) <: NZAxiomsSig.
diff --git a/theories/Numbers/NatInt/Makefile b/theories/Numbers/NatInt/Makefile
deleted file mode 100644
index e23d8dee2..000000000
--- a/theories/Numbers/NatInt/Makefile
+++ /dev/null
@@ -1,4 +0,0 @@
-.SUFFIXES: .v .vo .vi .g .html .tex .g.tex .g.html
-
-.v.vo:
- coqtop -boot -compile $*