aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-12 16:03:01 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-12 16:03:01 +0000
commitb9e593857a6b74568e964d68b48e3253dcd33592 (patch)
treed5445b50e6c7af3aa72ccb66f30aee4cb34c8272 /theories7
parent6c0e74dc503086b136136555721687d8acea3a17 (diff)
Ajout delimiteur pour bool_scope
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5321 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Bool/Bool.v9
1 files changed, 6 insertions, 3 deletions
diff --git a/theories7/Bool/Bool.v b/theories7/Bool/Bool.v
index 3d0a7a2f1..03061169f 100755
--- a/theories7/Bool/Bool.v
+++ b/theories7/Bool/Bool.v
@@ -175,9 +175,12 @@ 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).
-V8Notation "- b" := (negb b) : bool_scope.
-Open Local Scope bool_scope.
+Open Scope bool_scope.
+
+Delimits Scope bool_scope with bool.
+
+Bind Scope bool_scope with bool.
(**************************)
(** Lemmas about [negb] *)
@@ -212,7 +215,7 @@ Qed.
Lemma no_fixpoint_negb : (b:bool)~(negb b)=b.
Proof.
-NewDestruct b; Simpl; Unfold not; Intro; Apply diff_true_false; Auto with bool.
+NewDestruct b; Simpl; Intro; Apply diff_true_false; Auto with bool.
Qed.
Lemma eqb_negb1 : (b:bool)(eqb (negb b) b)=false.