aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-10-05 15:52:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-10-05 15:52:05 +0000
commite9d06d5adf1f941aff4aeb9eaef0f92f7cf96693 (patch)
treee53d657dbd2d55a6775366123eda6ab6d8ddbae2
parent8082d1faf85a0ab29f6c144a137791902a4e9c1f (diff)
Removing vernacular code mistakenly committed.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14515 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--theories/Logic/ExtensionalityFacts.v36
1 files changed, 0 insertions, 36 deletions
diff --git a/theories/Logic/ExtensionalityFacts.v b/theories/Logic/ExtensionalityFacts.v
index 631177beb..421bbebcf 100644
--- a/theories/Logic/ExtensionalityFacts.v
+++ b/theories/Logic/ExtensionalityFacts.v
@@ -36,42 +36,6 @@ Set Implicit Arguments.
Definition is_inverse A B f g := (forall a:A, g (f a) = a) /\ (forall b:B, f (g b) = b).
-Definition iscontr (X:Type) := {x:X| forall y, x=y}.
-Definition hfiber X Y (f:X -> Y) (y:Y) := {x:X| f x=y}.
-Definition isweq X Y (f:X -> Y) := forall y, iscontr (hfiber f y).
-
-Goal forall X Y (f:X->Y), isweq f -> {g|is_inverse f g}.
-Proof.
- intros * Hweq.
- set (g:=fun y => proj1_sig (proj1_sig (Hweq y))).
- exists g. split.
- - intro x. unfold g. destruct (Hweq (f x)) as ((x0,Hx0),Hxy). simpl.
- set (fiber0 := exist (fun x0 => f x0 = f x) x0 Hx0) in *.
- set (fiber := exist (fun x0 => f x0 = f x) x eq_refl).
- change (proj1_sig fiber0 = proj1_sig fiber).
- specialize Hxy with fiber.
- destruct Hxy.
- reflexivity.
- - intro y.
- unfold g.
- destruct (Hweq y) as ((x,Hxy),Hyuniq). simpl. assumption.
-Qed.
-
-Goal forall X Y (f:X->Y), {g|is_inverse f g} -> isweq f.
-Proof.
- destruct 1 as (g,(Hgf,Hfg)).
- intro y.
- set (fiber := exist (fun x => f x = y) (g y) (Hfg y)).
- exists fiber.
- destruct y0 as (y0,Hfy0).
- unfold fiber.
- rewrite <- Hfy0 in *.
- assert (forall y, f_equal f (Hgf y) = Hfg (f y)). admit.
- rewrite <- H.
- rewrite Hgf.
- reflexivity.
-Qed.
-
(** The diagonal over A and the one-one correspondence with A *)
Record Delta A := { pi1:A; pi2:A; eq:pi1=pi2 }.