aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Plus.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
commite10135925fa344ead0eb760c2c0fb7167d8dfc74 (patch)
treec00f1058346af155c3f54a297b452a1edd640197 /theories/Arith/Plus.v
parent634d52825790d8818883549616b3c8807655d2b8 (diff)
Independance vis a vis noms variables liees; partie sur bool dans Zbool
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4876 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Plus.v')
-rwxr-xr-xtheories/Arith/Plus.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/Arith/Plus.v b/theories/Arith/Plus.v
index d73b9820d..d44914499 100755
--- a/theories/Arith/Plus.v
+++ b/theories/Arith/Plus.v
@@ -61,11 +61,9 @@ Proof.
NewInduction n ; Simpl ; Auto with arith.
Qed.
-(** Relations with order *)
-
Lemma simpl_le_plus_l : (p,n,m:nat) (p+n)<=(p+m) -> n<=m.
Proof.
-NewInduction p; Simpl; Auto with arith.
+Intro p; NewInduction p; Simpl; Auto with arith.
Qed.
Lemma simpl_lt_plus_l : (n,m,p:nat) (p+n)<(p+m) -> n<m.
@@ -73,6 +71,8 @@ Proof.
NewInduction p; Simpl; Auto with arith.
Qed.
+(** Compatibility with order *)
+
Lemma le_reg_l : (n,m,p:nat) n<=m -> (p+n)<=(p+m).
Proof.
NewInduction p; Simpl; Auto with arith.
@@ -149,14 +149,14 @@ Qed.
Lemma plus_is_O : (m,n:nat) (m+n)=O -> m=O /\ n=O.
Proof.
- NewDestruct m; Auto.
+ Intro m; NewDestruct m; Auto.
Intros. Discriminate H.
Qed.
Definition plus_is_one :
(m,n:nat) (m+n)=(S O) -> {m=O /\ n=(S O)}+{m=(S O) /\ n=O}.
Proof.
- NewDestruct m; Auto.
+ Intro m; NewDestruct m; Auto.
NewDestruct n; Auto.
Intros.
Simpl in H. Discriminate H.
@@ -166,7 +166,7 @@ Defined.
Lemma plus_permute_2_in_4 : (m,n,p,q:nat) ((m+n)+(p+q))=((m+p)+(n+q)).
Proof.
- Intros.
+ Intros m n p q.
Rewrite <- (plus_assoc_l m n (p+q)). Rewrite (plus_assoc_l n p q).
Rewrite (plus_sym n p). Rewrite <- (plus_assoc_l p n q). Apply plus_assoc_l.
Qed.