Skip to content

Commit 3ebc913

Browse files
chore: tidy various files (#6924)
1 parent 3b8d2c9 commit 3ebc913

File tree

10 files changed

+101
-107
lines changed

10 files changed

+101
-107
lines changed

Mathlib/Analysis/NormedSpace/lpSpace.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -816,16 +816,16 @@ instance nonUnitalNormedRing : NonUnitalNormedRing (lp B ∞) :=
816816
mul_le_mul (lp.norm_apply_le_norm ENNReal.top_ne_zero f i)
817817
(lp.norm_apply_le_norm ENNReal.top_ne_zero g i) (norm_nonneg _) (norm_nonneg _) }
818818

819-
-- we also want a `non_unital_normed_comm_ring` instance, but this has to wait for #13719
819+
-- we also want a `NonUnitalNormedCommRing` instance, but this has to wait for mathlib3 #13719
820820
instance infty_isScalarTower {𝕜} [NormedRing 𝕜] [∀ i, Module 𝕜 (B i)] [∀ i, BoundedSMul 𝕜 (B i)]
821821
[∀ i, IsScalarTower 𝕜 (B i) (B i)] : IsScalarTower 𝕜 (lp B ∞) (lp B ∞) :=
822822
fun r f g => lp.ext <| smul_assoc (N := ∀ i, B i) (α := ∀ i, B i) r (⇑f) (⇑g)⟩
823823
#align lp.infty_is_scalar_tower lp.infty_isScalarTower
824824

825-
instance infty_sMulCommClass {𝕜} [NormedRing 𝕜] [∀ i, Module 𝕜 (B i)] [∀ i, BoundedSMul 𝕜 (B i)]
825+
instance infty_smulCommClass {𝕜} [NormedRing 𝕜] [∀ i, Module 𝕜 (B i)] [∀ i, BoundedSMul 𝕜 (B i)]
826826
[∀ i, SMulCommClass 𝕜 (B i) (B i)] : SMulCommClass 𝕜 (lp B ∞) (lp B ∞) :=
827827
fun r f g => lp.ext <| smul_comm (N := ∀ i, B i) (α := ∀ i, B i) r (⇑f) (⇑g)⟩
828-
#align lp.infty_smul_comm_class lp.infty_sMulCommClass
828+
#align lp.infty_smul_comm_class lp.infty_smulCommClass
829829

830830
section StarRing
831831

Mathlib/Data/Set/Intervals/ProjIcc.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -211,9 +211,9 @@ theorem IicExtend_apply (f : Iic b → β) (x : α) : IicExtend f x = f ⟨min b
211211
rfl
212212
#align set.Iic_extend_apply Set.IicExtend_apply
213213

214-
theorem iccExtend_apply (h : a ≤ b) (f : Icc a b → β) (x : α) :
214+
theorem IccExtend_apply (h : a ≤ b) (f : Icc a b → β) (x : α) :
215215
IccExtend h f x = f ⟨max a (min b x), le_max_left _ _, max_le h (min_le_left _ _)⟩ := rfl
216-
#align set.Icc_extend_apply Set.iccExtend_apply
216+
#align set.Icc_extend_apply Set.IccExtend_apply
217217

218218
@[simp]
219219
theorem range_IciExtend (f : Ici a → β) : range (IciExtend f) = range f := by

Mathlib/Geometry/Manifold/MFDeriv.lean

Lines changed: 15 additions & 13 deletions
Original file line numberDiff line numberDiff line change
@@ -316,15 +316,17 @@ section DerivativesProperties
316316

317317
/-! ### Unique differentiability sets in manifolds -/
318318

