mirror of
https://github.com/luau-lang/luau.git
synced 2025-05-04 10:33:46 +01:00
31 lines
786 B
Agda
31 lines
786 B
Agda
module Luau.VarCtxt where
|
||
|
||
open import Luau.Type using (Type; _∪_; _∩_)
|
||
open import Luau.Var using (Var)
|
||
open import FFI.Data.Aeson using (KeyMap; Key; empty; unionWith; singleton; insert; delete; lookup; fromString)
|
||
open import FFI.Data.Maybe using (Maybe; just; nothing)
|
||
|
||
VarCtxt : Set
|
||
VarCtxt = KeyMap Type
|
||
|
||
∅ : VarCtxt
|
||
∅ = empty
|
||
|
||
_⋒_ : VarCtxt → VarCtxt → VarCtxt
|
||
_⋒_ = unionWith _∩_
|
||
|
||
_⋓_ : VarCtxt → VarCtxt → VarCtxt
|
||
_⋓_ = unionWith _∪_
|
||
|
||
_[_] : VarCtxt → Var → Maybe Type
|
||
_[_] Γ x = lookup (fromString x) Γ
|
||
|
||
_⊝_ : VarCtxt → Var → VarCtxt
|
||
Γ ⊝ x = delete (fromString x) Γ
|
||
|
||
_↦_ : Var → Type → VarCtxt
|
||
x ↦ T = singleton (fromString x) T
|
||
|
||
_⊕_↦_ : VarCtxt → Var → Type → VarCtxt
|
||
Γ ⊕ x ↦ T = insert (fromString x) T Γ
|
||
|