File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed
Mathlib/CategoryTheory/Closed Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -157,12 +157,12 @@ noncomputable instance singleton_is_mono : Mono (singleton hPB) :=
157157 let PeqP' : P = P' := by
158158 unfold P P'
159159 rw[pullback_diag_eq_singleton hPB b, eq, ← pullback_diag_eq_singleton hPB b']
160- let ι : X ≅ Subobject.underlying.obj P :=
160+ let iso : X ≅ Subobject.underlying.obj P :=
161161 IsPullback.isoIsPullback_congr
162162 (Subobject.underlyingIso (cmdiag B)).symm (Iso.refl _) (Iso.refl _)
163163 (by simpa using Subobject.underlyingIso_hom_comp_eq_mk (cmdiag B)) (by simp)
164164 (pullback_of_diag b) (Subobject.isPullback (B ◁ b) B_sub)
165- let eq₁ : (lift b (𝟙 X)) = ι .hom ≫ P.arrow := by unfold P ι ; simp
165+ let eq₁ : (lift b (𝟙 X)) = iso .hom ≫ P.arrow := by unfold P iso ; simp
166166 let eq₂ := Eq.symm (Subobject.arrow_congr P P' PeqP')
167167 let eq₃ := Eq.symm (Subobject.isPullback (B ◁ b') B_sub).w
168168 let eq₄ := Eq.symm (Subobject.underlyingIso_hom_comp_eq_mk (cmdiag B))
You can’t perform that action at this time.
0 commit comments