mirror of
https://github.com/luau-lang/luau.git
synced 2025-05-04 10:33:46 +01:00
15 lines
334 B
Agda
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
|