aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Factorial.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:07 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:07 +0000
commitd56cb8c2382bc0c109e84d46bff9762275da38a5 (patch)
treef52bc569f066eaec2819512f5db47dd2b6820e30 /theories/Arith/Factorial.v
parente10135925fa344ead0eb760c2c0fb7167d8dfc74 (diff)
Noms canoniques pour les variables liees
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4877 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Factorial.v')
-rw-r--r--theories/Arith/Factorial.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Arith/Factorial.v b/theories/Arith/Factorial.v
index ca176a6c6..1d1ee00af 100644
--- a/theories/Arith/Factorial.v
+++ b/theories/Arith/Factorial.v
@@ -37,15 +37,15 @@ Apply lt_O_neq.
Apply lt_O_fact.
Qed.
-Lemma fact_growing : (m,n:nat) (le m n) -> (le (fact m) (fact n)).
+Lemma fact_growing : (n,m:nat) (le n m) -> (le (fact n) (fact m)).
Proof.
NewInduction 1.
Apply le_n.
-Assert (le (mult (S O) (fact m)) (mult (S m0) (fact m0))).
+Assert (le (mult (S O) (fact n)) (mult (S m) (fact m))).
Apply le_mult_mult.
Apply lt_le_S; Apply lt_O_Sn.
Assumption.
-Simpl (mult (S O) (fact m)) in H0.
+Simpl (mult (S O) (fact n)) in H0.
Rewrite <- plus_n_O in H0.
Assumption.
Qed.