Skip to content

Commit

Permalink
doc: add docstrings for ChartedSpace.{atlas,chartAt} and their aliases (
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Feb 6, 2024
1 parent f43e781 commit 9712171
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Geometry/Manifold/ChartedSpace.lean
Expand Up @@ -555,16 +555,20 @@ sometimes as a real manifold over `ℝ^(2n)`.
-/
@[ext]
class ChartedSpace (H : Type*) [TopologicalSpace H] (M : Type*) [TopologicalSpace M] where
/-- The atlas of charts in the `ChartedSpace`. -/
protected atlas : Set (PartialHomeomorph M H)
/-- The preferred chart at each point in the charted space. -/
protected chartAt : M → PartialHomeomorph M H
protected mem_chart_source : ∀ x, x ∈ (chartAt x).source
protected chart_mem_atlas : ∀ x, chartAt x ∈ atlas
#align charted_space ChartedSpace

/-- The atlas of charts in a `ChartedSpace`. -/
abbrev atlas (H : Type*) [TopologicalSpace H] (M : Type*) [TopologicalSpace M]
[ChartedSpace H M] : Set (PartialHomeomorph M H) :=
ChartedSpace.atlas

/-- The preferred chart at a point `x` in a charted space `M`. -/
abbrev chartAt (H : Type*) [TopologicalSpace H] {M : Type*} [TopologicalSpace M]
[ChartedSpace H M] (x : M) : PartialHomeomorph M H :=
ChartedSpace.chartAt x
Expand Down
4 changes: 0 additions & 4 deletions scripts/nolints.json
Expand Up @@ -43,13 +43,11 @@
["docBlame", "WriterT"],
["docBlame", "Xor'"],
["docBlame", "Zero"],
["docBlame", "atlas"],
["docBlame", "bit0"],
["docBlame", "bit1"],
["docBlame", "cancelDenominators"],
["docBlame", "cancelDenominatorsAt"],
["docBlame", "cancelDenominatorsTarget"],
["docBlame", "chartAt"],
["docBlame", "condM"],
["docBlame", "decidableEq_of_bool_pred"],
["docBlame", "eqns"],
Expand Down Expand Up @@ -121,8 +119,6 @@
["docBlame", "Cardinal.term𝔠"],
["docBlame", "CategoryTheory.«term_⟶[_]_»"],
["docBlame", "ChangeOfRings.«term_⊗ₜ[_,_]_»"],
["docBlame", "ChartedSpace.atlas"],
["docBlame", "ChartedSpace.chartAt"],
["docBlame", "ChartedSpaceCore.atlas"],
["docBlame", "ChartedSpaceCore.chartAt"],
["docBlame", "Combinator.I"],
Expand Down

0 comments on commit 9712171

Please sign in to comment.