5 lines
85 B
Text
5 lines
85 B
Text
import data.nat
|
|
open nat
|
|
|
|
example (a b : nat) : 0 + a + b + 1 = 1 + a + b :=
|
|
by simp
|