Skip to content

Commit 7672b7a

Browse files
authored
Merge pull request #214 from conal/SingletonSet-LevelPolymorphic
Use Data.Unit.Polymorphic instead, and drop explicit liftings
2 parents d82a741 + e471c41 commit 7672b7a

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

src/Categories/Category/Instance/SingletonSet.agda

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -3,10 +3,10 @@
33
open import Level
44

55
-- This is really a degenerate version of Categories.Category.Instance.One
6-
-- Here SingletonSet is not given an explicit name, it is an alias for Lift o
6+
-- Here SingletonSet is not given an explicit name, it is an alias for ⊤
77
module Categories.Category.Instance.SingletonSet where
88

9-
open import Data.Unit using (⊤; tt)
9+
open import Data.Unit.Polymorphic using (⊤; tt)
1010
open import Relation.Binary using (Setoid)
1111
open import Relation.Binary.PropositionalEquality using (refl)
1212

@@ -18,13 +18,13 @@ module _ {o : Level} where
1818
open Term (Sets o)
1919

2020
SingletonSet-⊤ : Terminal
21-
SingletonSet-⊤ = record { ⊤ = Lift o ⊤ ; ⊤-is-terminal = record { !-unique = λ _ refl } }
21+
SingletonSet-⊤ = record { ⊤ = ⊤ ; ⊤-is-terminal = record { !-unique = λ _ refl } }
2222

2323
module _ {c ℓ : Level} where
2424
open Term (Setoids c ℓ)
2525

2626
SingletonSetoid : Setoid c ℓ
27-
SingletonSetoid = record { Carrier = Lift c ⊤ ; _≈_ = λ _ _ Lift ℓ ⊤ }
27+
SingletonSetoid = record { Carrier = ⊤ ; _≈_ = λ _ _ ⊤ }
2828

2929
SingletonSetoid-⊤ : Terminal
3030
SingletonSetoid-⊤ = record { ⊤ = SingletonSetoid }

0 commit comments

Comments
 (0)