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

open import Relation.Binary using (Setoid)

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