mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-15 22:32:19 +03:00
8ddac9c1d5
We need to make sure they are inferred again when elaborating methods, so substitute in a _ in method types before substituting in the explicit parameters. In future, it might (probably will) also be useful to allow giving the implicit parameters explicitly when defining implementations. Fixes #374
13 lines
226 B
Idris
13 lines
226 B
Idris
module Meh
|
|
|
|
import public Control.WellFounded
|
|
|
|
public export
|
|
interface Argh (rel : a -> a -> Type) where
|
|
argh : (x : a) -> Accessible rel x
|
|
|
|
data Meh : Nat -> Nat -> Type where
|
|
|
|
implementation Argh Meh where
|
|
argh x = ?foo
|