lean2/tests/lean/show_tac.lean.expected.out
Leonardo de Moura c133d26505 feat(frontends/lean/builtin_exprs): change how 'show' is processed in tactics
Unresolved placeholders were not being reported
2015-05-19 16:23:50 -07:00

18 lines
536 B
Text

show_tac.lean:6:29: error: don't know how to synthesize placeholder
a b : Prop,
Hab : a ∧ b,
Ha : a,
Hb : b
⊢ b
show_tac.lean:6:2: error:invalid 'exact' tactic, term still contains metavariables after elaboration
show b ∧ a, from and.intro ?M_1 Ha
proof state:
a b : Prop,
Hab : a ∧ b,
Ha : a,
Hb : b
⊢ b ∧ a
show_tac.lean:7:0: error: failed to add declaration '14.0' to environment, value has metavariables
remark: set 'formatter.hide_full_terms' to false to see the complete term
λ (a b : Prop) (Hab : …),
?M_1