lean2/tests/lean/run/secnot.lean
2014-10-09 07:13:06 -07:00

25 lines
395 B
Text

import data.num
section
variable {A : Type}
definition f (a b : A) := a
infixl `◀`:65 := f
variables a b : A
check a ◀ b
end
inductive list (T : Type) : Type :=
nil {} : list T,
cons : T → list T → list T
namespace list
section
variable {T : Type}
notation `[` l:(foldr `,` (h t, cons h t) nil) `]` := l
check [10, 20, 30]
end
end list
open list
check [10, 20, 40]
check 10 ◀ 20