Skip to content

Commit

Permalink
Update Prelude.agda
Browse files Browse the repository at this point in the history
make refl and lift instances
  • Loading branch information
anshwad10 authored Jan 12, 2025
1 parent 2f085f5 commit 8daae10
Showing 1 changed file with 8 additions and 3 deletions.
11 changes: 8 additions & 3 deletions Cubical/Foundations/Prelude.agda
Original file line number Diff line number Diff line change
Expand Up @@ -43,9 +43,10 @@ private
B : A Type ℓ
x y z w : A

refl : x ≡ x
refl {x = x} _ = x
{-# INLINE refl #-}
instance
refl : x ≡ x
refl {x = x} _ = x
{-# INLINE refl #-}

sym : x ≡ y y ≡ x
sym p i = p (~ i)
Expand Down Expand Up @@ -638,3 +639,7 @@ liftExt x i = lift (x i)
liftFun : {ℓ ℓ' ℓ'' ℓ'''} {A : Type ℓ} {B : Type ℓ'}
(f : A B) Lift {j = ℓ''} A Lift {j = ℓ'''} B
liftFun f (lift a) = lift (f a)

instance
liftInstance : ⦃ A ⦄ Lift A
liftInstance ⦃ a ⦄ = lift a

0 comments on commit 8daae10

Please sign in to comment.