lean2/tests/lean/pattern_pp.lean.expected.out

6 lines
290 B
Text
Raw Normal View History

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)))}