Skip to content

Commit 603d009

Browse files
committed
fixed subobject/basic.lean
1 parent 16b5d12 commit 603d009

File tree

3 files changed

+791
-81
lines changed

3 files changed

+791
-81
lines changed

Mathlib/CategoryTheory/Subobject/Basic.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -191,8 +191,7 @@ def isoFromEq {A : C} {X Y : Subobject A} (h : X = Y) :=
191191

192192
@[simp]
193193
theorem arrow_congr {A : C} (X Y : Subobject A) (h : X = Y) :
194-
(isoFromEq h).hom ≫ Y.arrow = X.arrow := by
195-
unfold isoFromEq
194+
eqToHom (congr_arg (fun X : Subobject A => (X : C)) h) ≫ Y.arrow = X.arrow := by
196195
induction h
197196
simp
198197

Mathlib/CategoryTheory/Topos/Basic.lean

Lines changed: 0 additions & 79 deletions
This file was deleted.

0 commit comments

Comments
 (0)