We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
1 parent 16b5d12 commit 603d009Copy full SHA for 603d009
Mathlib/CategoryTheory/Subobject/Basic.lean
@@ -191,8 +191,7 @@ def isoFromEq {A : C} {X Y : Subobject A} (h : X = Y) :=
191
192
@[simp]
193
theorem arrow_congr {A : C} (X Y : Subobject A) (h : X = Y) :
194
- (isoFromEq h).hom ≫ Y.arrow = X.arrow := by
195
- unfold isoFromEq
+ eqToHom (congr_arg (fun X : Subobject A => (X : C)) h) ≫ Y.arrow = X.arrow := by
196
induction h
197
simp
198
Mathlib/CategoryTheory/Topos/Basic.lean
0 commit comments