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

open import Relation.Binary using (Setoid)

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

open import Cfe.Expression.Base setoid public