mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 01:01:59 +03:00
7 lines
328 B
Plaintext
7 lines
328 B
Plaintext
1/1: Building Issue2072 (Issue2072.idr)
|
|
Main> 2 holes:
|
|
Main.Types : (0 a : Type) -> Eq a => List Type
|
|
Main.body : {auto 0 conArg : Eq t1} -> {auto 0 _ : Elem Bool (Types t1)} -> (obj : t1) -> obj == obj = maybe (Delay True) (Delay (const False)) (if obj == obj then pure (let x = True in ()) else empty)
|
|
Main>
|
|
Bye for now!
|