Idris2/tests/idris2/pkg007/A/Path/Of/Dires/First.idr
2021-04-15 14:08:50 +01:00

9 lines
148 B
Idris

module A.Path.Of.Dires.First
%default total
public export
data Tree : Type -> Type where
Leaf : a -> Tree a
Node : Tree a -> Tree a -> Tree a