lean2/tests/lean/run/abstract_notation.lean

12 lines
178 B
Text
Raw Normal View History

import data.nat
open nat
notation `$`:max := abstract by blast end
definition foo (a b : nat) : a + b = b + a ∧ a = 0 + a :=
and.intro $ $
check foo_1
check foo_2
print foo