quox/lib/Quox/Typechecker.idr

499 lines
18 KiB
Idris
Raw Normal View History

2022-04-23 18:21:30 -04:00
module Quox.Typechecker
import public Quox.Typing
import public Quox.Equal
2022-04-23 18:21:30 -04:00
import Data.List
2023-03-26 10:09:47 -04:00
import Data.SnocVect
import Data.List1
2023-03-31 13:23:30 -04:00
import Quox.EffExtra
2022-04-23 18:21:30 -04:00
%default total
2023-01-20 20:34:28 -05:00
public export
2023-04-01 13:16:43 -04:00
0 TCEff : List (Type -> Type)
2023-05-01 21:06:25 -04:00
TCEff = [ErrorEff, DefsReader, NameGen]
2023-01-20 20:34:28 -05:00
public export
2023-04-01 13:16:43 -04:00
0 TC : Type -> Type
TC = Eff TCEff
2023-03-31 13:23:30 -04:00
2023-05-01 21:06:25 -04:00
export
runTCWith : NameSuf -> Definitions -> TC a -> (Either Error a, NameSuf)
runTCWith = runEqualWith
2023-03-31 13:23:30 -04:00
export
runTC : Definitions -> TC a -> Either Error a
2023-05-01 21:06:25 -04:00
runTC = runEqual
2023-01-20 20:34:28 -05:00
2023-05-01 21:06:25 -04:00
parameters (loc : Loc)
export
popQs : Has ErrorEff fs => QContext s -> QOutput (s + n) -> Eff fs (QOutput n)
popQs [<] qout = pure qout
popQs (pis :< pi) (qout :< rh) = do expectCompatQ loc rh pi; popQs pis qout
2022-04-23 18:21:30 -04:00
2023-05-01 21:06:25 -04:00
export %inline
popQ : Has ErrorEff fs => Qty -> QOutput (S n) -> Eff fs (QOutput n)
popQ pi = popQs [< pi]
2023-01-26 13:54:46 -05:00
export
2023-05-12 11:28:29 -04:00
lubs1 : List1 (QOutput n) -> QOutput n
lubs1 ([<] ::: _) = [<]
lubs1 ((qs :< p) ::: pqs) =
let (qss, ps) = unzip $ map unsnoc pqs in
2023-05-12 11:28:29 -04:00
lubs1 (qs ::: qss) :< foldl lub p ps
export
2023-05-12 11:28:29 -04:00
lubs : TyContext d n -> List (QOutput n) -> QOutput n
lubs ctx [] = zeroFor ctx
lubs ctx (x :: xs) = lubs1 $ x ::: xs
2022-04-23 18:21:30 -04:00
2023-04-15 09:13:01 -04:00
export
2023-05-01 21:06:25 -04:00
typecaseTel : (k : TyConKind) -> BContext (arity k) -> Universe ->
CtxExtension d n (arity k + n)
typecaseTel k xs u = case k of
2023-04-15 09:13:01 -04:00
KTYPE => [<]
-- A : ★ᵤ, B : 0.A → ★ᵤ
2023-05-01 21:06:25 -04:00
KPi =>
let [< a, b] = xs in
[< (Zero, a, TYPE u a.loc),
(Zero, b, Arr Zero (BVT 0 b.loc) (TYPE u b.loc) b.loc)]
KSig =>
let [< a, b] = xs in
[< (Zero, a, TYPE u a.loc),
(Zero, b, Arr Zero (BVT 0 b.loc) (TYPE u b.loc) b.loc)]
2023-04-15 09:13:01 -04:00
KEnum => [<]
-- A₀ : ★ᵤ, A₁ : ★ᵤ, A : (A₀ ≡ A₁ : ★ᵤ), L : A₀, R : A₀
2023-05-01 21:06:25 -04:00
KEq =>
let [< a0, a1, a, l, r] = xs in
[< (Zero, a0, TYPE u a0.loc),
(Zero, a1, TYPE u a1.loc),
(Zero, a, Eq0 (TYPE u a.loc) (BVT 1 a.loc) (BVT 0 a.loc) a.loc),
(Zero, l, BVT 2 l.loc),
(Zero, r, BVT 2 r.loc)]
2023-04-15 09:13:01 -04:00
KNat => [<]
-- A : ★ᵤ
2023-05-01 21:06:25 -04:00
KBOX => let [< a] = xs in [< (Zero, a, TYPE u a.loc)]
2023-04-15 09:13:01 -04:00
2023-04-03 11:46:23 -04:00
2023-04-01 13:16:43 -04:00
mutual
2023-02-19 11:04:57 -05:00
||| "Ψ | Γ ⊢ σ · s ⇐ A ⊳ Σ"
|||
2023-01-20 20:34:28 -05:00
||| `check ctx sg subj ty` checks that in the context `ctx`, the term
||| `subj` has the type `ty`, with quantity `sg`. if so, returns the
||| quantities of all bound variables that it used.
2023-02-19 11:51:44 -05:00
|||
||| if the dimension context is inconsistent, then return `Nothing`, without
||| doing any further work.
2022-04-23 18:21:30 -04:00
export covering %inline
2023-04-01 13:16:43 -04:00
check : (ctx : TyContext d n) -> SQty -> Term d n -> Term d n ->
TC (CheckResult ctx.dctx n)
2023-02-20 15:38:47 -05:00
check ctx sg subj ty = ifConsistent ctx.dctx $ checkC ctx sg subj ty
2022-04-23 18:21:30 -04:00
2023-02-19 11:04:57 -05:00
||| "Ψ | Γ ⊢₀ s ⇐ A"
|||
||| `check0 ctx subj ty` checks a term (as `check`) in a zero context.
2023-01-26 13:54:46 -05:00
export covering %inline
2023-04-01 13:16:43 -04:00
check0 : TyContext d n -> Term d n -> Term d n -> TC ()
2023-02-14 15:14:47 -05:00
check0 ctx tm ty = ignore $ check ctx szero tm ty
-- the output will always be 𝟎 because the subject quantity is 0
2023-01-26 13:54:46 -05:00
2023-02-19 11:51:44 -05:00
||| `check`, assuming the dimension context is consistent
export covering %inline
2023-04-01 13:16:43 -04:00
checkC : (ctx : TyContext d n) -> SQty -> Term d n -> Term d n ->
TC (CheckResult' n)
2023-02-19 11:51:44 -05:00
checkC ctx sg subj ty =
2023-02-19 11:54:39 -05:00
wrapErr (WhileChecking ctx sg.fst subj ty) $
let Element subj nc = pushSubsts subj in
2023-02-20 15:42:21 -05:00
check' ctx sg subj ty
2023-02-19 11:51:44 -05:00
||| "Ψ | Γ ⊢₀ s ⇐ ★ᵢ"
|||
||| `checkType ctx subj ty` checks a type (in a zero context). sometimes the
||| universe doesn't matter, only that a term is _a_ type, so it is optional.
export covering %inline
2023-04-01 13:16:43 -04:00
checkType : TyContext d n -> Term d n -> Maybe Universe -> TC ()
checkType ctx subj l = ignore $ ifConsistent ctx.dctx $ checkTypeC ctx subj l
export covering %inline
2023-04-01 13:16:43 -04:00
checkTypeC : TyContext d n -> Term d n -> Maybe Universe -> TC ()
checkTypeC ctx subj l =
wrapErr (WhileCheckingTy ctx subj l) $ checkTypeNoWrap ctx subj l
export covering %inline
2023-04-01 13:16:43 -04:00
checkTypeNoWrap : TyContext d n -> Term d n -> Maybe Universe -> TC ()
checkTypeNoWrap ctx subj l =
let Element subj nc = pushSubsts subj in
checkType' ctx subj l
2023-02-19 11:51:44 -05:00
2023-02-19 11:04:57 -05:00
||| "Ψ | Γ ⊢ σ · e ⇒ A ⊳ Σ"
|||
2023-01-20 20:34:28 -05:00
||| `infer ctx sg subj` infers the type of `subj` in the context `ctx`,
||| and returns its type and the bound variables it used.
2023-02-19 11:51:44 -05:00
|||
||| if the dimension context is inconsistent, then return `Nothing`, without
||| doing any further work.
export covering %inline
2023-04-01 13:16:43 -04:00
infer : (ctx : TyContext d n) -> SQty -> Elim d n ->
TC (InferResult ctx.dctx d n)
2023-02-20 15:38:47 -05:00
infer ctx sg subj = ifConsistent ctx.dctx $ inferC ctx sg subj
2023-02-19 11:51:44 -05:00
||| `infer`, assuming the dimension context is consistent
2022-04-23 18:21:30 -04:00
export covering %inline
2023-04-01 13:16:43 -04:00
inferC : (ctx : TyContext d n) -> SQty -> Elim d n ->
TC (InferResult' d n)
2023-02-19 11:51:44 -05:00
inferC ctx sg subj =
2023-02-19 11:54:39 -05:00
wrapErr (WhileInferring ctx sg.fst subj) $
let Element subj nc = pushSubsts subj in
2023-02-20 15:42:21 -05:00
infer' ctx sg subj
2022-04-23 18:21:30 -04:00
private covering
2023-04-01 13:16:43 -04:00
toCheckType : TyContext d n -> SQty ->
(subj : Term d n) -> (0 nc : NotClo subj) => Term d n ->
TC (CheckResult' n)
toCheckType ctx sg t ty = do
2023-05-01 21:06:25 -04:00
u <- expectTYPE !defs ctx ty.loc ty
expectEqualQ t.loc Zero sg.fst
checkTypeNoWrap ctx t (Just u)
pure $ zeroFor ctx
2023-02-19 11:51:44 -05:00
private covering
2023-04-01 13:16:43 -04:00
check' : TyContext d n -> SQty ->
(subj : Term d n) -> (0 nc : NotClo subj) => Term d n ->
TC (CheckResult' n)
2022-04-23 18:21:30 -04:00
2023-05-01 21:06:25 -04:00
check' ctx sg t@(TYPE {}) ty = toCheckType ctx sg t ty
2022-04-23 18:21:30 -04:00
check' ctx sg t@(Pi {}) ty = toCheckType ctx sg t ty
2022-04-27 15:58:09 -04:00
2023-05-01 21:06:25 -04:00
check' ctx sg (Lam body loc) ty = do
(qty, arg, res) <- expectPi !defs ctx ty.loc ty
2023-02-14 15:14:47 -05:00
-- if Ψ | Γ, x : A ⊢ σ · t ⇐ B ⊳ Σ, ρ·x
-- with ρ ≤ σπ
let qty' = sg.fst * qty
2023-03-15 10:54:51 -04:00
qout <- checkC (extendTy qty' body.name arg ctx) sg body.term res.term
-- then Ψ | Γ ⊢ σ · (λx ⇒ t) ⇐ (π·x : A) → B ⊳ Σ
2023-05-01 21:06:25 -04:00
popQ loc qty' qout
2023-01-26 13:54:46 -05:00
check' ctx sg t@(Sig {}) ty = toCheckType ctx sg t ty
2023-01-26 13:54:46 -05:00
2023-05-01 21:06:25 -04:00
check' ctx sg (Pair fst snd loc) ty = do
(tfst, tsnd) <- expectSig !defs ctx ty.loc ty
-- if Ψ | Γ ⊢ σ · s ⇐ A ⊳ Σ₁
2023-02-19 11:51:44 -05:00
qfst <- checkC ctx sg fst tfst
2023-05-01 21:06:25 -04:00
let tsnd = sub1 tsnd (Ann fst tfst fst.loc)
-- if Ψ | Γ ⊢ σ · t ⇐ B[s] ⊳ Σ₂
2023-02-19 11:51:44 -05:00
qsnd <- checkC ctx sg snd tsnd
-- then Ψ | Γ ⊢ σ · (s, t) ⇐ (x : A) × B ⊳ Σ₁ + Σ₂
2023-01-26 13:54:46 -05:00
pure $ qfst + qsnd
2022-04-27 15:58:09 -04:00
2023-05-01 21:06:25 -04:00
check' ctx sg t@(Enum {}) ty = toCheckType ctx sg t ty
2023-05-01 21:06:25 -04:00
check' ctx sg (Tag t loc) ty = do
tags <- expectEnum !defs ctx ty.loc ty
-- if t ∈ ts
2023-05-01 21:06:25 -04:00
unless (t `elem` tags) $ throw $ TagNotIn loc t tags
-- then Ψ | Γ ⊢ σ · t ⇐ {ts} ⊳ 𝟎
pure $ zeroFor ctx
check' ctx sg t@(Eq {}) ty = toCheckType ctx sg t ty
2023-01-20 20:34:28 -05:00
2023-05-01 21:06:25 -04:00
check' ctx sg (DLam body loc) ty = do
(ty, l, r) <- expectEq !defs ctx ty.loc ty
let ctx' = extendDim body.name ctx
ty = ty.term
body = body.term
-- if Ψ, i | Γ ⊢ σ · t ⇐ A ⊳ Σ
qout <- checkC ctx' sg body ty
-- if Ψ, i, i = 0 | Γ ⊢ t = l : A
2023-05-01 21:06:25 -04:00
lift $ equal loc (eqDim (B VZ loc) (K Zero loc) ctx') ty body (dweakT 1 l)
-- if Ψ, i, i = 1 | Γ ⊢ t = r : A
2023-05-01 21:06:25 -04:00
lift $ equal loc (eqDim (B VZ loc) (K One loc) ctx') ty body (dweakT 1 r)
2023-02-25 13:14:11 -05:00
-- then Ψ | Γ ⊢ σ · (δ i ⇒ t) ⇐ Eq [i ⇒ A] l r ⊳ Σ
2023-01-20 20:34:28 -05:00
pure qout
2023-05-01 21:06:25 -04:00
check' ctx sg t@(Nat {}) ty = toCheckType ctx sg t ty
2023-03-26 08:40:54 -04:00
2023-05-01 21:06:25 -04:00
check' ctx sg (Zero {}) ty = do
expectNat !defs ctx ty.loc ty
2023-03-26 08:40:54 -04:00
pure $ zeroFor ctx
2023-05-01 21:06:25 -04:00
check' ctx sg (Succ n {}) ty = do
expectNat !defs ctx ty.loc ty
checkC ctx sg n ty
2023-03-26 08:40:54 -04:00
2023-03-31 13:11:35 -04:00
check' ctx sg t@(BOX {}) ty = toCheckType ctx sg t ty
2023-05-01 21:06:25 -04:00
check' ctx sg (Box val loc) ty = do
(q, ty) <- expectBOX !defs ctx ty.loc ty
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ ⊢ σ · s ⇐ A ⊳ Σ
valout <- checkC ctx sg val ty
-- then Ψ | Γ ⊢ σ · [s] ⇐ [π.A] ⊳ πΣ
pure $ q * valout
2023-02-20 15:42:21 -05:00
check' ctx sg (E e) ty = do
-- if Ψ | Γ ⊢ σ · e ⇒ A' ⊳ Σ
2023-02-19 11:51:44 -05:00
infres <- inferC ctx sg e
-- if Ψ | Γ ⊢ A' <: A
2023-05-01 21:06:25 -04:00
lift $ subtype e.loc ctx infres.type ty
-- then Ψ | Γ ⊢ σ · e ⇐ A ⊳ Σ
2022-04-27 15:58:09 -04:00
pure infres.qout
2022-04-23 18:21:30 -04:00
private covering
2023-04-01 13:16:43 -04:00
checkType' : TyContext d n ->
(subj : Term d n) -> (0 nc : NotClo subj) =>
Maybe Universe -> TC ()
2023-05-01 21:06:25 -04:00
checkType' ctx (TYPE k loc) u = do
-- if 𝓀 < then Ψ | Γ ⊢₀ Type 𝓀 ⇐ Type
case u of
2023-05-01 21:06:25 -04:00
Just l => unless (k < l) $ throw $ BadUniverse loc k l
Nothing => pure ()
2023-05-01 21:06:25 -04:00
checkType' ctx (Pi qty arg res _) u = do
-- if Ψ | Γ ⊢₀ A ⇐ Type
checkTypeC ctx arg u
-- if Ψ | Γ, x : A ⊢₀ B ⇐ Type
2023-04-03 11:46:23 -04:00
checkTypeScope ctx arg res u
-- then Ψ | Γ ⊢₀ (π·x : A) → B ⇐ Type
checkType' ctx t@(Lam {}) u =
2023-05-01 21:06:25 -04:00
throw $ NotType t.loc ctx t
2023-05-01 21:06:25 -04:00
checkType' ctx (Sig fst snd _) u = do
-- if Ψ | Γ ⊢₀ A ⇐ Type
checkTypeC ctx fst u
-- if Ψ | Γ, x : A ⊢₀ B ⇐ Type
2023-04-03 11:46:23 -04:00
checkTypeScope ctx fst snd u
-- then Ψ | Γ ⊢₀ (x : A) × B ⇐ Type
checkType' ctx t@(Pair {}) u =
2023-05-01 21:06:25 -04:00
throw $ NotType t.loc ctx t
2023-05-01 21:06:25 -04:00
checkType' ctx (Enum {}) u = pure ()
-- Ψ | Γ ⊢₀ {ts} ⇐ Type
checkType' ctx t@(Tag {}) u =
2023-05-01 21:06:25 -04:00
throw $ NotType t.loc ctx t
2023-05-01 21:06:25 -04:00
checkType' ctx (Eq t l r _) u = do
-- if Ψ, i | Γ ⊢₀ A ⇐ Type
case t.body of
Y t' => checkTypeC (extendDim t.name ctx) t' u
N t' => checkTypeC ctx t' u
-- if Ψ | Γ ⊢₀ l ⇐ A0
2023-04-01 10:02:02 -04:00
check0 ctx l t.zero
-- if Ψ | Γ ⊢₀ r ⇐ A1
2023-04-01 10:02:02 -04:00
check0 ctx r t.one
-- then Ψ | Γ ⊢₀ Eq [i ⇒ A] l r ⇐ Type
checkType' ctx t@(DLam {}) u =
2023-05-01 21:06:25 -04:00
throw $ NotType t.loc ctx t
2023-05-01 21:06:25 -04:00
checkType' ctx (Nat {}) u = pure ()
checkType' ctx t@(Zero {}) u = throw $ NotType t.loc ctx t
checkType' ctx t@(Succ {}) u = throw $ NotType t.loc ctx t
2023-03-26 08:40:54 -04:00
2023-05-01 21:06:25 -04:00
checkType' ctx (BOX q ty _) u = checkType ctx ty u
checkType' ctx t@(Box {}) u = throw $ NotType t.loc ctx t
2023-03-31 13:11:35 -04:00
checkType' ctx (E e) u = do
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ ⊢₀ E ⇒ Type
infres <- inferC ctx szero e
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ ⊢ Type <: Type 𝓀
case u of
2023-05-01 21:06:25 -04:00
Just u => lift $ subtype e.loc ctx infres.type (TYPE u noLoc)
Nothing => ignore $ expectTYPE !defs ctx e.loc infres.type
2023-03-31 13:11:35 -04:00
-- then Ψ | Γ ⊢₀ E ⇐ Type 𝓀
2023-04-03 11:46:23 -04:00
private covering
checkTypeScope : TyContext d n -> Term d n ->
ScopeTerm d n -> Maybe Universe -> TC ()
2023-05-01 21:06:25 -04:00
checkTypeScope ctx s (S _ (N body)) u = checkType ctx body u
checkTypeScope ctx s (S [< x] (Y body)) u =
checkType (extendTy Zero x s ctx) body u
2023-04-03 11:46:23 -04:00
2023-02-19 11:51:44 -05:00
private covering
2023-04-01 13:16:43 -04:00
infer' : TyContext d n -> SQty ->
(subj : Elim d n) -> (0 nc : NotClo subj) =>
TC (InferResult' d n)
2022-04-23 18:21:30 -04:00
2023-05-01 21:06:25 -04:00
infer' ctx sg (F x loc) = do
2023-02-14 15:14:47 -05:00
-- if π·x : A {≔ s} in global context
2023-05-01 21:06:25 -04:00
g <- lookupFree x loc !defs
2023-01-26 13:54:46 -05:00
-- if σ ≤ π
2023-05-01 21:06:25 -04:00
expectCompatQ loc sg.fst g.qty.fst
-- then Ψ | Γ ⊢ σ · x ⇒ A ⊳ 𝟎
2023-04-03 11:46:23 -04:00
let Val d = ctx.dimLen; Val n = ctx.termLen
pure $ InfRes {type = g.type, qout = zeroFor ctx}
2022-04-23 18:21:30 -04:00
2023-05-01 21:06:25 -04:00
infer' ctx sg (B i _) =
2023-01-26 13:54:46 -05:00
-- if x : A ∈ Γ
2023-02-14 15:14:47 -05:00
-- then Ψ | Γ ⊢ σ · x ⇒ A ⊳ (𝟎, σ·x, 𝟎)
2023-02-19 11:51:44 -05:00
pure $ lookupBound sg.fst i ctx.tctx
2023-05-01 21:06:25 -04:00
where
2023-04-01 13:16:43 -04:00
lookupBound : forall n. Qty -> Var n -> TContext d n -> InferResult' d n
2023-04-15 09:13:01 -04:00
lookupBound pi VZ (ctx :< type) =
InfRes {type = weakT 1 type, qout = zeroFor ctx :< pi}
2023-02-22 01:40:19 -05:00
lookupBound pi (VS i) (ctx :< _) =
let InfRes {type, qout} = lookupBound pi i ctx in
2023-04-15 09:13:01 -04:00
InfRes {type = weakT 1 type, qout = qout :< Zero}
2022-04-27 15:58:09 -04:00
2023-05-01 21:06:25 -04:00
infer' ctx sg (App fun arg loc) = do
-- if Ψ | Γ ⊢ σ · f ⇒ (π·x : A) → B ⊳ Σ₁
2023-02-19 11:51:44 -05:00
funres <- inferC ctx sg fun
2023-05-01 21:06:25 -04:00
(qty, argty, res) <- expectPi !defs ctx fun.loc funres.type
2023-02-14 15:14:47 -05:00
-- if Ψ | Γ ⊢ σ ⨴ π · s ⇐ A ⊳ Σ₂
2023-02-19 11:51:44 -05:00
argout <- checkC ctx (subjMult sg qty) arg argty
-- then Ψ | Γ ⊢ σ · f s ⇒ B[s] ⊳ Σ₁ + πΣ₂
2023-01-20 20:34:28 -05:00
pure $ InfRes {
2023-05-01 21:06:25 -04:00
type = sub1 res $ Ann arg argty arg.loc,
qout = funres.qout + qty * argout
2023-01-20 20:34:28 -05:00
}
2023-05-01 21:06:25 -04:00
infer' ctx sg (CasePair pi pair ret body loc) = do
-- no check for 1 ≤ π, since pairs have a single constructor.
-- e.g. at 0 the components are also 0 in the body
--
-- if Ψ | Γ ⊢ σ · pair ⇒ (x : A) × B ⊳ Σ₁
pairres <- inferC ctx sg pair
-- if Ψ | Γ, p : (x : A) × B ⊢₀ ret ⇐ Type
2023-04-01 13:16:43 -04:00
checkTypeC (extendTy Zero ret.name pairres.type ctx) ret.term Nothing
2023-05-01 21:06:25 -04:00
(tfst, tsnd) <- expectSig !defs ctx pair.loc pairres.type
-- if Ψ | Γ, x : A, y : B ⊢ σ · body ⇐
-- ret[(x, y) ∷ (x : A) × B/p] ⊳ Σ₂, ρ₁·x, ρ₂·y
2023-02-23 04:04:00 -05:00
-- with ρ₁, ρ₂ ≤ πσ
let [< x, y] = body.names
2023-02-23 04:04:00 -05:00
pisg = pi * sg.fst
2023-03-15 10:54:51 -04:00
bodyctx = extendTyN [< (pisg, x, tfst), (pisg, y, tsnd.term)] ctx
2023-05-01 21:06:25 -04:00
bodyty = substCasePairRet body.names pairres.type ret
bodyout <- checkC bodyctx sg body.term bodyty >>=
popQs loc [< pisg, pisg]
2023-04-15 09:13:01 -04:00
-- then Ψ | Γ ⊢ σ · caseπ ⋯ ⇒ ret[pair/p] ⊳ πΣ₁ + Σ₂
2023-01-26 13:54:46 -05:00
pure $ InfRes {
type = sub1 ret pair,
2023-03-31 13:11:35 -04:00
qout = pi * pairres.qout + bodyout
2023-01-26 13:54:46 -05:00
}
2023-05-01 21:06:25 -04:00
infer' ctx sg (CaseEnum pi t ret arms loc) {d, n} = do
-- if Ψ | Γ ⊢ σ · t ⇒ {ts} ⊳ Σ₁
tres <- inferC ctx sg t
2023-05-01 21:06:25 -04:00
ttags <- expectEnum !defs ctx t.loc tres.type
-- if 1 ≤ π, OR there is only zero or one option
2023-05-01 21:06:25 -04:00
unless (length (SortedSet.toList ttags) <= 1) $ expectCompatQ loc One pi
-- if Ψ | Γ, x : {ts} ⊢₀ A ⇐ Type
2023-04-01 13:16:43 -04:00
checkTypeC (extendTy Zero ret.name tres.type ctx) ret.term Nothing
-- if for each "a ⇒ s" in arms,
2023-03-31 13:11:35 -04:00
-- Ψ | Γ ⊢ σ · s ⇐ A[a ∷ {ts}/x] ⊳ Σᵢ
-- with Σ₂ = lubs Σᵢ
let arms = SortedMap.toList arms
let armTags = SortedSet.fromList $ map fst arms
2023-05-01 21:06:25 -04:00
unless (ttags == armTags) $ throw $ BadCaseEnum loc ttags armTags
armres <- for arms $ \(a, s) =>
2023-05-01 21:06:25 -04:00
checkC ctx sg s $ sub1 ret $ Ann (Tag a s.loc) tres.type s.loc
pure $ InfRes {
type = sub1 ret t,
2023-05-12 11:28:29 -04:00
qout = pi * tres.qout + lubs ctx armres
}
2023-05-01 21:06:25 -04:00
infer' ctx sg (CaseNat pi pi' n ret zer suc loc) = do
2023-03-26 08:40:54 -04:00
-- if 1 ≤ π
2023-05-01 21:06:25 -04:00
expectCompatQ loc One pi
2023-03-26 08:40:54 -04:00
-- if Ψ | Γ ⊢ σ · n ⇒ ⊳ Σn
nres <- inferC ctx sg n
2023-05-01 21:06:25 -04:00
let nat = nres.type
expectNat !defs ctx n.loc nat
2023-03-26 08:40:54 -04:00
-- if Ψ | Γ, n : ⊢₀ A ⇐ Type
2023-05-01 21:06:25 -04:00
checkTypeC (extendTy Zero ret.name nat ctx) ret.term Nothing
2023-03-26 08:40:54 -04:00
-- if Ψ | Γ ⊢ σ · zer ⇐ A[0 ∷ /n] ⊳ Σz
2023-05-01 21:06:25 -04:00
zerout <- checkC ctx sg zer $ sub1 ret $ Ann (Zero zer.loc) nat zer.loc
2023-03-26 08:40:54 -04:00
-- if Ψ | Γ, n : , ih : A ⊢ σ · suc ⇐ A[succ p ∷ /n] ⊳ Σs, ρ₁.p, ρ₂.ih
-- with ρ₂ ≤ π'σ, (ρ₁ + ρ₂) ≤ πσ
2023-03-26 08:40:54 -04:00
let [< p, ih] = suc.names
pisg = pi * sg.fst
2023-05-01 21:06:25 -04:00
sucCtx = extendTyN [< (pisg, p, Nat p.loc), (pi', ih, ret.term)] ctx
sucType = substCaseSuccRet suc.names ret
2023-03-26 08:40:54 -04:00
sucout :< qp :< qih <- checkC sucCtx sg suc.term sucType
2023-05-01 21:06:25 -04:00
expectCompatQ loc qih (pi' * sg.fst)
2023-03-26 08:40:54 -04:00
-- [fixme] better error here
2023-05-01 21:06:25 -04:00
expectCompatQ loc (qp + qih) pisg
2023-04-15 09:13:01 -04:00
-- then Ψ | Γ ⊢ caseπ ⋯ ⇒ A[n] ⊳ πΣn + Σz + ωΣs
2023-03-26 08:40:54 -04:00
pure $ InfRes {
type = sub1 ret n,
2023-04-01 13:16:43 -04:00
qout = pi * nres.qout + zerout + Any * sucout
2023-03-26 08:40:54 -04:00
}
2023-05-01 21:06:25 -04:00
infer' ctx sg (CaseBox pi box ret body loc) = do
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ ⊢ σ · b ⇒ [ρ.A] ⊳ Σ₁
boxres <- inferC ctx sg box
2023-05-01 21:06:25 -04:00
(q, ty) <- expectBOX !defs ctx box.loc boxres.type
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ, x : [ρ.A] ⊢₀ R ⇐ Type
2023-04-01 13:16:43 -04:00
checkTypeC (extendTy Zero ret.name boxres.type ctx) ret.term Nothing
2023-03-31 13:11:35 -04:00
-- if Ψ | Γ, x : A ⊢ t ⇐ R[[x] ∷ [ρ.A/x]] ⊳ Σ₂, ς·x
-- with ς ≤ ρπσ
let qpisg = q * pi * sg.fst
2023-04-01 10:01:29 -04:00
bodyCtx = extendTy qpisg body.name ty ctx
2023-05-01 21:06:25 -04:00
bodyType = substCaseBoxRet body.name ty ret
bodyout <- checkC bodyCtx sg body.term bodyType >>= popQ loc qpisg
2023-04-15 09:13:01 -04:00
-- then Ψ | Γ ⊢ caseπ ⋯ ⇒ R[b/x] ⊳ Σ₁ + Σ₂
2023-03-31 13:11:35 -04:00
pure $ InfRes {
type = sub1 ret box,
qout = boxres.qout + bodyout
}
2023-05-01 21:06:25 -04:00
infer' ctx sg (DApp fun dim loc) = do
-- if Ψ | Γ ⊢ σ · f ⇒ Eq [𝑖 ⇒ A] l r ⊳ Σ
2023-02-19 11:51:44 -05:00
InfRes {type, qout} <- inferC ctx sg fun
2023-05-01 21:06:25 -04:00
ty <- fst <$> expectEq !defs ctx fun.loc type
-- then Ψ | Γ ⊢ σ · f p ⇒ Ap/𝑖 ⊳ Σ
2023-01-20 20:34:28 -05:00
pure $ InfRes {type = dsub1 ty dim, qout}
2023-05-01 21:06:25 -04:00
infer' ctx sg (Coe ty p q val loc) = do
checkType (extendDim ty.name ctx) ty.term Nothing
qout <- checkC ctx sg val $ dsub1 ty p
pure $ InfRes {type = dsub1 ty q, qout}
2023-04-15 09:13:01 -04:00
2023-05-01 21:06:25 -04:00
infer' ctx sg (Comp ty p q val r (S [< j0] val0) (S [< j1] val1) loc) = do
2023-04-15 09:13:01 -04:00
checkType ctx ty Nothing
qout <- checkC ctx sg val ty
let ty' = dweakT 1 ty; val' = dweakT 1 val; p' = weakD 1 p
2023-05-01 21:06:25 -04:00
ctx0 = extendDim j0 $ eqDim r (K Zero j0.loc) ctx
2023-04-15 09:13:01 -04:00
val0 = val0.term
qout0 <- check ctx0 sg val0 ty'
2023-05-01 21:06:25 -04:00
lift $ equal loc (eqDim (B VZ p.loc) p' ctx0) ty' val0 val'
let ctx1 = extendDim j1 $ eqDim r (K One j1.loc) ctx
2023-04-15 09:13:01 -04:00
val1 = val1.term
qout1 <- check ctx1 sg val1 ty'
2023-05-01 21:06:25 -04:00
lift $ equal loc (eqDim (B VZ p.loc) p' ctx1) ty' val1 val'
2023-05-12 11:28:29 -04:00
let qouts = qout :: catMaybes [toMaybe qout0, toMaybe qout1]
pure $ InfRes {type = ty, qout = lubs ctx qouts}
2023-04-15 09:13:01 -04:00
2023-05-01 21:06:25 -04:00
infer' ctx sg (TypeCase ty ret arms def loc) = do
2023-04-03 11:46:23 -04:00
-- if σ = 0
2023-05-01 21:06:25 -04:00
expectEqualQ loc Zero sg.fst
2023-04-03 11:46:23 -04:00
-- if Ψ, Γ ⊢₀ e ⇒ Type u
2023-05-01 21:06:25 -04:00
u <- expectTYPE !defs ctx ty.loc . type =<< inferC ctx szero ty
2023-04-15 09:13:01 -04:00
-- if Ψ, Γ ⊢₀ C ⇐ Type (non-dependent return type)
2023-04-03 11:46:23 -04:00
checkTypeC ctx ret Nothing
2023-04-15 09:13:01 -04:00
-- if Ψ, Γ' ⊢₀ A ⇐ C for each rhs A
for_ allKinds $ \k =>
for_ (lookupPrecise k arms) $ \(S names t) =>
2023-05-01 21:06:25 -04:00
check0 (extendTyN (typecaseTel k names u) ctx)
2023-04-15 09:13:01 -04:00
t.term (weakT (arity k) ret)
2023-04-03 11:46:23 -04:00
-- then Ψ, Γ ⊢₀ type-case ⋯ ⇒ C
pure $ InfRes {type = ret, qout = zeroFor ctx}
2023-05-01 21:06:25 -04:00
infer' ctx sg (Ann term type loc) = do
-- if Ψ | Γ ⊢₀ A ⇐ Type
checkTypeC ctx type Nothing
-- if Ψ | Γ ⊢ σ · s ⇐ A ⊳ Σ
2023-02-19 11:51:44 -05:00
qout <- checkC ctx sg term type
-- then Ψ | Γ ⊢ σ · (s ∷ A) ⇒ A ⊳ Σ
2023-01-20 20:34:28 -05:00
pure $ InfRes {type, qout}