aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ConstructiveEpsilon.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-22 18:48:21 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-22 18:48:21 +0000
commit5126dd10446860c28d8c586dd12180abf1512953 (patch)
treea5a89c868aee9befb32bb070f196b33fedb0efac /theories/Logic/ConstructiveEpsilon.v
parent62c5b810b7728b5cd1c2ebd927f03dcb6fbf61d1 (diff)
Backported r13308 (ConstructiveEpsilon.v) to branch v8.3
Also removed trailing spaces of the file git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13309 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 8352dde63..6a242ac8b 100644
--- a/theories/Logic/ConstructiveEpsilon.v
+++ b/theories/Logic/ConstructiveEpsilon.v
@@ -77,7 +77,7 @@ Fixpoint linear_search m (b : before_witness m) : {n : nat | P n} :=
| right no => linear_search (S m) (inv_before_witness m b no)
end.
-Definition constructive_indefinite_description_nat :
+Definition constructive_indefinite_description_nat :
(exists n, P n) -> {n:nat | P n} :=
fun e => linear_search O (let (n, p) := e in O_witness n (stop n p)).
@@ -99,9 +99,9 @@ Hypothesis P_decidable : forall n : nat, {P n} + {~ P n}.
given relation [R]. An element is accessible if there are no infinite
[R]-descending chains starting from it.
-To use [Fix_F], we define a relation R and prove that if [exists n, P 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}].
+definition of [Acc R 0], we show [{n : nat | P n}].
The relation [R] describes the connection between the two successive
numbers we try. Namely, [y] is [R]-less then [x] if we try [y] after