Skip to content

Commit

Permalink
liftC C is equivalent to C
Browse files Browse the repository at this point in the history
  • Loading branch information
Taneb committed Feb 26, 2025
1 parent 98c8a1b commit ed32ce5
Showing 1 changed file with 39 additions and 0 deletions.
39 changes: 39 additions & 0 deletions src/Categories/Category/Lift/Properties.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,39 @@
{-# OPTIONS --without-K --safe #-}

module Categories.Category.Lift.Properties where

open import Level

open import Categories.Category.Core
open import Categories.Category.Equivalence
open import Categories.Category.Lift
open import Categories.NaturalTransformation.NaturalIsomorphism
import Categories.Morphism.Reasoning.Core as MR

unliftF-liftF-weakInverse : {o ℓ e} o′ ℓ′ e′ (C : Category o ℓ e) WeakInverse (unliftF o′ ℓ′ e′ C) (liftF o′ ℓ′ e′ C)
unliftF-liftF-weakInverse o′ ℓ′ e′ C = record
{ F∘G≈id = niHelper record
{ η = λ X id
; η⁻¹ = λ X id
; commute = λ f id-comm-sym
; iso = λ X record
{ isoˡ = identity²
; isoʳ = identity²
}
}
; G∘F≈id = niHelper record
{ η = λ X lift id
; η⁻¹ = λ X lift id
; commute = λ f lift id-comm-sym
; iso = λ X record
{ isoˡ = lift identity²
; isoʳ = lift identity²
}
}
}
where
open Category C
open MR C

liftC-strongEquivalence : {o ℓ e} o′ ℓ′ e′ (C : Category o ℓ e) StrongEquivalence (liftC o′ ℓ′ e′ C) C
liftC-strongEquivalence o′ ℓ′ e′ C = record { weak-inverse = unliftF-liftF-weakInverse o′ ℓ′ e′ C }

0 comments on commit ed32ce5

Please sign in to comment.