aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ClassicalEpsilon.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-09 14:08:38 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-09 14:08:38 +0000
commitca13fb40562c9d664aa4f363755eab6e5f2eeaa5 (patch)
treea58e8cd8dc25955727191de22bf3ac7627a3d27e /theories/Logic/ClassicalEpsilon.v
parent2c1a2d07ab57e257ac84e3ab2c6706b47f52c68d (diff)
Déplacement Int.v dans ZArith, déplacement de DecidableType.v et DecidableTypeEx.v dans Logic
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8933 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/ClassicalEpsilon.v')
-rw-r--r--theories/Logic/ClassicalEpsilon.v24
1 files changed, 15 insertions, 9 deletions
diff --git a/theories/Logic/ClassicalEpsilon.v b/theories/Logic/ClassicalEpsilon.v
index b3efa5fad..79c1e56d2 100644
--- a/theories/Logic/ClassicalEpsilon.v
+++ b/theories/Logic/ClassicalEpsilon.v
@@ -6,9 +6,9 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id:$ i*)
+(*i $Id$ i*)
-(** This file provides classical logic and indefinite description
+(** *** This file provides classical logic and indefinite description
(Hilbert's epsilon operator) *)
(** Classical epsilon's operator (i.e. indefinite description) implies
@@ -25,7 +25,7 @@ Notation Local "'inhabited' A" := A (at level 200, only parsing).
Axiom constructive_indefinite_description :
forall (A : Type) (P : A->Prop),
- (exists x : A, P x) -> { x : A | P x }.
+ (ex P) -> { x : A | P x }.
Lemma constructive_definite_description :
forall (A : Type) (P : A->Prop),
@@ -43,11 +43,11 @@ Qed.
Theorem classical_indefinite_description :
forall (A : Type) (P : A->Prop), inhabited A ->
- { x : A | (exists x : A, P x) -> P x }.
+ { x : A | ex P -> P x }.
Proof.
intros A P i.
destruct (excluded_middle_informative (exists x, P x)) as [Hex|HnonP].
- apply constructive_indefinite_description with (P:= fun x => (exists x, P x) -> P x).
+ apply constructive_indefinite_description with (P:= fun x => ex P -> P x).
destruct Hex as (x,Hx).
exists x; intros _; exact Hx.
firstorder.
@@ -59,9 +59,11 @@ Definition epsilon (A : Type) (i:inhabited A) (P : A->Prop) : A
:= proj1_sig (classical_indefinite_description P i).
Definition epsilon_spec (A : Type) (i:inhabited A) (P : A->Prop) :
- (exists x:A, P x) -> P (epsilon i P)
+ (ex P) -> P (epsilon i P)
:= proj2_sig (classical_indefinite_description P i).
+Opaque epsilon.
+
(** Open question: is classical_indefinite_description constructively
provable from [relational_choice] and
[constructive_definite_description] (at least, using the fact that
@@ -70,7 +72,10 @@ Definition epsilon_spec (A : Type) (i:inhabited A) (P : A->Prop) :
[classical_indefinite_description] is provable (see
[relative_non_contradiction_of_indefinite_desc]). *)
-(** Weaker lemmas (compatibility lemmas) *)
+(** Remark: we use [ex P] rather than [exists x, P x] (which is [ex
+ (fun x => P x)] to ease unification *)
+
+(** *** Weaker lemmas (compatibility lemmas) *)
Theorem choice :
forall (A B : Type) (R : A->B->Prop),
@@ -78,7 +83,8 @@ Theorem choice :
(exists f : A->B, forall x : A, R x (f x)).
Proof.
intros A B R H.
-exists (fun x => proj1_sig (constructive_indefinite_description (R x) (H x))).
+exists (fun x => proj1_sig (constructive_indefinite_description (H x))).
intro x.
-apply (proj2_sig (constructive_indefinite_description (R x) (H x))).
+apply (proj2_sig (constructive_indefinite_description (H x))).
Qed.
+