lean2/tests/lean/interactive/t10.lean.expected.out
Leonardo de Moura a51139e63b feat(frontends/lean): position information in error messages
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-02-06 17:26:38 -08:00

20 lines
642 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: failed to create proof for the following proof 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