aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-01 22:03:52 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-01 22:03:52 +0000
commitf2fdab57784b34bab5ef7e0c9d34fee76c329a33 (patch)
treefd2b578aab6b67e6d47bd76dcef1685b7c19cbd0 /theories/Bool
parente805bb1b608befa007e3a17373fa972821ee8d9e (diff)
Finalement, niveau 0 pour l'argument du '-' uniare, pour eviter que les entiers positifs soient parentheses en tant qu'arguments de fonction; tant pis, il faudra ecrire '-(-x)' au lieu de '--x'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4751 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 984bd77c4..3d0a7a2f1 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -175,7 +175,7 @@ Definition negb := [b:bool]Cases b of
Infix "||" orb (at level 4, left associativity) : bool_scope.
Infix "&&" andb (at level 3, no associativity) : bool_scope
V8only (at level 40, left associativity).
-Notation "- b" := (negb b) : bool_scope V8only.
+V8Notation "- b" := (negb b) : bool_scope.
Open Local Scope bool_scope.