Idris2/tests/idris2/interface/interface029/ForwardImpl2.idr
2023-09-07 14:57:22 +01:00

17 lines
304 B
Idris

interface IsEven a where
isEven : a -> Bool
interface IsOdd b where
isOdd : b -> Bool
implementation IsOdd Nat
implementation IsEven Nat where
isEven 0 = True
isEven (S k) = not $ isOdd k
implementation Show Nat => IsOdd Nat where
isOdd 0 = True
isOdd (S k) = not $ isEven k