Skip to content

Commit a0765bc

Browse files
committed
chore: rename a bunch of stuff (#18886)
These are (in my opinion) improperly named things that I encountered over time. Happy to remove any of them if there are disagreements. * Remove manual instance names `IccManifold` and `Icc_smooth_manifold`. They're improper because the former is a `ChartedSpace` instance, while the latter is a `SmoothManifoldWithCorners` instance. As instances, they also probably shouldn't come up so high when searching for "Manifold" in the docs. Their names are now automatically generated, just like the two instances below them. * Rename `ManifoldWithCorners.metrizableSpace` to `Manifold.metrizableSpace`. * Rename `apply_(h)fdifferential` to `(h)fdifferential_apply`. This is to match the semantics of e.g. `ite_apply` and `apply_ite`.
1 parent 3d1502c commit a0765bc

File tree

5 files changed

+18
-14
lines changed

5 files changed

+18
-14
lines changed

Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -47,7 +47,7 @@ theorem ae_eq_zero_of_integral_smooth_smul_eq_zero [SigmaCompactSpace M]
4747
have := ChartedSpace.locallyCompactSpace H M
4848
have := I.secondCountableTopology
4949
have := ChartedSpace.secondCountable_of_sigma_compact H M
50-
have := ManifoldWithCorners.metrizableSpace I M
50+
have := Manifold.metrizableSpace I M
5151
let _ : MetricSpace M := TopologicalSpace.metrizableSpaceMetric M
5252
-- it suffices to show that the integral of the function vanishes on any compact set `s`
5353
apply ae_eq_zero_of_forall_setIntegral_isCompact_eq_zero' hf (fun s hs ↦ Eq.symm ?_)

Mathlib/Geometry/Manifold/Algebra/LeftInvariantDerivation.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -204,25 +204,25 @@ theorem left_invariant : 𝒅ₕ (smoothLeftMul_one I g) (evalAt (1 : G) X) = ev
204204

205205
theorem evalAt_mul : evalAt (g * h) X = 𝒅ₕ (L_apply I g h) (evalAt h X) := by
206206
ext f
207-
rw [← left_invariant, apply_hfdifferential, apply_hfdifferential, L_mul, fdifferential_comp,
208-
apply_fdifferential]
207+
rw [← left_invariant, hfdifferential_apply, hfdifferential_apply, L_mul, fdifferential_comp,
208+
fdifferential_apply]
209209
-- Porting note: more aggressive here
210210
erw [LinearMap.comp_apply]
211211
-- This used to be `rw`, but we need `erw` after leanprover/lean4#2644
212-
erw [apply_fdifferential, ← apply_hfdifferential, left_invariant]
212+
erw [fdifferential_apply, ← hfdifferential_apply, left_invariant]
213213

214214
theorem comp_L : (X f).comp (𝑳 I g) = X (f.comp (𝑳 I g)) := by
215215
ext h
216-
rw [ContMDiffMap.comp_apply, L_apply, ← evalAt_apply, evalAt_mul, apply_hfdifferential,
217-
apply_fdifferential, evalAt_apply]
216+
rw [ContMDiffMap.comp_apply, L_apply, ← evalAt_apply, evalAt_mul, hfdifferential_apply,
217+
fdifferential_apply, evalAt_apply]
218218

219219
instance : Bracket (LeftInvariantDerivation I G) (LeftInvariantDerivation I G) where
220220
bracket X Y :=
221221
⟨⁅(X : Derivation 𝕜 C^∞⟮I, G; 𝕜⟯ C^∞⟮I, G; 𝕜⟯), Y⁆, fun g => by
222222
ext f
223223
have hX := Derivation.congr_fun (left_invariant' g X) (Y f)
224224
have hY := Derivation.congr_fun (left_invariant' g Y) (X f)
225-
rw [apply_hfdifferential, apply_fdifferential, Derivation.evalAt_apply] at hX hY ⊢
225+
rw [hfdifferential_apply, fdifferential_apply, Derivation.evalAt_apply] at hX hY ⊢
226226
rw [comp_L] at hX hY
227227
rw [Derivation.commutator_apply, SmoothMap.coe_sub, Pi.sub_apply, coe_derivation]
228228
rw [coe_derivation] at hX hY ⊢

Mathlib/Geometry/Manifold/DerivationBundle.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -150,14 +150,16 @@ scoped[Manifold] notation "𝒅" => fdifferential
150150
scoped[Manifold] notation "𝒅ₕ" => hfdifferential
151151

152152
@[simp]
153-
theorem apply_fdifferential (f : C^∞⟮I, M; I', M'⟯) {x : M} (v : PointDerivation I x)
153+
theorem fdifferential_apply (f : C^∞⟮I, M; I', M'⟯) {x : M} (v : PointDerivation I x)
154154
(g : C^∞⟮I', M'; 𝕜⟯) : 𝒅 f x v g = v (g.comp f) :=
155155
rfl
156+
@[deprecated (since := "2024-11-11")] alias apply_fdifferential := fdifferential_apply
156157

157158
@[simp]
158-
theorem apply_hfdifferential {f : C^∞⟮I, M; I', M'⟯} {x : M} {y : M'} (h : f x = y)
159+
theorem hfdifferential_apply {f : C^∞⟮I, M; I', M'⟯} {x : M} {y : M'} (h : f x = y)
159160
(v : PointDerivation I x) (g : C^∞⟮I', M'; 𝕜⟯) : 𝒅ₕ h v g = 𝒅 f x v g :=
160161
rfl
162+
@[deprecated (since := "2024-11-11")] alias apply_hfdifferential := hfdifferential_apply
161163

162164
variable {E'' : Type*} [NormedAddCommGroup E''] [NormedSpace 𝕜 E''] {H'' : Type*}
163165
[TopologicalSpace H''] {I'' : ModelWithCorners 𝕜 E'' H''} {M'' : Type*} [TopologicalSpace M'']

Mathlib/Geometry/Manifold/Instances/Real.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -320,7 +320,7 @@ def IccRightChart (x y : ℝ) [h : Fact (x < y)] :
320320
/-- Charted space structure on `[x, y]`, using only two charts taking values in
321321
`EuclideanHalfSpace 1`.
322322
-/
323-
instance IccManifold (x y : ℝ) [h : Fact (x < y)] :
323+
instance IccChartedSpace (x y : ℝ) [h : Fact (x < y)] :
324324
ChartedSpace (EuclideanHalfSpace 1) (Icc x y) where
325325
atlas := {IccLeftChart x y, IccRightChart x y}
326326
chartAt z := if z.val < y then IccLeftChart x y else IccRightChart x y
@@ -335,7 +335,7 @@ instance IccManifold (x y : ℝ) [h : Fact (x < y)] :
335335

336336
/-- The manifold structure on `[x, y]` is smooth.
337337
-/
338-
instance Icc_smooth_manifold (x y : ℝ) [Fact (x < y)] :
338+
instance Icc_smoothManifoldWithCorners (x y : ℝ) [Fact (x < y)] :
339339
SmoothManifoldWithCorners (𝓡∂ 1) (Icc x y) := by
340340
have M : ContDiff ℝ ∞ (show EuclideanSpace ℝ (Fin 1) → EuclideanSpace ℝ (Fin 1)
341341
from fun z i => -z i + (y - x)) :=
@@ -373,8 +373,8 @@ instance Icc_smooth_manifold (x y : ℝ) [Fact (x < y)] :
373373
·-- `e = right chart`, `e' = right chart`
374374
exact (mem_groupoid_of_pregroupoid.mpr (symm_trans_mem_contDiffGroupoid _)).1
375375

376-
/-! Register the manifold structure on `Icc 0 1`, and also its zero and one. -/
377-
376+
/-! Register the manifold structure on `Icc 0 1`. These are merely special cases of
377+
`IccChartedSpace` and `Icc_smoothManifoldWithCorners`. -/
378378

379379
section
380380

Mathlib/Geometry/Manifold/Metrizable.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -19,11 +19,13 @@ open TopologicalSpace
1919

2020
/-- A σ-compact Hausdorff topological manifold over a finite dimensional real vector space is
2121
metrizable. -/
22-
theorem ManifoldWithCorners.metrizableSpace {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]
22+
theorem Manifold.metrizableSpace {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]
2323
[FiniteDimensional ℝ E] {H : Type*} [TopologicalSpace H] (I : ModelWithCorners ℝ E H)
2424
(M : Type*) [TopologicalSpace M] [ChartedSpace H M] [SigmaCompactSpace M] [T2Space M] :
2525
MetrizableSpace M := by
2626
haveI := I.locallyCompactSpace; haveI := ChartedSpace.locallyCompactSpace H M
2727
haveI := I.secondCountableTopology
2828
haveI := ChartedSpace.secondCountable_of_sigma_compact H M
2929
exact metrizableSpace_of_t3_second_countable M
30+
@[deprecated (since := "2024-11-11")] alias ManifoldWithCorners.metrizableSpace :=
31+
Manifold.metrizableSpace

0 commit comments

Comments
 (0)