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

open import Relation.Binary using (Setoid)

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