2 lines
103 B
Text
2 lines
103 B
Text
definition nat.add : ℕ → ℕ → ℕ :=
|
||
λ (a b : ℕ), nat.rec_on b a (λ (b₁ : ℕ), nat.succ)
|