luau/prototyping/Luau/AddrCtxt.agda
2022-02-11 18:24:02 -06:00

16 lines
385 B
Agda

module Luau.AddrCtxt where
open import Luau.Type using (Type)
open import Luau.Addr using (Addr)
open import FFI.Data.Vector using (Vector; empty; lookup)
open import FFI.Data.Maybe using (Maybe; just; nothing)
open import Luau.VarCtxt using (orNone)
AddrCtxt : Set
AddrCtxt = Vector Type
: AddrCtxt
= empty
_[_] : AddrCtxt Addr Type
Σ [ a ] = orNone(lookup Σ a)