aboutsummaryrefslogtreecommitdiff
path: root/Data/System/Values.agda
blob: bf8fa38df7ef03d73ba5a2dd3f6a8d61aa77531a (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
{-# OPTIONS --without-K --safe #-}

module Data.System.Values (A : Set) where

open import Data.Nat.Base using ()
open import Data.Vec.Functional using (Vector)
open import Level using (0)
open import Relation.Binary using (Rel; Setoid)
open import Data.Vec.Functional.Relation.Binary.Equality.Setoid using (≋-setoid)

import Relation.Binary.PropositionalEquality as Values :   Setoid 0 0ℓ
Values = ≋-setoid (≡.setoid A)

_≋_ : {n : }  Rel (Vector A n) 0ℓ
_≋_ {n} = Setoid._≈_ (Values n)

infix 4 _≋_

module ≋ {n : } = Setoid (Values n)