6 lines
290 B
Text
6 lines
290 B
Text
|
definition Sum_weird [forward] : ∀ (f g h : ℕ → ℕ) (n : ℕ), Sum n (λ (x : ℕ), f (g (h x))) = 1 :=
|
|||
|
λ (f g h : ℕ → ℕ) (n : ℕ), sorry
|
|||
|
(multi-)patterns:
|
|||
|
?M_1 : ℕ → ℕ, ?M_2 : ℕ → ℕ, ?M_3 : ℕ → ℕ, ?M_4 : ℕ
|
|||
|
{Sum ?M_4 (λ (x : ℕ), ?M_1 (?M_2 (?M_3 x)))}
|