Skip to content

Commit 73f6a3a

Browse files
committed
chore: remove use of erw in Algebra.Homology.HomotopyCofiber (#31855)
1 parent 2100ab2 commit 73f6a3a

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

Mathlib/Algebra/Homology/HomotopyCofiber.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -432,8 +432,7 @@ noncomputable abbrev inrX (i : ι) : (K ⊞ K).X i ⟶ K.cylinder.X i :=
432432
@[reassoc (attr := simp)]
433433
lemma inlX_π (i j : ι) (hij : c.Rel j i) :
434434
inlX K i j hij ≫ (π K).f j = 0 := by
435-
erw [homotopyCofiber.inlX_desc_f]
436-
simp [Homotopy.equivSubZero]
435+
simp [HomologicalComplex.cylinder.π, HomologicalComplex.cylinder.desc, Homotopy.equivSubZero]
437436

438437
@[reassoc (attr := simp)]
439438
lemma inrX_π (i : ι) :

0 commit comments

Comments
 (0)