Idris2/tests/idris2/misc/pretty001/Issue1328A.idr
André Videla 75032a7164
Emit warning for fixities with no export modifiers (#3234)
* Emit warning for fixities with no export modifiers

This is to help update all the existing code to program with explicit
fixity export directives in preparation for the behavioral change where
they will become private by default.
2024-04-03 15:41:57 +01:00

45 lines
664 B
Idris

module Issue1328A
%default total
private infix 4 `InCtx`
data InCtx : (a, b : Type) -> Type where
prop0 : a `InCtx` b
prop0 = ?undef_0
prop1 : (`InCtx` b) a
prop1 = ?undef_1
prop2 : (a `InCtx`) b
prop2 = ?undef_2
def0 : (m, n : Integer) -> Integer
def0 m n = m `div` n
def1 : (m, n : Integer) -> Integer
def1 m n = (`div` n) m
def2 : (m, n : Integer) -> Integer
def2 m n = (m `div`) n
private infix 4 |-
data (|-) : (a, b : Type) -> Type where
inProp0 : a |- b
inProp0 = ?undef_3
inProp1 : (|- b) a
inProp1 = ?undef_4
inProp2 : (a |-) b
inProp2 = ?undef_5
inDef0 : Nat
inDef0 = 42 + 21
inDef1 : Nat
inDef1 = (+ 21) 42
inDef2 : Nat
inDef2 = (42 +) 21