ba9a8f9d98
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
18 lines
No EOL
430 B
Text
18 lines
No EOL
430 B
Text
variables a b c d : Nat
|
|
axiom H : a + (b + c) = a + (b + d)
|
|
|
|
set_option pp::implicit true
|
|
|
|
using Nat
|
|
check add_succr a
|
|
|
|
scope
|
|
|
|
theorem mul_zerol2 (a : Nat) : 0 * a = 0
|
|
:= induction_on a
|
|
(show 0 * 0 = 0, from mul_zeror 0)
|
|
(λ (n : Nat) (iH : 0 * n = 0),
|
|
calc 0 * (n + 1) = (0 * n) + 0 : mul_succr 0 n
|
|
... = 0 + 0 : { iH }
|
|
... = 0 : add_zeror 0)
|
|
end |