Skip to content

Commit

Permalink
Preliminary definitions
Browse files Browse the repository at this point in the history
  • Loading branch information
siraben committed May 24, 2021
1 parent 995aecf commit 2e7cc35
Showing 1 changed file with 65 additions and 1 deletion.
66 changes: 65 additions & 1 deletion theories/Topology/Manifolds.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,9 @@
From Topology Require Import Homeomorphisms SubspaceTopology EuclideanSpaces.
Require Import Homeomorphisms.
Require Import SubspaceTopology.
Require Import EuclideanSpaces.
Require Import CountabilityAxioms.
Require Import SeparatednessAxioms.
Require Export Ensembles.

Definition restriction {X Y: Type} (f : X -> Y) (U : Ensemble X): {x | U x} -> {y | Im U f y}.
intro x.
Expand All @@ -17,3 +22,62 @@ Inductive local_homeomorphism {X Y : TopologicalSpace}
@homeomorphism (SubspaceTopology U) (SubspaceTopology (Im U f)) (restriction f U)) ->
local_homeomorphism f.

Inductive locally_homeomorphic (X Y:TopologicalSpace) : Prop :=
| intro_locally_homeomorphic: forall f:point_set X -> point_set Y,
local_homeomorphism f -> locally_homeomorphic X Y.


Lemma locally_homeomorphic_refl (X : TopologicalSpace) : locally_homeomorphic X X.
Proof.
apply intro_locally_homeomorphic with (f := (fun x => x)).
constructor.
intros x.
exists Full_set.
split.
- repeat constructor. apply open_full.
- split.
+ assert (surjective (fun x : X => x)).
{
econstructor.
reflexivity.
}
rewrite <- Im_Full_set_surj.
* apply open_full.
* assumption.
+ econstructor.
* admit.
* admit.
* admit.
* admit.
Admitted.

Definition Manifold (X:TopologicalSpace) (n : nat) : Prop :=
second_countable X /\ Hausdorff X
/\ locally_homeomorphic X (EuclideanSpace n).

(* R^n is a manifold *)

Require Import MetricSpaces.

Theorem EuclideanManifold (n : nat) : Manifold (EuclideanSpace n) n.
Proof.
constructor.
- (* need proof that second_countable (EuclideanSpace n) *)
admit.
- split.
+ (* need proof that R^n is Hausdorff *)
admit.
+ apply locally_homeomorphic_refl.
Admitted.

Theorem SphereManifold (n : nat) : Manifold (Sphere (S n)) n.
Proof.
constructor.
- (* provide an atlas for the sphere *)
admit.
- split.
+ (* sphere is Hausdorff *)
admit.
+ (* sphere is locally homeomorphic to R^n *)
admit.
Admited.

0 comments on commit 2e7cc35

Please sign in to comment.