Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
move lemmas to better place
Browse files Browse the repository at this point in the history
  • Loading branch information
winstonyin committed Jan 5, 2023
1 parent 69338e9 commit 6f3d20d
Show file tree
Hide file tree
Showing 2 changed files with 32 additions and 33 deletions.
33 changes: 0 additions & 33 deletions src/geometry/manifold/integral_curve.lean
Original file line number Diff line number Diff line change
Expand Up @@ -38,39 +38,6 @@ localized "notation (name := ext_chart_at) `𝓔(` I `, ` x `)` :=

open_locale manifold

namespace model_with_corners

variables
{𝕜 : Type*} [nontrivially_normed_field 𝕜]
{E : Type*} [normed_add_comm_group E] [normed_space 𝕜 E]
{H : Type*} [topological_space H] (I : model_with_corners 𝕜 E H)
{M : Type*} [topological_space M] [charted_space H M]

lemma boundaryless.is_open_target
[I.boundaryless] {x : M} : is_open (ext_chart_at I x).target :=
begin
rw [ext_chart_at_target, model_with_corners.boundaryless.range_eq_univ, set.inter_univ],
exact (model_with_corners.continuous_symm _).is_open_preimage _ (local_homeomorph.open_target _)
end

/-- An interior point of a manifold is a point whose image in the model vector space is in the
interior of the chart's target.
TODO : This definition refers to a chosen chart at `x`, but the property is independent of the
choice of chart. See Theorem 1.37 (for general manifolds) and Theorem 1.46 (for smooth manifolds) of
Introduction to Smooth Manifolds by John M. Lee.
-/
def is_interior_point (x : M) := 𝓔(I, x) x ∈ interior 𝓔(I, x).target

lemma boundaryless.is_interior_point
[I.boundaryless] {x : M} : I.is_interior_point x :=
begin
rw [is_interior_point, is_open.interior_eq (boundaryless.is_open_target I)],
exact local_equiv.map_source _ (mem_ext_chart_source _ _)
end

end model_with_corners

section

variables
Expand Down
32 changes: 32 additions & 0 deletions src/geometry/manifold/smooth_manifold_with_corners.lean
Original file line number Diff line number Diff line change
Expand Up @@ -971,3 +971,35 @@ lemma ext_chart_at_prod (x : M × M') :
by simp only with mfld_simps

end extended_charts

namespace model_with_corners

variables
{𝕜 : Type*} [nontrivially_normed_field 𝕜]
{E : Type*} [normed_add_comm_group E] [normed_space 𝕜 E]
{H : Type*} [topological_space H] (I : model_with_corners 𝕜 E H)
{M : Type*} [topological_space M] [charted_space H M]

lemma boundaryless.is_open_target
[I.boundaryless] {x : M} : is_open (ext_chart_at I x).target :=
begin
rw [ext_chart_at_target, model_with_corners.boundaryless.range_eq_univ, set.inter_univ],
exact (model_with_corners.continuous_symm _).is_open_preimage _ (local_homeomorph.open_target _)
end

/-- An interior point of a manifold is a point whose image in the model vector space is in the
interior of the chart's target.
TODO : This definition refers to a chosen chart at `x`, but the property is independent of the
choice of chart for finite-dimensional real manifolds. See Theorem 1.37 (for general manifolds) and
Theorem 1.46 (for smooth manifolds) of Introduction to Smooth Manifolds by John M. Lee. -/
def is_interior_point (x : M) := ext_chart_at I x x ∈ interior (ext_chart_at I x).target

lemma boundaryless.is_interior_point
[I.boundaryless] {x : M} : I.is_interior_point x :=
begin
rw [is_interior_point, is_open.interior_eq (boundaryless.is_open_target I)],
exact local_equiv.map_source _ (mem_ext_chart_source _ _)
end

end model_with_corners

0 comments on commit 6f3d20d

Please sign in to comment.