1
1
mirror of https://github.com/idris-lang/Idris2.git synced 2024-12-20 01:41:44 +03:00
Idris2/libs/contrib/Syntax/WithProof.idr

9 lines
209 B
Idris
Raw Normal View History

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