File tree Expand file tree Collapse file tree 1 file changed +4
-4
lines changed
src/Categories/Category/Instance Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change 3
3
open import Level
4
4
5
5
-- 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 ⊤
7
7
module Categories.Category.Instance.SingletonSet where
8
8
9
- open import Data.Unit using (⊤; tt)
9
+ open import Data.Unit.Polymorphic using (⊤; tt)
10
10
open import Relation.Binary using (Setoid)
11
11
open import Relation.Binary.PropositionalEquality using (refl)
12
12
@@ -18,13 +18,13 @@ module _ {o : Level} where
18
18
open Term (Sets o)
19
19
20
20
SingletonSet-⊤ : Terminal
21
- SingletonSet-⊤ = record { ⊤ = Lift o ⊤ ; ⊤-is-terminal = record { !-unique = λ _ → refl } }
21
+ SingletonSet-⊤ = record { ⊤ = ⊤ ; ⊤-is-terminal = record { !-unique = λ _ → refl } }
22
22
23
23
module _ {c ℓ : Level} where
24
24
open Term (Setoids c ℓ)
25
25
26
26
SingletonSetoid : Setoid c ℓ
27
- SingletonSetoid = record { Carrier = Lift c ⊤ ; _≈_ = λ _ _ → Lift ℓ ⊤ }
27
+ SingletonSetoid = record { Carrier = ⊤ ; _≈_ = λ _ _ → ⊤ }
28
28
29
29
SingletonSetoid-⊤ : Terminal
30
30
SingletonSetoid-⊤ = record { ⊤ = SingletonSetoid }
You can’t perform that action at this time.
0 commit comments