Skip to content

Commit

Permalink
feat: finite-dimensional manifolds are locally compact (#7822)
Browse files Browse the repository at this point in the history
... assuming they're modelled over a locally compact field. (Currently, the only such instances in mathlib are $\mathbb{R}$ and $\mathbb{C}$. Once local compactness of the $p$-adic numbers is added to mathlib, this theorem will apply to them also.)

- part of the road towards Sard's theorem
  • Loading branch information
grunweg committed Nov 3, 2023
1 parent a717942 commit 36d7949
Showing 1 changed file with 18 additions and 0 deletions.
18 changes: 18 additions & 0 deletions Mathlib/Geometry/Manifold/SmoothManifoldWithCorners.lean
Expand Up @@ -1563,3 +1563,21 @@ theorem writtenInExtChartAt_chartAt_symm_comp [ChartedSpace H H'] (x : M') {y}
simp_all only [mfld_simps, chartAt_comp]

end ExtendedCharts

section Topology
-- Let `M` be a topological manifold over the field π•œ.
variable
{E : Type*} {π•œ : Type*} [NontriviallyNormedField π•œ]
[NormedAddCommGroup E] [NormedSpace π•œ E] {H : Type*} [TopologicalSpace H]
(I : ModelWithCorners π•œ E H) {M : Type*} [TopologicalSpace M] [ChartedSpace H M]
[HasGroupoid M (contDiffGroupoid 0 I)]

/-- A finite-dimensional manifold modelled on a locally compact field
(such as ℝ, β„‚ or the `p`-adic numbers) is locally compact. -/
lemma Manifold.locallyCompact_of_finiteDimensional [LocallyCompactSpace π•œ]
[FiniteDimensional π•œ E] : LocallyCompactSpace M := by
have : ProperSpace E := FiniteDimensional.proper π•œ E
have : LocallyCompactSpace H := I.locallyCompactSpace
exact ChartedSpace.locallyCompactSpace H M

end Topology

0 comments on commit 36d7949

Please sign in to comment.