Idris2/tests/idris2/operators/operators010/Test.idr
2024-04-04 16:08:23 +01:00

11 lines
156 B
Idris

import Language.Reflection
%default total
%language ElabReflection
export infix 6 `op`
%runElab logSugaredTerm "debug" 0 "term with infix" `(a `op` b)