aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Cyclic/Int31
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-16 12:21:36 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-16 12:21:36 +0000
commit6c4cb0b91468ac0f7bc95d79f89b88417628127a (patch)
treec8e42704fae2d69398d8963445b24df3550c0f83 /theories/Numbers/Cyclic/Int31
parent9185da54dc70bf4009ae1bce6a52295cf6d77fe5 (diff)
Filename ZnZ (or Z_nZ in a later attempt) is neither pretty nor accurate
(n _must_ in fact be a power of 2). Worse: Z_31Z is just plain wrong since it is Z/(2^31)Z and not Z/31Z (my fault). As a consequence, switch to CyclicAxioms, Cyclic31, DoubleCyclic, etc git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10940 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Cyclic/Int31')
-rw-r--r--theories/Numbers/Cyclic/Int31/Cyclic31.v (renamed from theories/Numbers/Cyclic/Int31/Z_31Z.v)8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Numbers/Cyclic/Int31/Z_31Z.v b/theories/Numbers/Cyclic/Int31/Cyclic31.v
index 3b5944ed3..49a1a0b5b 100644
--- a/theories/Numbers/Cyclic/Int31/Z_31Z.v
+++ b/theories/Numbers/Cyclic/Int31/Cyclic31.v
@@ -8,14 +8,14 @@
(*i $Id$ i*)
-(** * Int31 numbers defines indeed a cyclic structure : Z/31Z *)
+(** * Int31 numbers defines indeed a cyclic structure : Z/(2^31)Z *)
(**
Author: Arnaud Spiwack
*)
Require Export Int31.
-Require Import Z_nZ.
+Require Import CyclicAxioms.
Open Scope int31_scope.
@@ -107,8 +107,8 @@ Definition int31_spec : znz_spec int31_op.
Admitted.
-Module Int31_words <: CyclicType.
+Module Int31Cyclic <: CyclicType.
Definition w := int31.
Definition w_op := int31_op.
Definition w_spec := int31_spec.
-End Int31_words.
+End Int31Cyclic.