summaryrefslogtreecommitdiff
path: root/src/Cfe/Context/Properties.agda
blob: 2acaf729d74914b59e8fe05141847d3bfbe4687b (plain)
1
2
3
4
5
6
7
{-# OPTIONS --without-K --safe #-}

open import Relation.Binary using (Setoid)

module Cfe.Context.Properties
  {c ℓ} (over : Setoid c ℓ)
  where