aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Between.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-24 08:54:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-24 08:54:16 +0000
commit8c63a877eb0908513b75e2b5e6ac1cd998547089 (patch)
treef7cd0f8e518de0ccd3bf1b63faa5eeae53d9fa13 /theories/Arith/Between.v
parent217ff530701d5fc3467659f093227680906c1c9a (diff)
Destruct/Induction -> NewDestruct/NewInduction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4469 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Between.v')
-rwxr-xr-xtheories/Arith/Between.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Between.v b/theories/Arith/Between.v
index 2d5104af2..14b245335 100755
--- a/theories/Arith/Between.v
+++ b/theories/Arith/Between.v
@@ -42,7 +42,7 @@ Lemma between_Sk_l : (k,l:nat)(between k l)->(le (S k) l)->(between (S k) l).
Proof.
NewInduction 1.
Intros; Absurd (le (S k) k); Auto with arith.
-Induction H; Auto with arith.
+NewDestruct H; Auto with arith.
Qed.
Hints Resolve between_Sk_l : arith v62.