aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Peano.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-01-10 12:15:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-01-10 12:15:06 +0000
commit4ff55199d062a25e7a3d678190552451121b1111 (patch)
treec365fe3ee8417bd633b3e502950fb2bf39093f14 /theories/Init/Peano.v
parent5719b93a439912b0fa1f32f4bb1d0369186e50ed (diff)
Modifs incongrues dans le précédent commit
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2385 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Peano.v')
-rwxr-xr-xtheories/Init/Peano.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v
index 724c3db2e..1ab517647 100755
--- a/theories/Init/Peano.v
+++ b/theories/Init/Peano.v
@@ -113,8 +113,8 @@ Hints Resolve mult_n_O : core v62.
Lemma mult_n_Sm : (n,m:nat) (plus (mult n m) n)=(mult n (S m)).
Proof.
- Intros n m; NewInduction n; Simpl; Auto.
- Rewrite <- IHn; Rewrite -> plus_n_Sm.
+ Intros; Elim n; Simpl; Auto.
+ Intros p H; Case H; Elim plus_n_Sm; Apply (f_equal nat nat S).
Pattern 1 3 m; Elim m; Simpl; Auto.
Qed.
Hints Resolve mult_n_Sm : core v62.