aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Wf_nat.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
commite10135925fa344ead0eb760c2c0fb7167d8dfc74 (patch)
treec00f1058346af155c3f54a297b452a1edd640197 /theories/Arith/Wf_nat.v
parent634d52825790d8818883549616b3c8807655d2b8 (diff)
Independance vis a vis noms variables liees; partie sur bool dans Zbool
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4876 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Wf_nat.v')
-rwxr-xr-xtheories/Arith/Wf_nat.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Arith/Wf_nat.v b/theories/Arith/Wf_nat.v
index e87f436ed..51df19b29 100755
--- a/theories/Arith/Wf_nat.v
+++ b/theories/Arith/Wf_nat.v
@@ -133,7 +133,7 @@ Defined.
Lemma lt_wf_ind : (p:nat)(P:nat->Prop)
((n:nat)((m:nat)(lt m n)->(P m))->(P n)) -> (P p).
-Intros; Elim (lt_wf p); Auto with arith.
+Intro p; Intros; Elim (lt_wf p); Auto with arith.
Qed.
Lemma gt_wf_rec : (p:nat)(P:nat->Set)
@@ -151,7 +151,7 @@ Lemma lt_wf_double_rec :
((n,m:nat)((p,q:nat)(lt p n)->(P p q))->((p:nat)(lt p m)->(P n p))->(P n m))
-> (p,q:nat)(P p q).
Intros P Hrec p; Pattern p; Apply lt_wf_rec.
-Intros; Pattern q; Apply lt_wf_rec; Auto with arith.
+Intros n H q; Pattern q; Apply lt_wf_rec; Auto with arith.
Defined.
Lemma lt_wf_double_ind :
@@ -159,7 +159,7 @@ Lemma lt_wf_double_ind :
((n,m:nat)((p,q:nat)(lt p n)->(P p q))->((p:nat)(lt p m)->(P n p))->(P n m))
-> (p,q:nat)(P p q).
Intros P Hrec p; Pattern p; Apply lt_wf_ind.
-Intros; Pattern q; Apply lt_wf_ind; Auto with arith.
+Intros n H q; Pattern q; Apply lt_wf_ind; Auto with arith.
Qed.
Hints Resolve lt_wf : arith.