lean2/tests/lean/run/592.lean

8 lines
143 B
Text
Raw Normal View History

import data.nat
open nat algebra
definition foo (a b : nat) := a * b
example (a : nat) : foo a 0 = 0 :=
calc a * 0 = 0 : by rewrite mul_zero