lean2/tests/lean/interactive/t2.lean.expected.out

13 lines
352 B
Text
Raw Normal View History

# Set: pp::colors
Set: pp::unicode
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a ∧ b
## Error (line: 5, pos: 0) unknown tactic 'foo'
## Error (line: 6, pos: 5) failed to prove theorem, proof has been aborted
Proof state:
a : Bool, b : Bool, H : a, H::1 : b ⊢ a ∧ b
# Assumed: a
Assumed: b
# variable a : Bool
variable b : Bool
#