Skip to content

Commit 32831aa

Browse files
committed
doc(Topology): fix typos (#32659)
Typos found and fixed by Codex.
1 parent e49e021 commit 32831aa

File tree

14 files changed

+36
-36
lines changed

14 files changed

+36
-36
lines changed

Mathlib/Topology/Algebra/InfiniteSum/UniformOn.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ public import Mathlib.Order.Filter.AtTopBot.Finset
1212
/-!
1313
# Infinite sum and products that converge uniformly
1414
15-
# Main definitions
15+
## Main definitions
1616
- `HasProdUniformlyOn f g s` : `∏ i, f i b` converges uniformly on `s` to `g`.
1717
- `HasProdLocallyUniformlyOn f g s` : `∏ i, f i b` converges locally uniformly on `s` to `g`.
1818
- `HasProdUniformly f g` : `∏ i, f i b` converges uniformly to `g`.

Mathlib/Topology/Bases.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -45,7 +45,7 @@ conditions are equivalent in this case).
4545
the space.
4646
4747
## Implementation Notes
48-
For our applications we are interested that there exists a countable basis, but we do not need the
48+
For our applications we are interested in the existence of a countable basis, but we do not need the
4949
concrete basis itself. This allows us to declare these type classes as `Prop` to use them as mixins.
5050
5151
## TODO

Mathlib/Topology/EMetricSpace/PairReduction.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -57,9 +57,9 @@ natural number `k` greater than zero such that `|{x ∈ V | d(t, x) ≤ kc}| ≤
5757
We construct a sequence `Vᵢ` of subsets of `J`, a sequence `tᵢ ∈ Vᵢ` and a sequence of `rᵢ : ℕ`
5858
inductively as follows (see `logSizeBallSeq`):
5959
60-
* `V₀ = J`, `tₒ` is chosen arbitrarily in `J`, `r₀` is the log-size radius of `t₀` in `V₀`
61-
* `Vᵢ₊ = Vᵢ \ Bᵢ` where `Bᵢ := {x ∈ V | d(t, x) ≤ (rᵢ - 1) c}`, `tᵢ₊₁` is chosen arbitrarily in
62-
`Vᵢ₊₁` (if it is nonempty), `rᵢ₊₁` is the log-size radius of `tᵢ₊₁` in `Vᵢ₊`.
60+
* `V₀ = J`, `t₀` is chosen arbitrarily in `J`, `r₀` is the log-size radius of `t₀` in `V₀`
61+
* `Vᵢ₊ = Vᵢ \ Bᵢ` where `Bᵢ := {x ∈ V | d(t, x) ≤ (rᵢ - 1) c}`, `tᵢ₊₁` is chosen arbitrarily in
62+
`Vᵢ₊₁` (if it is nonempty), `rᵢ₊₁` is the log-size radius of `tᵢ₊₁` in `Vᵢ₊`.
6363
6464
Then `Vᵢ` is a strictly decreasing sequence (see `card_finset_logSizeBallSeq_add_one_lt`) until
6565
`Vᵢ` is empty. In particular `Vᵢ = ∅` for `i ≥ |J|`
@@ -176,9 +176,9 @@ def logSizeBallStruct.ball (struct : logSizeBallStruct T) (c : ℝ≥0∞) :
176176
variable [DecidableEq T]
177177

178178
/-- We recursively define a log-size ball sequence `(Vᵢ, tᵢ, rᵢ)` by
179-
* `V₀ = J`, `tₒ` is chosen arbitrarily in `J`, `r₀` is the log-size radius of `t₀` in `V₀`
180-
* `Vᵢ₊ = Vᵢ \ {x ∈ V | d(t, x) ≤ (rᵢ - 1)c}`, `tᵢ₊₁` is chosen arbitrarily in `Vᵢ₊₁, rᵢ₊₁` is
181-
the log-size radius of `tᵢ₊₁` in `Vᵢ₊`. -/
179+
* `V₀ = J`, `t₀` is chosen arbitrarily in `J`, `r₀` is the log-size radius of `t₀` in `V₀`
180+
* `Vᵢ₊ = Vᵢ \ {x ∈ V | d(t, x) ≤ (rᵢ - 1)c}`, `tᵢ₊₁` is chosen arbitrarily in `Vᵢ₊₁`, `rᵢ₊₁` is
181+
the log-size radius of `tᵢ₊₁` in `Vᵢ₊`. -/
182182
noncomputable
183183
def logSizeBallSeq (J : Finset T) (hJ : J.Nonempty) (a c : ℝ≥0∞) : ℕ → logSizeBallStruct T
184184
| 0 => {finset := J, point := hJ.choose, radius := logSizeRadius hJ.choose J a c}

Mathlib/Topology/Homotopy/HSpaces.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -14,16 +14,16 @@ public import Mathlib.Topology.Path
1414
1515
This file defines H-spaces mainly following the approach proposed by Serre in his paper
1616
*Homologie singulière des espaces fibrés*. The idea beneath `H-spaces` is that they are topological
17-
spaces with a binary operation `⋀ : X → X → X` that is a homotopic-theoretic weakening of an
18-
operation what would make `X` into a topological monoid.
19-
In particular, there exists a "neutral element" `e : X` such that `fun x ↦e ⋀ x` and
17+
spaces with a binary operation `⋀ : X → X → X` that is a homotopy-theoretic weakening of an
18+
operation that would make `X` into a topological monoid.
19+
In particular, there exists a "neutral element" `e : X` such that `fun x ↦ e ⋀ x` and
2020
`fun x ↦ x ⋀ e` are homotopic to the identity on `X`, see
2121
[the Wikipedia page of H-spaces](https://en.wikipedia.org/wiki/H-space).
2222
2323
Some notable properties of `H-spaces` are
2424
* Their fundamental group is always abelian (by the same argument for topological groups);
2525
* Their cohomology ring comes equipped with a structure of a Hopf-algebra;
26-
* The loop space based at every `x : X` carries a structure of an `H-spaces`.
26+
* The loop space based at every `x : X` carries a structure of an `H-space`.
2727
2828
## Main Results
2929
@@ -32,14 +32,14 @@ Some notable properties of `H-spaces` are
3232
* Given two `H-spaces` `X` and `Y`, their product is again an `H`-space. We show in an example that
3333
starting with two topological groups `G, G'`, the `H`-space structure on `G × G'` is
3434
definitionally equal to the product of `H-space` structures on `G` and `G'`.
35-
* The loop space based at every `x : X` carries a structure of an `H-spaces`.
35+
* The loop space based at every `x : X` carries a structure of an `H-space`.
3636
3737
## To Do
3838
* Prove that for every `NormedAddTorsor Z` and every `z : Z`, the operation
3939
`fun x y ↦ midpoint x y` defines an `H-space` structure with `z` as a "neutral element".
4040
* Prove that `S^0`, `S^1`, `S^3` and `S^7` are the unique spheres that are `H-spaces`, where the
4141
first three inherit the structure because they are topological groups (they are Lie groups,
42-
actually), isomorphic to the invertible elements in `ℤ`, in `ℂ` and in the quaternion; and the
42+
actually), isomorphic to the invertible elements in `ℤ`, in `ℂ` and in the quaternions; and the
4343
fourth from the fact that `S^7` coincides with the octonions of norm 1 (it is not a group, in
4444
particular, only has an instance of `MulOneClass`).
4545

