Idris2/libs/contrib/Syntax/WithProof.idr

10 lines
208 B
Idris
Raw Normal View History

2020-05-18 15:59:07 +03:00
module Syntax.WithProof
prefix 10 @@
2020-05-18 15:59:07 +03:00
||| Until Idris2 supports the 'with (...) proof p' construct, here's a
||| poor-man's replacement.
public export
2021-01-16 17:18:34 +03:00
(@@) : (t : a) -> (u : a ** t = u)
(@@) x = (x ** Refl)