Skip to content

Commit

Permalink
tweaking modules parameters to debug issue of CI running out of memor…
Browse files Browse the repository at this point in the history
…y...
  • Loading branch information
marcinjangrzybowski committed Oct 26, 2023
1 parent 1786fcd commit 5c34283
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Cubical/Categories/NaturalTransformation/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -111,6 +111,8 @@ module _ {C : Category ℓC ℓC'} {D : Category ℓD ℓD'} where
-- Natural isomorphism is path when the target category is univalent.

module _
{C : Category ℓC ℓC'}
{D : Category ℓD ℓD'}
(isUnivD : isUnivalent D)
{F G : Functor C D} where

Expand Down

0 comments on commit 5c34283

Please sign in to comment.