aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-12 14:04:00 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-12 14:04:00 +0000
commit412c877f20ffceb407f2622bdfe6557a3df4062a (patch)
tree9c07cd012dbf709cf969bf9246307237e8147f81 /theories/Arith
parent398ac6536c4d4bd73105bc24c24f31e90cbe34d9 (diff)
Sorry for the mistake in r13702
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13704 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith')
-rw-r--r--theories/Arith/Plus.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Arith/Plus.v b/theories/Arith/Plus.v
index eb2d4df4c..02975d8f1 100644
--- a/theories/Arith/Plus.v
+++ b/theories/Arith/Plus.v
@@ -1,4 +1,4 @@
-(************************************************************************)
+ (************************************************************************)
(* v * The Coq Proof Assistant / The Coq Development Team *)
(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2010 *)
(* \VV/ **************************************************************)
@@ -26,7 +26,7 @@ Implicit Types m n p q : nat.
(** * Zero is neutral
Deprecated : Already in Init/Peano.v *)
-Definition plus_0_l n := eq_sym (plus_O_n n).
+Notation plus_0_l := plus_O_n (only parsing).
Definition plus_0_r n := eq_sym (plus_n_O n).
(** * Commutativity *)