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

open import Relation.Binary using (Setoid)

module Cfe.Language
  {a ℓ} (setoid : Setoid a ℓ)
  where

open import Cfe.Language.Base setoid public