From 8c63a877eb0908513b75e2b5e6ac1cd998547089 Mon Sep 17 00:00:00 2001 From: herbelin Date: Wed, 24 Sep 2003 08:54:16 +0000 Subject: Destruct/Induction -> NewDestruct/NewInduction git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4469 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Arith/Plus.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/Arith/Plus.v') diff --git a/theories/Arith/Plus.v b/theories/Arith/Plus.v index 2285c544c..843ba0739 100755 --- a/theories/Arith/Plus.v +++ b/theories/Arith/Plus.v @@ -176,6 +176,6 @@ Fixpoint plus_acc [q,n:nat] : nat := Definition tail_plus := [n,m:nat](plus_acc m n). Lemma plus_tail_plus : (n,m:nat)(n+m)=(tail_plus n m). -Induction n; Unfold tail_plus; Simpl; Auto. -Intros p H m; Rewrite <- H; Simpl; Auto. +Unfold tail_plus; NewInduction n as [|n IHn]; Simpl; Auto. +Intro m; Rewrite <- IHn; Simpl; Auto. Qed. -- cgit v1.2.3