lean2/tests/lean/interactive/t10.lean.expected.out
Leonardo de Moura f7c7dd4ed4 feat(frontends/lean): include filename in error messages, use GNU error message style
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-09 11:01:27 -08:00

20 lines
645 B
Text

# Set: pp::colors
Set: pp::unicode
Proof state:
A : Bool, B : Bool, H : A ∧ B ⊢ A
## Proof state:
no goals
## Proof state:
A : Bool, B : Bool, H : A ∧ B, H1 : A ⊢ B
## stdin:15:3 error: unknown tactic 'simple2_tac'
## stdin:15:16 error: invalid 'done' command, proof cannot be produced from this state
Proof state:
A : Bool, B : Bool, H : A ∧ B, H1 : A ⊢ B
## Proof state:
no goals
## Proof state:
A : Bool, B : Bool, H : A ∧ B, H1 : A, H2 : B ⊢ B ∧ A
## stdin:18:0 error: failed to prove theorem, proof has been aborted
Proof state:
A : Bool, B : Bool, H : A ∧ B, H1 : A, H2 : B ⊢ B ∧ A
# echo command after failure