1
1
mirror of https://github.com/idris-lang/Idris2.git synced 2025-01-08 00:40:10 +03:00
Idris2/tests/idris2/reg033/test.idr

14 lines
250 B
Idris
Raw Normal View History

import Language.Reflection
import DerivingEq
%language ElabReflection
-- This tree doesn't work
data TreeTwo a = BranchTwo (TreeTwo a) a (TreeTwo a)
| Leaf
covering
Eq a => Eq (TreeTwo a) where
(==) = %runElab genEq `{ TreeTwo }