luau/prototyping/Luau/AddrCtxt.agda
2022-02-10 16:53:59 -06:00

15 lines
334 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)
AddrCtxt : Set
AddrCtxt = Vector Type
: AddrCtxt
= empty
_[_] : AddrCtxt Addr Maybe Type
_[_] = lookup