lean2/tests/lean/interactive/t1.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

23 lines
No EOL
751 B
Text

# Set: pp::colors
Set: pp::unicode
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a ∧ b
## [stdin]:5:0: error: failed to create proof for the following proof state
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a ∧ b
## [stdin]:6:0: error: failed to create proof for the following proof state
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a ∧ b
## [stdin]:7:0: error: unknown tactic 'imp_tac2'
## [stdin]:8:0: error: unknown tactic 'foo'
## Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a
a : Bool, b : Bool, H : a, H::1 : b ⊢ b
## [stdin]:10:0: error: failed to backtrack
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a
a : Bool, b : Bool, H : a, H::1 : b ⊢ b
## Proof state:
no goals
## Proved: T2
#