aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-27 12:30:24 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-27 12:30:24 +0000
commite7b37fb18dc0e1aaca4f8f1e02656118eb8d10e6 (patch)
tree7346e6f273ff4f73131dda690188a7981cc900b2 /theories/QArith
parent7e5ae3dc23fb4823f8ff8851a01023733fc056f8 (diff)
Oups (on refait le 11268 en mieux)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11270 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/QArith')
-rw-r--r--theories/QArith/QArith_base.v4
1 files changed, 1 insertions, 3 deletions
diff --git a/theories/QArith/QArith_base.v b/theories/QArith/QArith_base.v
index a4e3a21a7..2c80aff40 100644
--- a/theories/QArith/QArith_base.v
+++ b/theories/QArith/QArith_base.v
@@ -43,9 +43,7 @@ Notation Qge a b := (Qle b a) (only parsing).
Infix "==" := Qeq (at level 70, no associativity) : Q_scope.
Infix "<" := Qlt : Q_scope.
-Infix ">" := Qgt : Q_scope.
-Infix "<=" := Qle : Q_scope (only parsing).
-Infix ">=" := Qge : Q_scope (only parsing).
+Infix "<=" := Qle : Q_scope.
Notation "x > y" := (Qlt y x)(only parsing) : Q_scope.
Notation "x >= y" := (Qle y x)(only parsing) : Q_scope.
Notation "x <= y <= z" := (x<=y/\y<=z) : Q_scope.