aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 13:36:45 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 13:36:45 +0000
commitac952fc310b1ba17c8e5a243ec617351130e1d81 (patch)
treedd4bda79ff66c17a08bc3fb01f76903f8a790eec /theories7
parent561dcedd6bb9bf037d60a64385433c13bf9196a0 (diff)
Meilleure robustesse des reordonnement d'arguments (3eme)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5050 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Arith/Plus.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories7/Arith/Plus.v b/theories7/Arith/Plus.v
index f6ea71de7..a00cde396 100755
--- a/theories7/Arith/Plus.v
+++ b/theories7/Arith/Plus.v
@@ -83,7 +83,7 @@ Notation "'simpl_plus_l' c a b" := (plus_reg_l a b c)
Notation simpl_plus_l := plus_reg_l.
].
-Lemma plus_le_reg_l : (n,m,p:nat) (p+n)<=(p+m) -> n<=m.
+Lemma plus_le_reg_l : (n,m,p:nat)((p+n)<=(p+m))->(n<=m).
Proof.
NewInduction p; Simpl; Auto with arith.
Qed.
@@ -95,7 +95,7 @@ Notation "'simpl_le_plus_l' c a" := [b:nat](plus_le_reg_l a b c)
(at level 10, a, c at next level).
Notation "'simpl_le_plus_l' c a b" := (plus_le_reg_l a b c)
(at level 10, a, b, c at next level).
-Notation simpl_le_plus_l := plus_reg_l.
+Notation simpl_le_plus_l := plus_le_reg_l.
].
Lemma simpl_lt_plus_l : (n,m,p:nat) (p+n)<(p+m) -> n<m.