aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--Makefile.common7
-rw-r--r--theories/Numbers/Cyclic/Abstract/NZCyclic.v (renamed from theories/Numbers/Integer/TreeMod/ZTreeMod.v)12
2 files changed, 9 insertions, 10 deletions
diff --git a/Makefile.common b/Makefile.common
index 6ffc7f82a..fbd29d0b0 100644
--- a/Makefile.common
+++ b/Makefile.common
@@ -617,7 +617,7 @@ NUMBERSCOMMONVO:=$(addprefix theories/Numbers/, \
QRewrite.vo NumPrelude.vo BigNumPrelude.vo )
CYCLICABSTRACTVO:=$(addprefix theories/Numbers/Cyclic/Abstract/, \
- ZnZ.vo )
+ ZnZ.vo NZCyclic.vo )
CYCLICINT31VO:=$(addprefix theories/Numbers/Cyclic/Int31/, \
Int31.vo Z31Z.vo )
@@ -659,14 +659,11 @@ INTEGERBINARYVO:=$(addprefix theories/Numbers/Integer/Binary/, \
INTEGERNATPAIRSVO:=$(addprefix theories/Numbers/Integer/NatPairs/, \
ZNatPairs.vo )
-INTEGERTREEMODVO:=$(addprefix theories/Numbers/Integer/TreeMod/, \
- ZTreeMod.vo )
-
INTEGERBIGZVO:=$(addprefix theories/Numbers/Integer/BigZ/, \
ZMake.vo BigZ.vo )
INTEGERVO:=$(INTEGERABSTRACTVO) $(INTEGERBINARYVO) $(INTEGERNATPAIRSVO) \
- $(INTEGERTREEMODVO) $(INTEGERBIGZVO)
+ $(INTEGERBIGZVO)
RATIONALBIGQVO:=$(addprefix theories/Numbers/Rational/BigQ/, \
QMake_base.vo QpMake.vo QvMake.vo Q0Make.vo \
diff --git a/theories/Numbers/Integer/TreeMod/ZTreeMod.v b/theories/Numbers/Cyclic/Abstract/NZCyclic.v
index 591d245a6..7cc4e5434 100644
--- a/theories/Numbers/Integer/TreeMod/ZTreeMod.v
+++ b/theories/Numbers/Cyclic/Abstract/NZCyclic.v
@@ -11,12 +11,14 @@
(*i $Id$ i*)
Require Export NZAxioms.
-Require Import NMake. (* contains CyclicType *)
-Require Import ZnZ.
-Require Import Basic_type. (* contains base *)
Require Import BigNumPrelude.
+Require Import Basic_type.
+Require Import ZnZ.
+
+(** * A Z/nZ representation (module type [CyclicType]) implements
+ [NZAxiomsSig], e.g. the common properties between N and Z. *)
-Module NZBigIntsAxiomsMod (Import BoundedIntsMod : CyclicType) <: NZAxiomsSig.
+Module NZCyclicAxiomsMod (Import Cyclic : CyclicType) <: NZAxiomsSig.
Open Local Scope Z_scope.
@@ -226,4 +228,4 @@ rewrite Zplus_mod_idemp_l, Zmult_mod_idemp_l.
now rewrite Zmult_plus_distr_l, Zmult_1_l.
Qed.
-End NZBigIntsAxiomsMod.
+End NZCyclicAxiomsMod.