agda-spa/Main.agda

26 lines
538 B
Plaintext
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

module Main where
open import Language
open import Analysis.Sign
open import Data.Vec using (Vec; _∷_; [])
open import IO
open import Level using (0)
testCode : Vec Stmt _
testCode =
("zero" ← (# 0)) ∷
("pos" ← ((` "zero") Expr.+ (# 1))) ∷
("neg" ← ((` "zero") Expr.- (# 1))) ∷
("unknown" ← ((` "pos") Expr.+ (` "neg"))) ∷
[]
testProgram : Program
testProgram = record
{ length = _
; stmts = testCode
}
open WithProg testProgram using (output)
main = run {0} (putStrLn output)