blog/src/pmltt-lang.agda
Michael Zhang 0e0249d113
Some checks failed
ci/woodpecker/push/woodpecker Pipeline failed
sad
2023-10-12 17:22:58 -05:00

16 lines
348 B
Agda

open import Data.String
-- Chapter 3.6
data Arity : Set where
zero : Arity
_⊗_ : Arity Arity Arity
_-→_ : Arity Arity Arity
data Expr : Set where
Var : String Arity Expr
PrimConst : Arity Expr
App : Expr Expr Expr
Abs : String Expr Expr
arity-of : (e : Expr) Arity