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