Idris2/tests/ttimp/record004/Record.yaff

16 lines
221 B
Plaintext
Raw Normal View History

data Nat : Type where
Z : Nat
S : Nat -> Nat
namespace A
public export
record Dup where
constructor MkDup
label : Nat
namespace B
public export
record Dup where
constructor MkDup
label : Nat