aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Integer
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-16 00:53:17 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-16 00:53:17 +0000
commit18e543106f358272138a87bf331c4d1964a385f5 (patch)
tree5714692f140688b634eb789f3897e8dc1860b3c4 /theories/Numbers/Integer
parent49a7bb129b8a7f9d5a9175b7a340112c20e95d96 (diff)
More BigNum cleanup:
* View of Int31 as a Z/nZ moved to file Z31Z.v (TO FINISH: specs are still admitted!) * Modular specification of Z/nZ moved to ZnZ and renamed CyclicType * More isolation between Cyclic/Abstract and Cyclic/DoubleCyclic * A few comments git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10936 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Integer')
-rw-r--r--theories/Numbers/Integer/TreeMod/ZTreeMod.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Numbers/Integer/TreeMod/ZTreeMod.v b/theories/Numbers/Integer/TreeMod/ZTreeMod.v
index 2bb9bec4b..591d245a6 100644
--- a/theories/Numbers/Integer/TreeMod/ZTreeMod.v
+++ b/theories/Numbers/Integer/TreeMod/ZTreeMod.v
@@ -11,12 +11,12 @@
(*i $Id$ i*)
Require Export NZAxioms.
-Require Import NMake. (* contains W0Type *)
+Require Import NMake. (* contains CyclicType *)
Require Import ZnZ.
Require Import Basic_type. (* contains base *)
Require Import BigNumPrelude.
-Module NZBigIntsAxiomsMod (Import BoundedIntsMod : W0Type) <: NZAxiomsSig.
+Module NZBigIntsAxiomsMod (Import BoundedIntsMod : CyclicType) <: NZAxiomsSig.
Open Local Scope Z_scope.