aboutsummaryrefslogtreecommitdiff
path: root/Data/Setoid/Unit.agda
blob: 8b8eddef914de59ef2f2990dd7d5db2c8075c0ca (plain)
1
2
3
4
5
6
7
8
9
10
11
{-# OPTIONS --without-K --safe #-}

open import Level using (Level)

module Data.Setoid.Unit {c  : Level} where

open import Categories.Category.Instance.SingletonSet using (SingletonSetoid)
open import Relation.Binary using (Setoid)

⊤ₛ : Setoid c ℓ
⊤ₛ = SingletonSetoid {c} {}