Idris2/tests/idris2/basic/basic003/Ambig2.idr
André Videla 75032a7164
Emit warning for fixities with no export modifiers (#3234)
* Emit warning for fixities with no export modifiers

This is to help update all the existing code to program with explicit
fixity export directives in preparation for the behavioral change where
they will become private by default.
2024-04-03 15:41:57 +01:00

27 lines
421 B
Idris

private infixr 5 ::
export
data List a = Nil | (::) a (List a)
export
data Nat = Z | S Nat
export
data Vect : Type -> Type where
export
data Set : Type -> Type where
namespace Vect
export
toList : Vect a -> List a
export
fromList : List a -> Vect a
namespace Set
export
toList : Set a -> List a
export
fromList : List a -> Set a
keepUnique : List b -> List b
keepUnique {b} xs = toList (fromList xs)