aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-17 16:33:07 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-17 16:33:07 +0000
commitae44b65793be9fd821dbf48389144d93dbd7d58f (patch)
tree8f19892940d47d32d017f259ac0ef2d5aaa0d995
parent5b318ca418ef27d1bf2b155bebbf2425f65b4f1f (diff)
Syntaxe 'x=y:>T'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3940 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/Init/LogicSyntax.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Init/LogicSyntax.v b/theories/Init/LogicSyntax.v
index 8326de6f8..483221be2 100644
--- a/theories/Init/LogicSyntax.v
+++ b/theories/Init/LogicSyntax.v
@@ -17,7 +17,9 @@ Notation "< P , Q > { p , q }" := (conj P Q p q) (P annot, at level 1).
Notation "~ x" := (not x) (at level 5, right associativity)
V8only (at level 55, right associativity).
+Notation "x = y :> T" := (!eq T x y) (at level 5, y at next level, no associativity).
Notation "x = y" := (eq ? x y) (at level 5, no associativity).
+Notation "x <> y :> T" := (not (!eq T x y)) (at level 5, y at next level, no associativity).
Notation "x <> y" := (not (eq ? x y)) (at level 5, no associativity).
Infix RIGHTA 6 "/\\" and.