Mathlib/Topology/MetricSpace/Bounded.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -336,7 +336,7 @@ theorem isBounded_Ioc (a b : α) : IsBounded (Ioc a b) :=
336336
theorem isBounded_Ioo (a b : α) : IsBounded (Ioo a b) :=
337337
(totallyBounded_Ioo a b).isBounded
338338

339-
/-- In a pseudo metric space with a conditionally complete linear order such that the order and the
339+
/-- In a pseudometric space with a conditionally complete linear order such that the order and the
340340
metric structure give the same topology, any order-bounded set is metric-bounded. -/
341341
theorem isBounded_of_bddAbove_of_bddBelow {s : Set α} (h₁ : BddAbove s) (h₂ : BddBelow s) :
342342
IsBounded s :=

Mathlib/Topology/MetricSpace/Gluing.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -450,7 +450,7 @@ variable {X : Type u} {Y : Type v} {Z : Type w}
450450
variable [Nonempty Z] [MetricSpace Z] [MetricSpace X] [MetricSpace Y] {Φ : Z → X} {Ψ : Z → Y}
451451
{ε : ℝ}
452452

453-
/-- Given two isometric embeddings `Φ : Z → X` and `Ψ : Z → Y`, we define a pseudo metric space
453+
/-- Given two isometric embeddings `Φ : Z → X` and `Ψ : Z → Y`, we define a pseudometric space
454454
structure on `X ⊕ Y` by declaring that `Φ x` and `Ψ x` are at distance `0`. -/
455455
def gluePremetric (hΦ : Isometry Φ) (hΨ : Isometry Ψ) : PseudoMetricSpace (X ⊕ Y) where
456456
dist := glueDist Φ Ψ 0

Mathlib/Topology/MetricSpace/PiNat.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -810,7 +810,7 @@ attribute [scoped instance] PiCountable.edist
810810
section PseudoEMetricSpace
811811
variable [∀ i, PseudoEMetricSpace (F i)]
812812

