mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 00:10:31 +03:00
14 lines
320 B
Idris
14 lines
320 B
Idris
module Issue735
|
|
|
|
-- Not allowed to pattern-match on under-applied constructors
|
|
isCons : (a -> List a -> List a) -> Bool
|
|
isCons (::) = True
|
|
isCons _ = False
|
|
|
|
interface A a where
|
|
|
|
-- Not allowed to pattern-match on under-applied type constructors
|
|
test : (kind : Type -> Type) -> Maybe Nat
|
|
test A = Just 1
|
|
test _ = Nothing
|