aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ConstructiveEpsilon.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-23 11:38:38 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-23 11:38:38 +0000
commit32c11b16f7d7ff0ea3aee584103bd60f5b94dedb (patch)
treebee8e00e6f0b19cab2de4c20217e4933deafd28b /theories/Logic/ConstructiveEpsilon.v
parentf7cd707fe388f0cfd990664c18a2d09d49890744 (diff)
Nettoyage Wf.v et unification (suite remarques faites sur cocorico)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10712 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/ConstructiveEpsilon.v')
-rw-r--r--theories/Logic/ConstructiveEpsilon.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Logic/ConstructiveEpsilon.v b/theories/Logic/ConstructiveEpsilon.v
index 36ff2681b..322f2d9be 100644
--- a/theories/Logic/ConstructiveEpsilon.v
+++ b/theories/Logic/ConstructiveEpsilon.v
@@ -20,14 +20,14 @@ show [{n : nat | P n}]. However, one can perform a recursion on an
inductive predicate in sort [Prop] so that the returning type of the
recursion is in [Set]. This trick is described in Coq'Art book, Sect.
14.2.3 and 15.4. In particular, this trick is used in the proof of
-[Acc_iter] in the module Coq.Init.Wf. There, recursion is done on an
+[Fix_F] in the module Coq.Init.Wf. There, recursion is done on an
inductive predicate [Acc] and the resulting type is in [Type].
The predicate [Acc] delineates elements that are accessible via a
given relation [R]. An element is accessible if there are no infinite
[R]-descending chains starting from it.
-To use [Acc_iter], we define a relation R and prove that if [exists n,
+To use [Fix_F], we define a relation R and prove that if [exists n,
P n] then 0 is accessible with respect to R. Then, by induction on the
definition of [Acc R 0], we show [{n : nat | P n}]. *)
@@ -79,7 +79,7 @@ Defined.
Theorem acc_implies_P_eventually : acc 0 -> {n : nat | P n}.
Proof.
-intros Acc_0. pattern 0. apply Acc_iter with (R := R); [| assumption].
+intros Acc_0. pattern 0. apply Fix_F with (R := R); [| assumption].
clear Acc_0; intros x IH.
destruct (P_decidable x) as [Px | not_Px].
exists x; simpl; assumption.