lean2/tests/lean/check_expr.lean

9 lines
141 B
Text
Raw Normal View History

import data.list
open sigma list
theorem foo (A : Type) (l : list A): A → A → list A :=
begin
intros [a, b],
check_expr (a::l),
end