Skip to content

Commit da6bd14

Browse files
committed
doc: add missing spaces around doc code blocks (#31917)
Issues found and fixed with help from Codex.
1 parent 16e4c58 commit da6bd14

File tree

35 files changed

+44
-44
lines changed

35 files changed

+44
-44
lines changed

Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -754,7 +754,7 @@ theorem ext_of_adjoin_eq_top {s : Set A} (h : adjoin R s = ⊤) ⦃φ₁ φ₂ :
754754
(hs : s.EqOn φ₁ φ₂) : φ₁ = φ₂ :=
755755
ext fun _x => adjoin_le_equalizer φ₁ φ₂ hs <| h.symm ▸ trivial
756756

757-
/-- Two algebra morphisms are equal on `Algebra.span s`iff they are equal on s -/
757+
/-- Two algebra morphisms are equal on `Algebra.span s` iff they are equal on `s`. -/
758758
theorem eqOn_adjoin_iff {φ ψ : A →ₐ[R] B} {s : Set A} :
759759
Set.EqOn φ ψ (adjoin R s) ↔ Set.EqOn φ ψ s := by
760760
have (S : Set A) : S ≤ equalizer φ ψ ↔ Set.EqOn φ ψ S := Iff.rfl

Mathlib/Algebra/Homology/Embedding/Connect.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -177,7 +177,7 @@ noncomputable def homologyIsoPos (n : ℕ) [NeZero n] (m : ℤ) (hm : m = n)
177177
(by simp; cutsat) (by simp; cutsat) (by simp) (by simp)).symm ≪≫
178178
HomologicalComplex.homologyMapIso h.restrictionGEIso n
179179

180-
/-- Given `h : ConnectData K L` and `n : ℕ`non-zero, the homology
180+
/-- Given `h : ConnectData K L` and `n : ℕ` non-zero, the homology
181181
of `h.cochainComplex` in degree `-(n + 1)` identifies to the homology of `K` in degree `n`. -/
182182
noncomputable def homologyIsoNeg (n : ℕ) [NeZero n] (m : ℤ) (hm : m = -(n + 1 : ℕ))
183183
[h.cochainComplex.HasHomology m] [K.HasHomology n] :

