File tree Expand file tree Collapse file tree 2 files changed +3
-8
lines changed Expand file tree Collapse file tree 2 files changed +3
-8
lines changed Original file line number Diff line number Diff line change @@ -518,11 +518,7 @@ def kernelIsoKer {G H : AddCommGrp.{u}} (f : G ⟶ H) :
518
518
change _ = _ + _
519
519
dsimp
520
520
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
526
522
hom_inv_id := by
527
523
-- Porting note (#11041): it would be nice to do the next two steps by a single `ext`,
528
524
-- but this will require thinking carefully about the relative priorities of `@[ext]` lemmas.
Original file line number Diff line number Diff line change @@ -94,7 +94,6 @@ instance (i : I) : Functor.Full (incl i : C i ⥤ Σi, C i) where
94
94
map_surjective := fun ⟨f⟩ => ⟨f, rfl⟩
95
95
96
96
instance (i : I) : Functor.Faithful (incl i : C i ⥤ Σi, C i) where
97
- -- Porting note (#10936): was `tidy`
98
97
map_injective {_ _ _ _} h := by injection h
99
98
100
99
section
@@ -236,11 +235,11 @@ def mapId : map C (id : I → I) ≅ 𝟭 (Σi, C i) :=
236
235
237
236
variable {I} {K : Type w₃}
238
237
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
240
239
-- so that the suitable category instances could be found
241
240
/-- The functor `Sigma.map` applied to a composition is a composition of functors. -/
242
241
@[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) :=
244
243
(descUniq _ _) fun k =>
245
244
(isoWhiskerRight (inclCompMap (fun i => C (g i)) f k) (map C g : _) : _) ≪≫ inclCompMap _ _ _
246
245
#align category_theory.sigma.map_comp CategoryTheory.Sigma.mapComp
You can’t perform that action at this time.
0 commit comments