aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Bool.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:16:54 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:16:54 +0000
commiteb0ece31f16b90e0809f0cec59185c92b51fd702 (patch)
tree4961727abe59a8c251019c29a4bf7fe970897e07 /theories/Bool/Bool.v
parentd2edc017ee972bb4a1779ceb4a1961a6ab89f409 (diff)
Notations
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4047 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Bool.v')
-rwxr-xr-xtheories/Bool/Bool.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index afc9840e1..96160f091 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -175,6 +175,7 @@ Definition negb := [b:bool]Cases b of
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.
+Open Scope bool_scope.
(**************************)
(** Lemmas about [negb] *)