813-
/-- Given a countable family of extended pseudo metric spaces,
813+
/-- Given a countable family of extended pseudometric spaces,
814814
one may put an extended distance on their product `Π i, E i`.
815815
816816
It is highly non-canonical, though, and therefore not registered as a global instance.

Mathlib/Topology/MetricSpace/ProperSpace.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -60,7 +60,7 @@ instance Metric.sphere.compactSpace {α : Type*} [PseudoMetricSpace α] [ProperS
6060
variable [PseudoMetricSpace α]
6161

6262
-- see Note [lower instance priority]
63-
/-- A proper pseudo metric space is sigma compact, and therefore second countable. -/
63+
/-- A proper pseudometric space is sigma compact, and therefore second countable. -/
6464
instance (priority := 100) secondCountable_of_proper [ProperSpace α] :
6565
SecondCountableTopology α := by
6666
-- We already have `sigmaCompactSpace_of_locallyCompact_secondCountable`, so we don't

Mathlib/Topology/MetricSpace/Pseudo/Defs.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -133,7 +133,7 @@ class PseudoMetricSpace (α : Type u) : Type u extends Dist α where
133133
cobounded_sets : (Bornology.cobounded α).sets =
134134
{ s | ∃ C : ℝ, ∀ x ∈ sᶜ, ∀ y ∈ sᶜ, dist x y ≤ C } := by intros; rfl
135135

136-
/-- Two pseudo metric space structures with the same distance function coincide. -/
136+
/-- Two pseudometric space structures with the same distance function coincide. -/
137137
@[ext]
138138
theorem PseudoMetricSpace.ext {α : Type*} {m m' : PseudoMetricSpace α}
139139
(h : m.toDist = m'.toDist) : m = m' := by
@@ -990,7 +990,7 @@ example {α} [U : UniformSpace α] (m : PseudoMetricSpace α)
990990
(PseudoMetricSpace.replaceUniformity m H).toBornology = m.toBornology := by
991991
with_reducible_and_instances rfl
992992

993-
/-- Build a new pseudo metric space from an old one where the bundled topological structure is
993+
/-- Build a new pseudometric space from an old one where the bundled topological structure is
994994
provably (but typically non-definitionaly) equal to some given topological structure.
995995
See Note [forgetful inheritance].
996996
See Note [reducible non-instances].

Mathlib/Topology/Metrizable/Basic.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -29,7 +29,7 @@ namespace TopologicalSpace
2929
variable {ι X Y : Type*} {A : ι → Type*} [TopologicalSpace X] [TopologicalSpace Y] [Finite ι]
3030
[∀ i, TopologicalSpace (A i)]
3131

32-
/-- A topological space is *pseudo metrizable* if there exists a pseudo metric space structure
32+
/-- A topological space is *pseudometrizable* if there exists a pseudometric space structure
3333
compatible with the topology. To minimize imports, we implement this class in terms of the
3434
existence of a countably generated unifomity inducing the topology, which is mathematically
3535
equivalent.
@@ -41,7 +41,7 @@ class PseudoMetrizableSpace (X : Type*) [t : TopologicalSpace X] : Prop where
4141
exists_countably_generated :
4242
∃ u : UniformSpace X, u.toTopologicalSpace = t ∧ (uniformity X).IsCountablyGenerated
4343

44-
/-- A uniform space with countably generated `𝓤 X` is pseudo metrizable. -/
44+
/-- A uniform space with countably generated `𝓤 X` is pseudometrizable. -/
4545
instance (priority := 100) _root_.UniformSpace.pseudoMetrizableSpace {X : Type*}
4646
[u : UniformSpace X] [hu : IsCountablyGenerated (uniformity X)] : PseudoMetrizableSpace X :=
4747
⟨⟨u, rfl, hu⟩⟩
@@ -75,8 +75,8 @@ instance pseudoMetrizableSpace_prod [PseudoMetrizableSpace X] [PseudoMetrizableS
7575
pseudoMetrizableSpaceUniformity_countably_generated Y
7676
inferInstance
7777

78-
/-- Given an inducing map of a topological space into a pseudo metrizable space, the source space
79-
is also pseudo metrizable. -/
78+
/-- Given an inducing map of a topological space into a pseudometrizable space, the source space
79+
is also pseudometrizable. -/
8080
theorem _root_.Topology.IsInducing.pseudoMetrizableSpace [PseudoMetrizableSpace Y] {f : X → Y}
8181
(hf : IsInducing f) : PseudoMetrizableSpace X :=
8282
let u : UniformSpace Y := pseudoMetrizableSpaceUniformity Y

0 commit comments

Comments
 (0)