mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 16:21:46 +03:00
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
|