2013-10-31 23:27:36 +00:00
|
|
|
|
Set: pp::colors
|
|
|
|
|
Set: pp::unicode
|
|
|
|
|
Assumed: i
|
|
|
|
|
λ x : ℤ, x + i : ℤ → ℤ
|
|
|
|
|
λ x : ℕ, x + 1 : ℕ → ℕ
|
2013-12-21 06:00:50 +00:00
|
|
|
|
Error (line: 4, pos: 10) invalid expression, it still contains metavariables after elaboration, metavariable: ?M::0, type:
|
|
|
|
|
(Type U)
|
2013-10-31 23:27:36 +00:00
|
|
|
|
λ x y : ℤ, y + i + 1 + x : ℤ → ℤ → ℤ
|
|
|
|
|
(λ x : ℤ, x) i : ℤ
|
|
|
|
|
(λ x : ℤ → ℤ → ℤ, x i) (λ x y : ℤ, x + 1 + y) : ℤ → ℤ
|
|
|
|
|
(λ x : ℕ → ℕ → ℕ, x) (λ x y : ℕ, x + 1 + y) : ℕ → ℕ → ℕ
|