lean2/tests/lean/tuple.lean

10 lines
156 B
Text
Raw Normal View History

import data.prod
open nat prod
set_option pp.universes true
definition tuple (A : Type) (n : nat) : Type :=
nat.rec_on n A (λ n r, r × A)
check @tuple