aboutsummaryrefslogtreecommitdiff
path: root/theories/Bool
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 96160f0918..d17741295b 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -173,7 +173,8 @@ Definition negb := [b:bool]Cases b of
end.
Infix "||" orb (at level 4, left associativity) : bool_scope.
-Infix "&&" andb (at level 3, left associativity) : bool_scope.
+Infix "&&" andb (at level 3, no associativity) : bool_scope
+ V8only (at level 30, left associativity).
Notation "!! b" := (negb b) (at level 0, right associativity) : bool_scope.
Open Scope bool_scope.