2015-03-13 03:28:56 +00:00
|
|
|
|
rewrite_fail.lean:5:15: error:invalid 'rewrite' tactic, rewrite step failed using pattern
|
|
|
|
|
a
|
|
|
|
|
no subterm in the goal matched the pattern
|
2015-02-17 00:56:42 +00:00
|
|
|
|
proof state:
|
|
|
|
|
a b : ℕ,
|
|
|
|
|
Ha : a = 0,
|
|
|
|
|
Hb : b = 0
|
|
|
|
|
⊢ 0 + b = 0
|
|
|
|
|
rewrite_fail.lean:6:0: error: don't know how to synthesize placeholder
|
|
|
|
|
a b : ℕ,
|
|
|
|
|
Ha : a = 0,
|
|
|
|
|
Hb : b = 0
|
|
|
|
|
⊢ a + b = 0
|
|
|
|
|
rewrite_fail.lean:6:0: error: failed to add declaration '14.0' to environment, value has metavariables
|
2015-03-13 19:42:57 +00:00
|
|
|
|
remark: set 'formatter.hide_full_terms' to false to see the complete term
|
|
|
|
|
λ (a b : ℕ) (Ha : …) (Hb : …),
|
2015-02-17 00:56:42 +00:00
|
|
|
|
?M_1
|
|
|
|
|
rewrite_fail.lean:11:2: error:invalid tactic, there are no goals to be solved
|
|
|
|
|
proof state:
|
|
|
|
|
no goals
|
|
|
|
|
rewrite_fail.lean:12:0: error: don't know how to synthesize placeholder
|
|
|
|
|
a : ℕ
|
|
|
|
|
⊢ a = a
|
|
|
|
|
rewrite_fail.lean:12:0: error: failed to add declaration '14.1' to environment, value has metavariables
|
2015-03-13 19:42:57 +00:00
|
|
|
|
remark: set 'formatter.hide_full_terms' to false to see the complete term
|
2015-02-17 00:56:42 +00:00
|
|
|
|
λ (a : ℕ),
|
|
|
|
|
?M_1
|