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

8 lines
227 B
Idris

module A
-- Check that this doesn't go into a loop when resolving Show. because
-- f itself is a candidate when elaborating the top level f function!
public export
interface F (p : Type -> Type) where
f : Show a => p a -> a