aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Bool.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-22 10:35:04 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-22 10:35:04 +0000
commit6475388a91c899e8bcf7b69b223180025d4f85ff (patch)
tree6031dc6e72bb676fa9d9e4f9f2be8ab50c1ca2e3 /theories/Bool/Bool.v
parent9da09a4da10aa36699538bde01086172c64689eb (diff)
reorganisation des niveaux (ex: = est a 70)
Hint Destruct: syntaxe similaire aux autres hints... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4696 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Bool.v')
-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 e2ff55b23..984bd77c4 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -174,7 +174,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).
+ V8only (at level 40, left associativity).
Notation "- b" := (negb b) : bool_scope V8only.
Open Local Scope bool_scope.