aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 12:24:30 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 12:24:30 +0000
commitb723d087151837ebfd285490858671544db3b1e1 (patch)
treea9df7afdd3fd71d279b0a1c975a040f9783e6a81 /theories7
parent02d962bcf43380c8660846f103c188ae2bd70976 (diff)
Meilleure robustesse des reordonnement d'arguments
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5048 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Arith/Plus.v18
1 files changed, 16 insertions, 2 deletions
diff --git a/theories7/Arith/Plus.v b/theories7/Arith/Plus.v
index ffa94fcd0..efd8ce83a 100755
--- a/theories7/Arith/Plus.v
+++ b/theories7/Arith/Plus.v
@@ -73,7 +73,14 @@ Proof.
Intros m p n; NewInduction n ; Simpl ; Auto with arith.
Qed.
V7only [
-Notation simpl_plus_l := [n,m,p:nat](plus_reg_l m p n).
+(* Compatibility order of arguments *)
+Notation "'simpl_plus_l' c" := [a,b:nat](plus_reg_l a b c)
+ (at level 10, c at next level).
+Notation "'simpl_plus_l' c a" := [b:nat](plus_reg_l a b c)
+ (at level 10, a, c at next level).
+Notation "'simpl_plus_l' c a b" := (plus_reg_l a b c)
+ (at level 10, a, b, c at next level).
+Notation simpl_plus_l := plus_reg_l.
].
Lemma plus_le_reg_l : (n,m,p:nat) (p+n)<=(p+m) -> n<=m.
@@ -81,7 +88,14 @@ Proof.
NewInduction p; Simpl; Auto with arith.
Qed.
V7only [
-Notation simpl_le_plus_l := [p,n,m:nat](plus_le_reg_l n m p).
+(* Compatibility order of arguments *)
+Notation "'simpl_le_plus_l' c" := [a,b:nat](plus_le_reg_l a b c)
+ (at level 10, c at next level).
+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.
].
Lemma simpl_lt_plus_l : (n,m,p:nat) (p+n)<(p+m) -> n<m.