Idris2/libs/contrib/Syntax/WithProof.idr
2020-05-29 10:37:04 +01:00

10 lines
210 B
Idris

module Syntax.WithProof
prefix 10 @@
||| Until Idris2 supports the 'with (...) proof p' construct, here's a
||| poor-man's replacement.
public export
(@@) : (t : a ) -> (u : a ** t = u)
(@@) x = ( x ** Refl)