2015-12-07 20:39:51 +00:00
|
|
|
|
definition Sum_weird [forward] : ∀ (f g h : ℕ → ℕ) (n : ℕ), Sum n (λ (x : ℕ), f (g (h x))) = 1 :=
|
2016-06-01 02:14:42 +00:00
|
|
|
|
λ f g h n, sorry
|
2015-12-07 20:39:51 +00:00
|
|
|
|
(multi-)patterns:
|
|
|
|
|
?M_1 : ℕ → ℕ, ?M_2 : ℕ → ℕ, ?M_3 : ℕ → ℕ, ?M_4 : ℕ
|
2016-06-01 02:14:42 +00:00
|
|
|
|
{Sum ?M_4 (λ x, ?M_1 (?M_2 (?M_3 x)))}
|