Skip to content

Commit

Permalink
feat(differential_object/iso_app): extract the isomorphism of underly…
Browse files Browse the repository at this point in the history
…ing objects (#6083)

From `lean-liquid`.

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Feb 8, 2021
1 parent 0c6fa28 commit d62d793
Showing 1 changed file with 13 additions and 0 deletions.
13 changes: 13 additions & 0 deletions src/category_theory/differential_object.lean
Expand Up @@ -102,6 +102,19 @@ variables {C}
@[simp]
lemma zero_f (P Q : differential_object C) : (0 : P ⟶ Q).f = 0 := rfl

/--
An isomorphism of differential objects gives an isomorphism of the underlying objects.
-/
@[simps] def iso_app {X Y : differential_object C} (f : X ≅ Y) : X.X ≅ Y.X :=
⟨f.hom.f, f.inv.f, by { dsimp, rw [← comp_f, iso.hom_inv_id, id_f] },
by { dsimp, rw [← comp_f, iso.inv_hom_id, id_f] }⟩

@[simp] lemma iso_app_refl (X : differential_object C) : iso_app (iso.refl X) = iso.refl X.X := rfl
@[simp] lemma iso_app_symm {X Y : differential_object C} (f : X ≅ Y) :
iso_app f.symm = (iso_app f).symm := rfl
@[simp] lemma iso_app_trans {X Y Z : differential_object C} (f : X ≅ Y) (g : Y ≅ Z) :
iso_app (f ≪≫ g) = iso_app f ≪≫ iso_app g := rfl

end differential_object

namespace functor
Expand Down

0 comments on commit d62d793

Please sign in to comment.