aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Mult.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/Mult.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/Mult.v')
-rwxr-xr-xtheories/Arith/Mult.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/theories/Arith/Mult.v b/theories/Arith/Mult.v
index 8955b1ea3..86404aca3 100755
--- a/theories/Arith/Mult.v
+++ b/theories/Arith/Mult.v
@@ -26,8 +26,8 @@ Hints Resolve mult_plus_distr : arith v62.
Lemma mult_plus_distr_r : (n,m,p:nat) (mult n (plus m p))=(plus (mult n m) (mult n p)).
Proof.
- Induction n. Trivial.
- Intros. Simpl. Rewrite (H m p). Apply sym_eq. Apply plus_permute_2_in_4.
+ NewInduction n. Trivial.
+ Intros. Simpl. Rewrite (IHn m p). Apply sym_eq. Apply plus_permute_2_in_4.
Qed.
Lemma mult_minus_distr : (n,m,p:nat)((mult (minus n m) p)=(minus (mult n p) (mult m p))).
@@ -39,7 +39,7 @@ Hints Resolve mult_minus_distr : arith v62.
Lemma mult_O_le : (n,m:nat)(m=O)\/(le n (mult m n)).
Proof.
-Induction m; Simpl; Auto with arith.
+NewInduction m; Simpl; Auto with arith.
Qed.
Hints Resolve mult_O_le : arith v62.
@@ -76,16 +76,16 @@ Hints Resolve mult_n_1 : arith v62.
Lemma mult_le : (m,n,p:nat) (le n p) -> (le (mult m n) (mult m p)).
Proof.
- Induction m. Intros. Simpl. Apply le_n.
+ NewInduction m. Intros. Simpl. Apply le_n.
Intros. Simpl. Apply le_plus_plus. Assumption.
- Apply H. Assumption.
+ Apply IHm. Assumption.
Qed.
Hints Resolve mult_le : arith.
Lemma mult_lt : (m,n,p:nat) (lt n p) -> (lt (mult (S m) n) (mult (S m) p)).
Proof.
- Induction m. Intros. Simpl. Rewrite <- plus_n_O. Rewrite <- plus_n_O. Assumption.
- Intros. Exact (lt_plus_plus ? ? ? ? H0 (H ? ? H0)).
+ NewInduction m. Intros. Simpl. Rewrite <- plus_n_O. Rewrite <- plus_n_O. Assumption.
+ Intros. Exact (lt_plus_plus ? ? ? ? H (IHm ? ? H)).
Qed.
Hints Resolve mult_lt : arith.