aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Bool.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-29 12:07:39 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-29 12:07:39 +0000
commit184af744a27807d6cb239a8fafb19dfcf61e48c5 (patch)
tree2b54bd612d3e08902b62c7fae21087d13c4d450a /theories/Bool/Bool.v
parent48be85eef75634e11545fc24c3afb96fc9abc58d (diff)
Notations
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3979 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Bool.v')
-rwxr-xr-xtheories/Bool/Bool.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index f2c9bfc8e..afc9840e1 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -172,6 +172,9 @@ Definition negb := [b:bool]Cases b of
| false => true
end.
+Infix "||" orb (at level 4, left associativity) : bool_scope.
+Infix "&&" andb (at level 3, left associativity) : bool_scope.
+Notation "!! b" := (negb b) (at level 0, right associativity) : bool_scope.
(**************************)
(** Lemmas about [negb] *)