mirror of
https://github.com/luau-lang/luau.git
synced 2024-12-13 13:30:40 +00:00
cd18adc20e
Adds support for binary operations on numbers.
27 lines
1.4 KiB
Agda
27 lines
1.4 KiB
Agda
module Luau.RuntimeError where
|
|
|
|
open import Agda.Builtin.Equality using (_≡_)
|
|
open import Luau.Heap using (Heap; _[_])
|
|
open import FFI.Data.Maybe using (just; nothing)
|
|
open import FFI.Data.String using (String)
|
|
open import Luau.Syntax using (Block; Expr; nil; var; addr; block_is_end; _$_; local_←_; return; done; _∙_; number; binexp)
|
|
open import Luau.RuntimeType using (RuntimeType; valueType)
|
|
open import Luau.Value using (val)
|
|
open import Properties.Equality using (_≢_)
|
|
|
|
data RuntimeErrorᴮ {a} (H : Heap a) : Block a → Set
|
|
data RuntimeErrorᴱ {a} (H : Heap a) : Expr a → Set
|
|
|
|
data RuntimeErrorᴱ H where
|
|
TypeMismatch : ∀ t v → (t ≢ valueType v) → RuntimeErrorᴱ H (val v)
|
|
UnboundVariable : ∀ x → RuntimeErrorᴱ H (var x)
|
|
SEGV : ∀ a → (H [ a ] ≡ nothing) → RuntimeErrorᴱ H (addr a)
|
|
app₁ : ∀ {M N} → RuntimeErrorᴱ H M → RuntimeErrorᴱ H (M $ N)
|
|
app₂ : ∀ {M N} → RuntimeErrorᴱ H N → RuntimeErrorᴱ H (M $ N)
|
|
block : ∀ b {B} → RuntimeErrorᴮ H B → RuntimeErrorᴱ H (block b is B end)
|
|
bin₁ : ∀ {M N op} → RuntimeErrorᴱ H M → RuntimeErrorᴱ H (binexp M op N)
|
|
bin₂ : ∀ {M N op} → RuntimeErrorᴱ H N → RuntimeErrorᴱ H (binexp M op N)
|
|
|
|
data RuntimeErrorᴮ H where
|
|
local : ∀ x {M B} → RuntimeErrorᴱ H M → RuntimeErrorᴮ H (local x ← M ∙ B)
|
|
return : ∀ {M B} → RuntimeErrorᴱ H M → RuntimeErrorᴮ H (return M ∙ B)
|