File tree Expand file tree Collapse file tree 1 file changed +18
-0
lines changed
src/Categories/NaturalTransformation Expand file tree Collapse file tree 1 file changed +18
-0
lines changed Original file line number Diff line number Diff line change @@ -71,6 +71,24 @@ record NaturalIsomorphism {C : Category o ℓ e}
71
71
}
72
72
}
73
73
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
+
74
92
-- This helper definition lets us specify only one of the commuting
75
93
-- squares and have the other one derived.
76
94
You can’t perform that action at this time.
0 commit comments