aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-28 17:56:52 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-28 17:56:52 +0000
commit4b7c4f63039593833c349944c29c5fffc95e3c97 (patch)
tree0d400eeef621f73b9cddb4b4341a5bcc4ef3a0de /theories/ZArith
parente123d91faac12f9d304e7b245365ce5326e77f7a (diff)
Pas d'associativité gauche au niveau 3 en vieille syntaxe !
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3803 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Zdiv.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index 65b4422a1..f3cf93e0c 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -288,8 +288,10 @@ Syntax constr
-> [ (ZEXPR $n1):E " %" [1 0] (ZEXPR $n2):L ]
.
].
-Infix 3 "/" Zdiv : Z_scope.
-Infix 3 "mod" Zmod : Z_scope.
+
+
+Infix 3 "/" Zdiv (no associativity) : Z_scope V8only (left associativity).
+Infix 3 "mod" Zmod (no associativity) : Z_scope V8only (left associativity).
(** Other lemmas (now using the syntax for [Zdiv] and [Zmod]). *)