aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-21 22:05:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-21 22:05:23 +0000
commit45a33238f36b0d3ced493f83c2db9b9e150a214f (patch)
tree732758a2b82777196e8e7fd482630cd2bf2a83c3 /theories/ZArith
parentefffc572428b14f1f59b5820b1f23d452d29a1e7 (diff)
Les notations 'x <= y <= z' sont réservées et s'appliquent maintenant aussi à nat
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4427 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/zarith_aux.v14
1 files changed, 4 insertions, 10 deletions
diff --git a/theories/ZArith/zarith_aux.v b/theories/ZArith/zarith_aux.v
index c7fc10ee7..9798c4710 100644
--- a/theories/ZArith/zarith_aux.v
+++ b/theories/ZArith/zarith_aux.v
@@ -32,16 +32,10 @@ V8Infix "<" Zlt : Z_scope.
V8Infix ">=" Zge : Z_scope.
V8Infix ">" Zgt : Z_scope.
-V8Notation "x <= y <= z" := (Zle x y)/\(Zle y z)
- (at level 50, y at next level):Z_scope.
-V8Notation "x <= y < z" := (Zle x y)/\(Zlt y z)
- (at level 50, y at next level):Z_scope.
-V8Notation "x < y < z" := (Zlt x y)/\(Zlt y z)
- (at level 50, y at next level):Z_scope.
-V8Notation "x < y <= z" := (Zlt x y)/\(Zle y z)
- (at level 50, y at next level):Z_scope.
-V8Notation "x = y = z" := x=y/\y=z
- (at level 50, y at next level) : Z_scope.
+V8Notation "x <= y <= z" := (Zle x y)/\(Zle y z) :Z_scope.
+V8Notation "x <= y < z" := (Zle x y)/\(Zlt y z) :Z_scope.
+V8Notation "x < y < z" := (Zlt x y)/\(Zlt y z) :Z_scope.
+V8Notation "x < y <= z" := (Zlt x y)/\(Zle y z) :Z_scope.
(** Sign function *)
Definition Zsgn [z:Z] : Z :=