2015-12-02 19:28:45 -07:00
|
|
|
|
definition foo₁ [forward] : ∀ (x : ℕ), f x ∧ g x :=
|
|
|
|
|
sorry
|
|
|
|
|
(multi-)patterns:
|
2015-12-07 11:51:44 -08:00
|
|
|
|
?M_1 : ℕ
|
2015-12-02 19:28:45 -07:00
|
|
|
|
{g ?M_1}
|
2016-02-10 17:17:22 -08:00
|
|
|
|
{f ?M_1}
|
2015-12-02 19:28:45 -07:00
|
|
|
|
definition foo₂ [forward] : ∀ (x : ℕ), (:f x:) ∧ g x :=
|
|
|
|
|
sorry
|
|
|
|
|
(multi-)patterns:
|
2015-12-07 11:51:44 -08:00
|
|
|
|
?M_1 : ℕ
|
2015-12-02 19:28:45 -07:00
|
|
|
|
{f ?M_1}
|
|
|
|
|
definition foo₃ [forward] : ∀ (x : ℕ), (:f (id x):) ∧ g x :=
|
|
|
|
|
sorry
|
|
|
|
|
(multi-)patterns:
|
2015-12-07 11:51:44 -08:00
|
|
|
|
?M_1 : ℕ
|
2015-12-02 19:28:45 -07:00
|
|
|
|
{f ?M_1}
|