Skip to content

Commit

Permalink
feat(category_theory/isomorphism): is_iso versions (#5355)
Browse files Browse the repository at this point in the history
add `is_iso` versions of some existing `iso` lemmas
  • Loading branch information
b-mehta committed Dec 15, 2020
1 parent dbb6b04 commit 2ee0f1e
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/category_theory/isomorphism.lean
Expand Up @@ -254,6 +254,12 @@ instance (f : X ⟶ Y) : subsingleton (is_iso f) :=
lemma is_iso.inv_eq_inv {f g : X ⟶ Y} [is_iso f] [is_iso g] : inv f = inv g ↔ f = g :=
iso.inv_eq_inv (as_iso f) (as_iso g)

lemma hom_comp_eq_id (g : X ⟶ Y) [is_iso g] {f : Y ⟶ X} : g ≫ f = 𝟙 X ↔ f = inv g :=
(as_iso g).hom_comp_eq_id

lemma comp_hom_eq_id (g : X ⟶ Y) [is_iso g] {f : Y ⟶ X} : f ≫ g = 𝟙 Y ↔ f = inv g :=
(as_iso g).comp_hom_eq_id

namespace iso

/-!
Expand Down

0 comments on commit 2ee0f1e

Please sign in to comment.