Skip to content

Commit

Permalink
feat(category_theory/natural_isomorphism): a simp lemma cancelling in…
Browse files Browse the repository at this point in the history
…verses (#14299)

I am not super happy to be adding lemmas like this, because it feels like better designed simp normal forms (or something else) could just avoid the need.

However my efforts to think about this keep getting stuck on the shift functor hole we're in, and this lemma is useful in the meantime to dig my way out of it. :-)




Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed May 22, 2022
1 parent e4a8db1 commit eae0510
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/category_theory/natural_isomorphism.lean
Expand Up @@ -155,6 +155,10 @@ instance is_iso_app_of_is_iso (α : F ⟶ G) [is_iso α] (X) : is_iso (α.app X)
@[simp] lemma is_iso_inv_app (α : F ⟶ G) [is_iso α] (X) : (inv α).app X = inv (α.app X) :=
by { ext, rw ←nat_trans.comp_app, simp, }

@[simp] lemma inv_map_inv_app (F : C ⥤ D ⥤ E) {X Y : C} (e : X ≅ Y) (Z : D) :
inv ((F.map e.inv).app Z) = (F.map e.hom).app Z :=
by { ext, simp, }

/--
Construct a natural isomorphism between functors by giving object level isomorphisms,
and checking naturality only in the forward direction.
Expand Down

0 comments on commit eae0510

Please sign in to comment.