319-
variable {𝕜 : Type*} [NontriviallyNormedField 𝕜] {E : Type*} [NormedAddCommGroup E]
320-
[NormedSpace 𝕜 E] {H : Type*} [TopologicalSpace H] (I : ModelWithCorners 𝕜 E H) {M : Type*}
321-
[TopologicalSpace M] [ChartedSpace H M]
322-
--
323-
{E' : Type*}
324-
[NormedAddCommGroup E'] [NormedSpace 𝕜 E'] {H' : Type*} [TopologicalSpace H']
325-
{I' : ModelWithCorners 𝕜 E' H'} {M' : Type*} [TopologicalSpace M'] [ChartedSpace H' M']
326-
{E'' : Type*} [NormedAddCommGroup E''] [NormedSpace 𝕜 E''] {H'' : Type*} [TopologicalSpace H'']
327-
{I'' : ModelWithCorners 𝕜 E'' H''} {M'' : Type*} [TopologicalSpace M''] [ChartedSpace H'' M'']
319+
variable
320+
{𝕜 : Type*} [NontriviallyNormedField 𝕜]
321+
{E : Type*} [NormedAddCommGroup E] [NormedSpace 𝕜 E]
322+
{H : Type*} [TopologicalSpace H] (I : ModelWithCorners 𝕜 E H)
323+
{M : Type*} [TopologicalSpace M] [ChartedSpace H M]
324+
{E' : Type*} [NormedAddCommGroup E'] [NormedSpace 𝕜 E']
325+
{H' : Type*} [TopologicalSpace H'] {I' : ModelWithCorners 𝕜 E' H'}
326+
{M' : Type*} [TopologicalSpace M'] [ChartedSpace H' M']
327+
{E'' : Type*} [NormedAddCommGroup E''] [NormedSpace 𝕜 E'']
328+
{H'' : Type*} [TopologicalSpace H''] {I'' : ModelWithCorners 𝕜 E'' H''}
329+
{M'' : Type*} [TopologicalSpace M''] [ChartedSpace H'' M'']
328330
{f f₀ f₁ : M → M'} {x : M} {s t : Set M} {g : M' → M''} {u : Set M'}
329331

330332
theorem uniqueMDiffWithinAt_univ : UniqueMDiffWithinAt I univ x := by
@@ -1105,7 +1107,7 @@ alias ⟨HasMFDerivAt.hasFDerivAt, HasFDerivAt.hasMFDerivAt⟩ := hasMFDerivAt_i
11051107
#align has_mfderiv_at.has_fderiv_at HasMFDerivAt.hasFDerivAt
11061108
#align has_fderiv_at.has_mfderiv_at HasFDerivAt.hasMFDerivAt
11071109

1108-
/-- For maps between vector spaces, `MDifferentiableWithinAt` and `fdifferentiable_within_at`
1110+
/-- For maps between vector spaces, `MDifferentiableWithinAt` and `DifferentiableWithinAt`
11091111
coincide -/
11101112
theorem mdifferentiableWithinAt_iff_differentiableWithinAt :
11111113
MDifferentiableWithinAt 𝓘(𝕜, E) 𝓘(𝕜, E') f s x ↔ DifferentiableWithinAt 𝕜 f s x := by
@@ -2021,7 +2023,7 @@ variable {𝕜 : Type*} [NontriviallyNormedField 𝕜] {E : Type*} [NormedAddCom
20212023
{I' : ModelWithCorners 𝕜 E' H'} {M' : Type*} [TopologicalSpace M'] [ChartedSpace H' M']
20222024
[SmoothManifoldWithCorners I' M'] {s : Set M}
20232025

2024-
/-- If `s` has the unique differential property at `x`, `f` is differetiable within `s` at x` and
2026+
/-- If `s` has the unique differential property at `x`, `f` is differentiable within `s` at x` and
20252027
its derivative has Dense range, then `f '' s` has the Unique differential property at `f x`. -/
20262028
theorem UniqueMDiffWithinAt.image_denseRange (hs : UniqueMDiffWithinAt I s x)
20272029
{f : M → M'} {f' : E →L[𝕜] E'} (hf : HasMFDerivWithinAt I I' f s x f')
@@ -2035,7 +2037,7 @@ theorem UniqueMDiffWithinAt.image_denseRange (hs : UniqueMDiffWithinAt I s x)
20352037
rintro _ ⟨y, ⟨⟨hys, hfy⟩, -⟩, rfl⟩
20362038
exact ⟨⟨_, hys, ((extChartAt I' (f x)).left_inv hfy).symm⟩, mem_range_self _⟩
20372039

2038-
/-- If `s` has the unique differential, `f` is differetiable on `s` and its derivative at every
2040+
/-- If `s` has the unique differential, `f` is differentiable on `s` and its derivative at every
20392041
point of `s` has dense range, then `f '' s` has the unique differential property. This version
20402042
uses `HaMFDerivWithinAt` predicate. -/
20412043
theorem UniqueMDiffOn.image_denseRange' (hs : UniqueMDiffOn I s) {f : M → M'}
@@ -2044,7 +2046,7 @@ theorem UniqueMDiffOn.image_denseRange' (hs : UniqueMDiffOn I s) {f : M → M'}
20442046
UniqueMDiffOn I' (f '' s) :=
20452047
ball_image_iff.2 fun x hx ↦ (hs x hx).image_denseRange (hf x hx) (hd x hx)
20462048

2047-
/-- If `s` has the unique differential, `f` is differetiable on `s` and its derivative at every
2049+
/-- If `s` has the unique differential, `f` is differentiable on `s` and its derivative at every
20482050
point of `s` has dense range, then `f '' s` has the unique differential property. -/
20492051
theorem UniqueMDiffOn.image_denseRange (hs : UniqueMDiffOn I s) {f : M → M'}
20502052
(hf : MDifferentiableOn I I' f s) (hd : ∀ x ∈ s, DenseRange (mfderivWithin I I' f s x)) :

Mathlib/Logic/Equiv/Array.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -78,9 +78,9 @@ instance for `array` was)
7878
/-- If `α` is encodable, then so is `Array α`. -/
7979
instance Array.encodable {α} [Encodable α] : Encodable (Array α) :=
8080
Encodable.ofEquiv _ (Equiv.arrayEquivList _)
81-
#align array.encodable Array.encodable
81+
#noalign array.encodable
8282

8383
/-- If `α` is countable, then so is `Array α`. -/
8484
instance Array.countable {α} [Countable α] : Countable (Array α) :=
8585
Countable.of_equiv _ (Equiv.arrayEquivList α).symm
86-
#align array.countable Array.countable
86+
#noalign array.countable

Mathlib/MeasureTheory/Function/LocallyIntegrable.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -526,7 +526,7 @@ theorem IntegrableOn.continuousOn_mul [T2Space X] (hg : ContinuousOn g K)
526526

527527
end Mul
528528

529-
section Smul
529+
section SMul
530530

531531
variable {𝕜 : Type*} [NormedField 𝕜] [NormedSpace 𝕜 E]
532532

@@ -550,7 +550,7 @@ theorem IntegrableOn.smul_continuousOn [T2Space X] [SecondCountableTopologyEithe
550550
· exact hf.1.smul (hg.aestronglyMeasurable hK.measurableSet)
551551
#align measure_theory.integrable_on.smul_continuous_on MeasureTheory.IntegrableOn.smul_continuousOn
552552

553-
end Smul
553+
end SMul
554554

555555
namespace LocallyIntegrableOn
556556

0 commit comments

Comments
 (0)