aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Plus.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-05 19:04:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-05 19:04:16 +0000
commit83c56744d7e232abeb5f23e6d0f23cd0abc14a9c (patch)
tree6d7d4c2ce3bb159b8f81a4193abde1e3573c28d4 /theories/Arith/Plus.v
parentf7351ff222bad0cc906dbee3c06b20babf920100 (diff)
Expérimentation de NewDestruct et parfois NewInduction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1880 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Plus.v')
-rwxr-xr-xtheories/Arith/Plus.v20
1 files changed, 10 insertions, 10 deletions
diff --git a/theories/Arith/Plus.v b/theories/Arith/Plus.v
index 1b70e1512..69bbd975a 100755
--- a/theories/Arith/Plus.v
+++ b/theories/Arith/Plus.v
@@ -32,7 +32,7 @@ Qed.
Lemma simpl_plus_l : (n,m,p:nat)((plus n m)=(plus n p))->(m=p).
Proof.
-Induction n ; Simpl ; Auto with arith.
+NewInduction n ; Simpl ; Auto with arith.
Qed.
Lemma plus_assoc_l : (n,m,p:nat)((plus n (plus m p))=(plus (plus n m) p)).
@@ -54,18 +54,18 @@ Hints Resolve plus_assoc_r : arith v62.
Lemma simpl_le_plus_l : (p,n,m:nat)(le (plus p n) (plus p m))->(le n m).
Proof.
-Induction p; Simpl; Auto with arith.
+NewInduction p; Simpl; Auto with arith.
Qed.
Lemma le_reg_l : (n,m,p:nat)(le n m)->(le (plus p n) (plus p m)).
Proof.
-Induction p; Simpl; Auto with arith.
+NewInduction p; Simpl; Auto with arith.
Qed.
Hints Resolve le_reg_l : arith v62.
Lemma le_reg_r : (a,b,c:nat) (le a b)->(le (plus a c) (plus b c)).
Proof.
-Induction 1 ; Simpl; Auto with arith.
+NewInduction 1 ; Simpl; Auto with arith.
Qed.
Hints Resolve le_reg_r : arith v62.
@@ -78,7 +78,7 @@ Qed.
Lemma le_plus_l : (n,m:nat)(le n (plus n m)).
Proof.
-Induction n; Simpl; Auto with arith.
+NewInduction n; Simpl; Auto with arith.
Qed.
Hints Resolve le_plus_l : arith v62.
@@ -96,12 +96,12 @@ Hints Resolve le_plus_trans : arith v62.
Lemma simpl_lt_plus_l : (n,m,p:nat)(lt (plus p n) (plus p m))->(lt n m).
Proof.
-Induction p; Simpl; Auto with arith.
+NewInduction p; Simpl; Auto with arith.
Qed.
Lemma lt_reg_l : (n,m,p:nat)(lt n m)->(lt (plus p n) (plus p m)).
Proof.
-Induction p; Simpl; Auto with arith.
+NewInduction p; Simpl; Auto with arith.
Qed.
Hints Resolve lt_reg_l : arith v62.
@@ -138,15 +138,15 @@ Qed.
Lemma plus_is_O : (m,n:nat) (plus m n)=O -> m=O /\ n=O.
Proof.
- Destruct m; Auto.
+ NewDestruct m; Auto.
Intros. Discriminate H.
Qed.
Lemma plus_is_one :
(m,n:nat) (plus m n)=(S O) -> {m=O /\ n=(S O)}+{m=(S O) /\ n=O}.
Proof.
- Destruct m; Auto.
- Destruct n; Auto.
+ NewDestruct m; Auto.
+ NewDestruct n; Auto.
Intros.
Simpl in H. Discriminate H.
Qed.