Please enable JavaScript in your browser!
Home
Esplora
Aiuto
Accedi
caryoscelus
/
agda
Segui
1
Vota
0
Forka
0
File
Problemi
0
Pull Requests
0
Wiki
Albero (Tree):
ce9b406819
Rami (Branch)
Tag
js_amd
js_amd_patch
working
agda
/
test
/
Compiler
/
simple
/
Issue2222.agda
Issue2222.agda
81 B
Cronologia
Originale
1
2
3
4
5
6
7
open import Common.IO
header = putStrLn "foo"
main : IO _
main = putStrLn "42"