aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-03 07:05:12 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-03 07:05:12 +0000
commite781edb69ae6c9e9d5c52646716b60332f98ff59 (patch)
tree4cf7f9013d456cb44d2bfdb3ff5d7c7cf422322d /theories/Bool
parentf2ea9fec68e0ae8193381513f650321c1b1f6900 (diff)
Compatibilité des noms longs de Bool déplacés dans Datatypes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9936 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rw-r--r--theories/Bool/Bool.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 1bd56a1ee..5cb4bcd5a 100644
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -691,3 +691,11 @@ Lemma negb_prop_involutive : forall b, Is_true b -> ~ Is_true (negb b).
Proof.
destruct b; intuition.
Qed.
+
+(* Compatibility *)
+
+Notation andb := Datatypes.andb (only parsing).
+Notation orb := Datatypes.orb (only parsing).
+Notation implb := Datatypes.implb (only parsing).
+Notation xorb := Datatypes.xorb (only parsing).
+Notation negb := Datatypes.negb (only parsing).