summaryrefslogtreecommitdiff
path: root/src/Cfe/Language.agda
blob: 7469ef5fd3e9bfb820ce88a99e688cf787295074 (plain)
1
2
3
4
5
6
7
8
9
10
{-# 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
open import Cfe.Language.Properties setoid public