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

module Cfe.Expression
  {ℓ} (A : Set ℓ)
  where

open import Cfe.Expression.Base A public