aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-08 20:24:51 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-08 20:24:51 +0000
commit29863a4dc9feeb75a184587b7b994626db7b94ce (patch)
tree0fc4182bbf72bd17b67e5aa8319f14e8fba271a1 /theories/Init/Datatypes.v
parent47e5f716f7ded0eec43b00d49955d56c370c3596 (diff)
- Patch sur "intros until 0"
- MAJ CHANGES et COMPATIBILITY - Réservation de || et && dans Notations.v - code mort et MAJ suite commit 11072 (tactics.ml et changes.txt) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11073 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Datatypes.v')
-rw-r--r--theories/Init/Datatypes.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index eb12be1a0..1e8a5b062 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -48,8 +48,8 @@ Definition xorb (b1 b2:bool) : bool :=
Definition negb (b:bool) := if b then false else true.
-Infix "||" := orb (at level 50, left associativity) : bool_scope.
-Infix "&&" := andb (at level 40, left associativity) : bool_scope.
+Infix "||" := orb : bool_scope.
+Infix "&&" := andb : bool_scope.
(*******************************)
(** * Properties of [andb] *)