aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 12:31:32 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 12:31:32 +0000
commit561dcedd6bb9bf037d60a64385433c13bf9196a0 (patch)
treee1ce356383643c3b7106c85d811aeeebeaeae866 /theories7
parentb723d087151837ebfd285490858671544db3b1e1 (diff)
Meilleure robustesse des reordonnement d'arguments (2eme)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5049 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Arith/Plus.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories7/Arith/Plus.v b/theories7/Arith/Plus.v
index efd8ce83a..f6ea71de7 100755
--- a/theories7/Arith/Plus.v
+++ b/theories7/Arith/Plus.v
@@ -68,7 +68,7 @@ Hints Resolve plus_assoc_r : arith v62.
(** Simplification *)
-Lemma plus_reg_l : (n,m,p:nat)((p+n)=(p+m))->(n=m).
+Lemma plus_reg_l : (m,p,n:nat)((n+m)=(n+p))->(m=p).
Proof.
Intros m p n; NewInduction n ; Simpl ; Auto with arith.
Qed.