mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-11 06:14:41 +03:00
a972778eab
They don't all pass yet, for minor reasons. Coming shortly... Unfortunately the startup overhead for chez is really noticeable here!
933 B
933 B
My First Idris2 Program
This is a literate Idris2 Org-Mode file that the Idris2 understands.
We can have visibile code blocks using source blocks in idris.
data Natural = Zero | Succ Natural
data Vect : Natural -> Type -> Type where
Empty : Vect Zero a
Cons : a -> Vect k a -> Vect (Succ k) a
We can have hidden literate lines that Idris will understand.
However, we Idris2' literate support is greedy and does not understand all of the supported literate modes comments and verbatim blocks.
Thus:
#+IDRIS: plus : Natural -> Natural -> Natural
is also an active code line.
We can also abuse org-mode comments to hide code not required for publication.
cannotSeeThis : Natural -> Natural
main : IO ()
main = putStrLn "Hello!"