mirror of
https://github.com/luau-lang/luau.git
synced 2024-11-15 22:35:43 +08:00
7f867ac166
Adds number support to the prototype. Binary operators are next.
9 lines
351 B
Agda
9 lines
351 B
Agda
module Examples.OpSem where
|
|
|
|
open import Luau.OpSem using (_⊢_⟶ᴱ_⊣_; _⊢_⟶ᴮ_⊣_; subst)
|
|
open import Luau.Syntax using (Block; var; nil; local_←_; _∙_; done; return; block_is_end)
|
|
open import Luau.Heap using (∅)
|
|
|
|
ex1 : ∅ ⊢ (local (var "x") ← nil ∙ return (var "x") ∙ done) ⟶ᴮ (return nil ∙ done) ⊣ ∅
|
|
ex1 = subst
|