14 lines
301 B
Text
14 lines
301 B
Text
|
definition foo₁ [forward] : ∀ (x : ℕ), f x ∧ g x :=
|
|||
|
sorry
|
|||
|
(multi-)patterns:
|
|||
|
{f ?M_1}
|
|||
|
{g ?M_1}
|
|||
|
definition foo₂ [forward] : ∀ (x : ℕ), (:f x:) ∧ g x :=
|
|||
|
sorry
|
|||
|
(multi-)patterns:
|
|||
|
{f ?M_1}
|
|||
|
definition foo₃ [forward] : ∀ (x : ℕ), (:f (id x):) ∧ g x :=
|
|||
|
sorry
|
|||
|
(multi-)patterns:
|
|||
|
{f ?M_1}
|