Skip to content

Commit d421f15

Browse files
committed
chore: more indentation fixes (#27502)
Found by the linter in #27473.
1 parent ce6e378 commit d421f15

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

68 files changed

+180
-193
lines changed

Mathlib/Algebra/Algebra/NonUnitalHom.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -86,7 +86,7 @@ namespace NonUnitalAlgHomClass
8686

8787
-- See note [lower instance priority]
8888
instance (priority := 100) toNonUnitalRingHomClass
89-
{F R S A B : Type*} {_ : Monoid R} {_ : Monoid S} {φ : outParam (R →* S)}
89+
{F R S A B : Type*} {_ : Monoid R} {_ : Monoid S} {φ : outParam (R →* S)}
9090
{_ : NonUnitalNonAssocSemiring A} [DistribMulAction R A]
9191
{_ : NonUnitalNonAssocSemiring B} [DistribMulAction S B] [FunLike F A B]
9292
[NonUnitalAlgSemiHomClass F φ A B] : NonUnitalRingHomClass F A B :=

Mathlib/Algebra/Azumaya/Defs.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -32,8 +32,7 @@ variable (R A : Type*) [CommSemiring R] [Semiring A] [Algebra R A]
3232
open TensorProduct MulOpposite
3333

3434
/-- `A` as a `A ⊗[R] Aᵐᵒᵖ`-module (or equivalently, an `A`-`A` bimodule). -/
35-
abbrev instModuleTensorProductMop :
36-
Module (A ⊗[R] Aᵐᵒᵖ) A := TensorProduct.Algebra.module
35+
abbrev instModuleTensorProductMop : Module (A ⊗[R] Aᵐᵒᵖ) A := TensorProduct.Algebra.module
3736

3837
/-- The canonical map from `A ⊗[R] Aᵐᵒᵖ` to `Module.End R A` where
3938
`a ⊗ b` maps to `f : x ↦ a * x * b`. -/

Mathlib/Algebra/Category/FGModuleCat/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -87,7 +87,7 @@ section Ring
8787
variable (R : Type u) [Ring R]
8888

8989
@[simp] lemma hom_comp (A B C : FGModuleCat.{v} R) (f : A ⟶ B) (g : B ⟶ C) :
90-
(f ≫ g).hom = g.hom.comp f.hom := rfl
90+
(f ≫ g).hom = g.hom.comp f.hom := rfl
9191

9292
@[simp] lemma hom_id (A : FGModuleCat.{v} R) : (𝟙 A : A ⟶ A).hom = LinearMap.id := rfl
9393

@@ -100,7 +100,7 @@ abbrev of (V : Type v) [AddCommGroup V] [Module R V] [Module.Finite R V] : FGMod
100100

101101
@[simp]
102102
lemma of_carrier (V : Type v) [AddCommGroup V] [Module R V] [Module.Finite R V] :
103-
of R V = V := rfl
103+
of R V = V := rfl
104104

105105
variable {R} in
106106
/-- Lift a linear map between finitely generated modules to `FGModuleCat R`. -/

Mathlib/Algebra/Category/Grp/Basic.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -378,8 +378,7 @@ lemma hom_ext {X Y : CommGrp} {f g : X ⟶ Y} (hf : f.hom = g.hom) : f = g :=
378378
Hom.ext hf
379379

380380
@[to_additive (attr := simp)]
381-
lemma hom_ofHom {X Y : Type u} [CommGroup X] [CommGroup Y] (f : X →* Y) :
382-
(ofHom f).hom = f := rfl
381+
lemma hom_ofHom {X Y : Type u} [CommGroup X] [CommGroup Y] (f : X →* Y) : (ofHom f).hom = f := rfl
383382

384383
@[to_additive (attr := simp)]
385384
lemma ofHom_hom {X Y : CommGrp} (f : X ⟶ Y) :

Mathlib/Algebra/Category/Grp/Limits.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -170,8 +170,7 @@ instance forget₂Mon_preservesLimitsOfSize [UnivLE.{v, u}] :
170170
preservesLimitsOfShape {J _} := { }
171171

172172
@[to_additive]
173-
instance forget₂Mon_preservesLimits :
174-
PreservesLimits (forget₂ Grp.{u} MonCat.{u}) :=
173+
instance forget₂Mon_preservesLimits : PreservesLimits (forget₂ Grp.{u} MonCat.{u}) :=
175174
Grp.forget₂Mon_preservesLimitsOfSize.{u, u}
176175

177176
/-- If `J` is `u`-small, the forgetful functor from `Grp.{u}` preserves limits of shape `J`. -/

Mathlib/Algebra/Category/GrpWithZero.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -64,8 +64,7 @@ lemma coe_id {X : GrpWithZero} : (𝟙 X : X → X) = id := rfl
6464

6565
lemma coe_comp {X Y Z : GrpWithZero} {f : X ⟶ Y} {g : Y ⟶ Z} : (f ≫ g : X → Z) = g ∘ f := rfl
6666

67-
@[simp] lemma forget_map {X Y : GrpWithZero} (f : X ⟶ Y) :
68-
(forget GrpWithZero).map f = f := rfl
67+
@[simp] lemma forget_map {X Y : GrpWithZero} (f : X ⟶ Y) : (forget GrpWithZero).map f = f := rfl
6968

7069
instance hasForgetToBipointed : HasForget₂ GrpWithZero Bipointed where
7170
forget₂ :=

Mathlib/Algebra/Category/ModuleCat/Colimits.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -147,6 +147,6 @@ example (R : Type u) [Ring R] : HasCoequalizers (ModuleCat.{u} R) := by
147147
instance : HasCoequalizers (ModuleCat.{v} R) where
148148

149149
noncomputable example (R : Type u) [Ring R] :
150-
PreservesColimits (forget₂ (ModuleCat.{u} R) AddCommGrp) := inferInstance
150+
PreservesColimits (forget₂ (ModuleCat.{u} R) AddCommGrp) := inferInstance
151151

152152
end ModuleCat

Mathlib/Algebra/Category/ModuleCat/Presheaf.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -375,7 +375,7 @@ noncomputable def forgetToPresheafModuleCatObjMap {Y Z : Cᵒᵖ} (f : Y ⟶ Z)
375375

376376
@[simp]
377377
lemma forgetToPresheafModuleCatObjMap_apply {Y Z : Cᵒᵖ} (f : Y ⟶ Z) (m : M.obj Y) :
378-
(forgetToPresheafModuleCatObjMap X hX M f).hom m = M.map f m := rfl
378+
(forgetToPresheafModuleCatObjMap X hX M f).hom m = M.map f m := rfl
379379

380380
/--
381381
Implementation of the functor `PresheafOfModules R ⥤ Cᵒᵖ ⥤ ModuleCat (R.obj X)`

Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean

Lines changed: 6 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -89,16 +89,14 @@ abbrev ofHom {X Y : Type v}
8989
[AddCommGroup X] [Module R X] [TopologicalSpace X] [ContinuousAdd X] [ContinuousSMul R X]
9090
[AddCommGroup Y] [Module R Y] [TopologicalSpace Y] [ContinuousAdd Y] [ContinuousSMul R Y]
9191
(f : X →L[R] Y) :
92-
(ofHom f).hom = f := rfl
92+
(ofHom f).hom = f := rfl
9393

94-
@[simp] lemma ofHom_hom {X Y : TopModuleCat R} (f : X.Hom Y) :
95-
ofHom f.hom = f := rfl
94+
@[simp] lemma ofHom_hom {X Y : TopModuleCat R} (f : X.Hom Y) : ofHom f.hom = f := rfl
9695

9796
@[simp] lemma hom_comp {X Y Z : TopModuleCat R} (f : X ⟶ Y) (g : Y ⟶ Z) :
98-
(f ≫ g).hom = g.hom.comp f.hom := rfl
97+
(f ≫ g).hom = g.hom.comp f.hom := rfl
9998

100-
@[simp] lemma hom_id (X : TopModuleCat R) :
101-
hom (𝟙 X) = .id _ _ := rfl
99+
@[simp] lemma hom_id (X : TopModuleCat R) : hom (𝟙 X) = .id _ _ := rfl
102100

103101
/-- Use the `ConcreteCategory.hom` projection for `@[simps]` lemmas. -/
104102
def Hom.Simps.hom (A B : TopModuleCat.{v} R) (f : A.Hom B) :=
@@ -157,8 +155,7 @@ instance [CommRing S] : Linear S (TopModuleCat S) where
157155
comp_smul _ _ _ _ _ _ := ConcreteCategory.ext (ContinuousLinearMap.smul_comp _ _ _)
158156

159157
@[simp]
160-
lemma hom_smul {M₁ M₂ : TopModuleCat S} (s : S) (φ : M₁ ⟶ M₂) :
161-
(s • φ).hom = s • φ.hom := rfl
158+
lemma hom_smul {M₁ M₂ : TopModuleCat S} (s : S) (φ : M₁ ⟶ M₂) : (s • φ).hom = s • φ.hom := rfl
162159

163160
end CommRing
164161

@@ -184,7 +181,7 @@ instance : (forget₂ (TopModuleCat R) TopCat).ReflectsIsomorphisms where
184181

185182
@[simp]
186183
lemma hom_forget₂_TopCat_map {X Y : TopModuleCat R} (f : X ⟶ Y) :
187-
((forget₂ _ TopCat).map f).hom = f.hom := rfl
184+
((forget₂ _ TopCat).map f).hom = f.hom := rfl
188185

189186
@[simp]
190187
lemma forget₂_TopCat_obj {X : TopModuleCat R} : ((forget₂ _ TopCat).obj X : Type _) = X := rfl

Mathlib/Algebra/Category/MonCat/FilteredColimits.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -75,8 +75,8 @@ variable [IsFiltered J]
7575
@[to_additive
7676
"As `J` is nonempty, we can pick an arbitrary object `j₀ : J`. We use this object to
7777
define the \"zero\" in the colimit as the equivalence class of `⟨j₀, 0 : F.obj j₀⟩`."]
78-
noncomputable instance colimitOne :
79-
One (M.{v, u} F) where one := M.mk F ⟨IsFiltered.nonempty.some,1
78+
noncomputable instance colimitOne : One (M.{v, u} F) where
79+
one := M.mk F ⟨IsFiltered.nonempty.some,1
8080

8181
/-- The definition of the "one" in the colimit is independent of the chosen object of `J`.
8282
In particular, this lemma allows us to "unfold" the definition of `colimit_one` at a custom chosen

0 commit comments

Comments
 (0)