Skip to content

Commit a109603

Browse files
Merge pull request #359 from 91khr/master
Add `IsNI` to be consistent with `IsIso` in for morphisms
2 parents 42d2d68 + 7b8c211 commit a109603

File tree

1 file changed

+18
-0
lines changed

1 file changed

+18
-0
lines changed

src/Categories/NaturalTransformation/NaturalIsomorphism.agda

Lines changed: 18 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -71,6 +71,24 @@ record NaturalIsomorphism {C : Category o ℓ e}
7171
}
7272
}
7373

74+
-- Like IsIso for morphisms, a natural transformation may be an isomorphism
75+
-- if there exists some inverse to it.
76+
-- To be consistent, there's also an IsNI for natural isomorphisms
77+
record IsNI {C : Category o ℓ e}
78+
{D : Category o′ ℓ′ e′}
79+
{F G : Functor C D}
80+
(F⇒G : NaturalTransformation F G) : Set (o ⊔ ℓ ⊔ ℓ′ ⊔ e′) where
81+
field
82+
F⇐G : NaturalTransformation G F
83+
iso : X Morphism.Iso D (NaturalTransformation.η F⇒G X) (NaturalTransformation.η F⇐G X)
84+
85+
natiso : NaturalIsomorphism F G
86+
natiso = record
87+
{ F⇒G = F⇒G
88+
; F⇐G = F⇐G
89+
; iso = iso
90+
}
91+
7492
-- This helper definition lets us specify only one of the commuting
7593
-- squares and have the other one derived.
7694

0 commit comments

Comments
 (0)