Skip to content

Commit 60b7d34

Browse files
committed
chore: tidy three miscellaneous porting notes (#14511)
One porting note seems clearly superfluous now. In another, make the note match the statement below it (some variable renaming had made them go out of sync). Fix a third porting note; to me, the new proof feels good enough.
1 parent 411ac5c commit 60b7d34

File tree

2 files changed

+3
-8
lines changed

2 files changed

+3
-8
lines changed

Mathlib/Algebra/Category/Grp/Limits.lean

Lines changed: 1 addition & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -518,11 +518,7 @@ def kernelIsoKer {G H : AddCommGrp.{u}} (f : G ⟶ H) :
518518
change _ = _ + _
519519
dsimp
520520
simp }
521-
inv := kernel.lift f (AddSubgroup.subtype f.ker) <| by
522-
-- Porting note (#10936): used to be `tidy`, but `aesop` can't do it
523-
refine DFunLike.ext _ _ ?_
524-
rintro ⟨x, (hx : f _ = 0)⟩
525-
exact hx
521+
inv := kernel.lift f (AddSubgroup.subtype f.ker) <| by ext x; exact x.2
526522
hom_inv_id := by
527523
-- Porting note (#11041): it would be nice to do the next two steps by a single `ext`,
528524
-- but this will require thinking carefully about the relative priorities of `@[ext]` lemmas.

Mathlib/CategoryTheory/Sigma/Basic.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -94,7 +94,6 @@ instance (i : I) : Functor.Full (incl i : C i ⥤ Σi, C i) where
9494
map_surjective := fun ⟨f⟩ => ⟨f, rfl⟩
9595

9696
instance (i : I) : Functor.Faithful (incl i : C i ⥤ Σi, C i) where
97-
-- Porting note (#10936): was `tidy`
9897
map_injective {_ _ _ _} h := by injection h
9998

10099
section
@@ -236,11 +235,11 @@ def mapId : map C (id : I → I) ≅ 𝟭 (Σi, C i) :=
236235

237236
variable {I} {K : Type w₃}
238237

239-
-- Porting note: Had to expand (G ∘ g) to (fun i => C (g i)) in lemma statement
238+
-- Porting note: Had to expand (C ∘ g) to (fun x => C (g x)) in lemma statement
240239
-- so that the suitable category instances could be found
241240
/-- The functor `Sigma.map` applied to a composition is a composition of functors. -/
242241
@[simps!]
243-
def mapComp (f : K → J) (g : J → I) : map (fun x => C (g x)) f ⋙ (map C g : _) ≅ map C (g ∘ f) :=
242+
def mapComp (f : K → J) (g : J → I) : map (fun x C (g x)) f ⋙ (map C g : _) ≅ map C (g ∘ f) :=
244243
(descUniq _ _) fun k =>
245244
(isoWhiskerRight (inclCompMap (fun i => C (g i)) f k) (map C g : _) : _) ≪≫ inclCompMap _ _ _
246245
#align category_theory.sigma.map_comp CategoryTheory.Sigma.mapComp

0 commit comments

Comments
 (0)