Mathlib/Analysis/Calculus/ContDiff/Operations.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -183,7 +183,7 @@ theorem ContDiffAt.add {f g : E → F} (hf : ContDiffAt 𝕜 n f x) (hg : ContDi
183183
ContDiffAt 𝕜 n (fun x => f x + g x) x := by
184184
rw [← contDiffWithinAt_univ] at *; exact hf.add hg
185185

186-
/-- The sum of two `C^n`functions is `C^n`. -/
186+
/-- The sum of two `C^n` functions is `C^n`. -/
187187
@[fun_prop]
188188
theorem ContDiff.add {f g : E → F} (hf : ContDiff 𝕜 n f) (hg : ContDiff 𝕜 n g) :
189189
ContDiff 𝕜 n fun x => f x + g x :=
@@ -264,7 +264,7 @@ theorem ContDiffWithinAt.neg {s : Set E} {f : E → F} (hf : ContDiffWithinAt
264264
theorem ContDiffAt.neg {f : E → F} (hf : ContDiffAt 𝕜 n f x) :
265265
ContDiffAt 𝕜 n (fun x => -f x) x := by rw [← contDiffWithinAt_univ] at *; exact hf.neg
266266

267-
/-- The negative of a `C^n`function is `C^n`. -/
267+
/-- The negative of a `C^n` function is `C^n`. -/
268268
@[fun_prop]
269269
theorem ContDiff.neg {f : E → F} (hf : ContDiff 𝕜 n f) : ContDiff 𝕜 n fun x => -f x :=
270270
contDiff_neg.comp hf
@@ -409,7 +409,7 @@ nonrec theorem ContDiffAt.mul {f g : E → 𝔸} (hf : ContDiffAt 𝕜 n f x) (h
409409
theorem ContDiffOn.mul {f g : E → 𝔸} (hf : ContDiffOn 𝕜 n f s) (hg : ContDiffOn 𝕜 n g s) :
410410
ContDiffOn 𝕜 n (fun x => f x * g x) s := fun x hx => (hf x hx).mul (hg x hx)
411411

412-
/-- The product of two `C^n`functions is `C^n`. -/
412+
/-- The product of two `C^n` functions is `C^n`. -/
413413
@[fun_prop]
414414
theorem ContDiff.mul {f g : E → 𝔸} (hf : ContDiff 𝕜 n f) (hg : ContDiff 𝕜 n g) :
415415
ContDiff 𝕜 n fun x => f x * g x :=

Mathlib/Analysis/Normed/Module/FiniteDimension.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -46,7 +46,7 @@ linear maps are continuous. Moreover, a finite-dimensional subspace is always co
4646
The fact that all norms are equivalent is not written explicitly, as it would mean having two norms
4747
on a single space, which is not the way type classes work. However, if one has a
4848
finite-dimensional vector space `E` with a norm, and a copy `E'` of this type with another norm,
49-
then the identities from `E` to `E'` and from `E'`to `E` are continuous thanks to
49+
then the identities from `E` to `E'` and from `E'` to `E` are continuous thanks to
5050
`LinearMap.continuous_of_finiteDimensional`. This gives the desired norm equivalence.
5151
-/
5252

Mathlib/Analysis/RCLike/Inner.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,7 @@ from `RCLike.innerProductSpace`.
1818
1919
* Build a non-instance `InnerProductSpace` from `wInner`.
2020
* `cWeight` is a poor name. Can we find better? It doesn't hugely matter for typing, since it's
21-
hidden behind the `⟪f, g⟫ₙ_[𝕝] `notation, but it does show up in lemma names
21+
hidden behind the `⟪f, g⟫ₙ_[𝕝]` notation, but it does show up in lemma names
2222
`⟪f, g⟫_[𝕝, cWeight]` is called `wInner_cWeight`. Maybe we should introduce some naming
2323
convention, similarly to `MeasureTheory.average`?
2424
-/

Mathlib/Analysis/SpecialFunctions/Exponential.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -91,7 +91,7 @@ variable {𝕂 𝔸 : Type*} [NontriviallyNormedField 𝕂] [NormedCommRing 𝔸
9191

9292
/-- The exponential map in a commutative Banach algebra `𝔸` over a normed field `𝕂` of
9393
characteristic zero has Fréchet derivative `NormedSpace.exp 𝕂 x • 1 : 𝔸 →L[𝕂] 𝔸`
94-
at any point `x`in the disk of convergence. -/
94+
at any point `x` in the disk of convergence. -/
9595
theorem hasFDerivAt_exp_of_mem_ball [CharZero 𝕂] {x : 𝔸}
9696
(hx : x ∈ EMetric.ball (0 : 𝔸) (expSeries 𝕂 𝔸).radius) :
9797
HasFDerivAt (exp 𝕂) (exp 𝕂 x • (1 : 𝔸 →L[𝕂] 𝔸)) x := by

Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -106,7 +106,7 @@ def LeftExtension.IsPointwiseLeftKanExtension.postcompose
106106
LeftExtension.postcompose₂ L F G |>.obj E |>.IsPointwiseLeftKanExtension := fun c ↦
107107
(hE c).postcompose G
108108

109-
/-- The cocone at a point of the whiskering right by `G`of an extension is isomorphic to the
109+
/-- The cocone at a point of the whiskering right by `G` of an extension is isomorphic to the
110110
action of `G` on the cocone at that point for the original extension. -/
111111
@[simps!]
112112
def LeftExtension.coconeAtWhiskerRightIso (E : LeftExtension L F) (c : C) :
@@ -358,7 +358,7 @@ def RightExtension.IsPointwiseRightKanExtension.postcompose
358358
RightExtension.postcompose₂ L F G |>.obj E |>.IsPointwiseRightKanExtension := fun c ↦
359359
(hE c).postcompose G
360360

361-
/-- The cone at a point of the whiskering right by `G`of an extension is isomorphic to the
361+
/-- The cone at a point of the whiskering right by `G` of an extension is isomorphic to the
362362
action of `G` on the cone at that point for the original extension. -/
363363
@[simps!]
364364
def RightExtension.coneAtWhiskerRightIso (E : RightExtension L F) (c : C) :

Mathlib/CategoryTheory/InducedCategory.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ public import Mathlib.CategoryTheory.Functor.FullyFaithful
1010
/-!
1111
# Induced categories and full subcategories
1212
13-
Given a category `D` and a function `F : C → D `from a type `C` to the
13+
Given a category `D` and a function `F : C → D` from a type `C` to the
1414
objects of `D`, there is an essentially unique way to give `C` a
1515
category structure such that `F` becomes a fully faithful functor,
1616
namely by taking $$ Hom_C(X, Y) = Hom_D(FX, FY) $$. We call this the

Mathlib/CategoryTheory/Sites/Sheaf.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -152,7 +152,7 @@ theorem isLimit_iff_isSheafFor :
152152

153153
/-- Given sieve `S` and presheaf `P : Cᵒᵖ ⥤ A`, their natural associated cone admits at most one
154154
morphism from every cone in the same category (i.e. over the same diagram),
155-
iff `Hom (E, P -)`is separated for the sieve `S` and all `E : A`. -/
155+
iff `Hom (E, P -)` is separated for the sieve `S` and all `E : A`. -/
156156
theorem subsingleton_iff_isSeparatedFor :
157157
(∀ c, Subsingleton (c ⟶ P.mapCone S.arrows.cocone.op)) ↔
158158
∀ E : Aᵒᵖ, IsSeparatedFor (P ⋙ coyoneda.obj E) S.arrows := by

Mathlib/Combinatorics/SetFamily/Compression/Down.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -186,7 +186,7 @@ it suffices to prove it for
186186
* the finset family which only contains the empty finset.
187187
* `{s ∪ {a} | s ∈ 𝒜}` assuming the property for `𝒜` a family of finsets not containing `a`.
188188
* `ℬ ∪ 𝒞` assuming the property for `ℬ` and `𝒞`, where `a` is an element of the ground type and
189-
`ℬ`is a family of finsets not containing `a` and `𝒞` a family of finsets containing `a`.
189+
`ℬ` is a family of finsets not containing `a` and `𝒞` a family of finsets containing `a`.
190190
Note that instead of giving `ℬ` and `𝒞`, the `subfamily` case gives you `𝒜 = ℬ ∪ 𝒞`, so that
191191
`ℬ = {s ∈ 𝒜 | a ∉ s}` and `𝒞 = {s ∈ 𝒜 | a ∈ s}`.
192192

0 commit comments

Comments
 (0)