aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
Diffstat (limited to 'theories')
-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 4fa0d7273..e2ff55b23 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 30, left associativity).
-Notation "- b" := (negb b) : bool_scope V8only
+Notation "- b" := (negb b) : bool_scope V8only.
Open Local Scope bool_scope.