Skip to content

Commit

Permalink
Prove that id is a homeomorphism
Browse files Browse the repository at this point in the history
  • Loading branch information
Columbus240 committed Jun 2, 2021
1 parent 702e317 commit 0d14ee2
Showing 1 changed file with 6 additions and 3 deletions.
9 changes: 6 additions & 3 deletions theories/Topology/Homeomorphisms.v
Original file line number Diff line number Diff line change
Expand Up @@ -57,6 +57,11 @@ rewrite H4.
auto.
Qed.

Lemma homeomorphism_id (X : TopologicalSpace) : homeomorphism (@id X).
Proof.
exists id; auto using continuous_identity.
Qed.

Inductive homeomorphic (X Y:TopologicalSpace) : Prop :=
| intro_homeomorphic: forall f:point_set X -> point_set Y,
homeomorphism f -> homeomorphic X Y.
Expand All @@ -67,9 +72,7 @@ From ZornsLemma Require Import Relation_Definitions_Implicit.
Lemma homeomorphic_equiv: equivalence homeomorphic.
Proof.
constructor.
- intro X.
exists id, id; trivial;
apply continuous_identity.
- eexists; eapply homeomorphism_id.
- intros X Y Z ? ?.
destruct H as [f [finv]].
destruct H0 as [g [ginv]].
Expand Down

0 comments on commit 0d14ee2

Please sign in to comment.