Haskell.agda 94 B

12345678
  1. module Issue2486.Haskell where
  2. {-# FOREIGN GHC
  3. data MyList a = Nil | Cons a (MyList a)
  4. #-}