lean2/tests/lean/pattern_hint1.lean.expected.out

17 lines
334 B
Text
Raw Permalink Normal View History

definition foo₁ [forward] : ∀ (x : ), f x ∧ g x :=
sorry
(multi-)patterns:
?M_1 :
{g ?M_1}
{f ?M_1}
definition foo₂ [forward] : ∀ (x : ), (:f x:) ∧ g x :=
sorry
(multi-)patterns:
?M_1 :
{f ?M_1}
definition foo₃ [forward] : ∀ (x : ), (:f (id x):) ∧ g x :=
sorry
(multi-)patterns:
?M_1 :
{f ?M_1}