mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-29 03:24:02 +03:00
11 lines
152 B
Idris
11 lines
152 B
Idris
%logging "declare.def.lhs" 10
|
|
|
|
|
|
data Tup : (a,b : Type) -> Type where
|
|
MkTup : (1 f : a) -> (1 s : b) -> Tup a b
|
|
|
|
f : Tup a b -> a
|
|
f (MkTup f s) = f
|
|
|
|
|