{-# OPTIONS --postfix-projections #-}
module V2.TypeChecker where
open import Library
import V2.AST as A
open import V2.WellTypedSyntax
Name = String
idToName : A.Id → Name
idToName (A.mkId x) = String.fromList x
TCCxt : (Γ : Cxt) → Set
TCCxt Γ = AssocList Name Γ
data TypeError : Set where
unboundVariable : Name → TypeError
typeMismatch : (tinf texp : Type) → tinf ≢ texp → TypeError
instance
PrintError : Print TypeError
print {{PrintError}} = λ where
(unboundVariable x) → "unbound variable " String.++ x
(typeMismatch tinf texp _) → String.concat $
"type mismatch: expected " ∷ print texp ∷
", but inferred " ∷ print tinf ∷ []
open ErrorMonad {E = TypeError}
lookupVar : {Γ : Cxt} (γ : TCCxt Γ) (x : Name)
→ Error (Σ Type (λ t → Var Γ t))
lookupVar {[]} [] x = throwError $ unboundVariable x
lookupVar {t ∷ Γ} (x' ∷ γ) x = case x ≟ x' of λ where
(yes refl) → ok (t , here)
(no _) → case lookupVar γ x of λ where
(ok (t , i)) → ok (t , there i)
(fail err) → fail err
module CheckExpressions {Γ : Cxt} (γ : TCCxt Γ) where
mutual
inferExp : (e : A.Exp) → Error (Σ Type (λ t → Exp Γ t))
inferExp (A.eInt i) = return (int , eInt i)
inferExp (A.eBool b) = return (bool , eBool b)
inferExp (A.eId x) = do
(t , x') ← lookupVar γ (idToName x)
return (t , eVar x')
inferExp (A.ePlus e₁ e₂) = inferOp plus e₁ e₂
inferExp (A.eGt e₁ e₂) = inferOp gt e₁ e₂
inferExp (A.eAnd e₁ e₂) = inferOp and e₁ e₂
inferExp (A.eCond e₁ e₂ e₃) = do
e₁' ← checkExp e₁ bool
(t , e₂') ← inferExp e₂
e₃' ← checkExp e₃ t
return (t , eCond e₁' e₂' e₃')
checkExp : (e : A.Exp) (t : Type) → Error (Exp Γ t)
checkExp e t = do
(t' , e') ← inferExp e
case t' ≟ t of λ where
(yes refl) → return e'
(no t'≢t) → throwError (typeMismatch t' t t'≢t)
inferOp : ∀{t t'} (op : Op t t') (e₁ e₂ : A.Exp) → Error (Σ Type (λ t → Exp Γ t))
inferOp {t} {t'} op e₁ e₂ = do
e₁' ← checkExp e₁ t
e₂' ← checkExp e₂ t
return (t' , eOp op e₁' e₂')
record TCExp Γ (A : Set) : Set where
field
runTCExp : TCCxt Γ → Error A
open TCExp
checkExp : ∀{Γ} (e : A.Exp) (t : Type) → TCExp Γ (Exp Γ t)
checkExp e t .runTCExp γ = CheckExpressions.checkExp γ e t
record TCDecl Γ Γ' (A : Set) : Set where
field
runTCDecl : TCCxt Γ → Error (A × TCCxt Γ')
open TCDecl
module CheckDeclarations where
private
returnTCDecl : ∀ {Γ A} (a : A) → TCDecl Γ Γ A
returnTCDecl a .runTCDecl γ = ok (a , γ)
bindTCDecl : ∀{Γ Γ′ Γ″ A B}
(m : TCDecl Γ Γ′ A)
(k : A → TCDecl Γ′ Γ″ B)
→ TCDecl Γ Γ″ B
bindTCDecl m k .runTCDecl γ =
case m .runTCDecl γ of λ where
(fail err) → fail err
(ok (a , γ')) → k a .runTCDecl γ'
instance
functorTCDecl : ∀ {Γ Γ′} → Functor (TCDecl Γ Γ′)
fmap {{functorTCDecl}} f m = bindTCDecl m (returnTCDecl ∘′ f)
iApplicativeTCDecl : IApplicative TCDecl
pure {{iApplicativeTCDecl}} = returnTCDecl
_<*>_ {{iApplicativeTCDecl}} mf mx = bindTCDecl mf (_<$> mx)
iMonadTCDecl : IMonad TCDecl
_>>=_ {{iMonadTCDecl}} = bindTCDecl
lift : ∀{Γ A} (m : TCExp Γ A) → TCDecl Γ Γ A
lift m .runTCDecl γ =
case m .runTCExp γ of λ where
(fail err) → fail err
(ok a) → ok (a , γ)
addVar : ∀{Γ} (x : Name) t → TCDecl Γ (t ∷ Γ) ⊤
addVar {Γ = Γ} x t .runTCDecl γ = ok (_ , (t ↦ x ∷ γ))
Next : (Γ : Cxt) (s : A.Decl) → Cxt
Next Γ s = A.declType s ∷ Γ
Nexts : (Γ : Cxt) (ss : List A.Decl) → Cxt
Nexts = foldl Next
mutual
checkDecl : ∀ {Γ} (d : A.Decl) (let t = A.declType d)
→ TCDecl Γ (t ∷ Γ) (Decl Γ t)
checkDecl (A.dInit t x e) = do
e' ← lift $ checkExp e t
addVar (idToName x) t
return (dInit e')
checkDecls : ∀ {Γ} (ds : List A.Decl) (let Γ' = Nexts Γ ds)
→ TCDecl Γ Γ' (Decls Γ Γ')
checkDecls [] = return []
checkDecls (d ∷ ds) = do
d' ← checkDecl d
(d' ∷_) <$> checkDecls ds
checkProgram : (prg : A.Program) (let Γ = Nexts [] (A.theDecls prg))
→ TCDecl [] Γ Program
checkProgram (A.program ds e) = do
ds' ← checkDecls ds
e' ← lift $ checkExp e int
return (program ds' e')
checkProgram : (prg : A.Program) → Error Program
checkProgram prg = proj₁ <$> CheckDeclarations.checkProgram prg .runTCDecl []