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

13 lines
338 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
## stdin:5:0 error: unknown tactic 'foo'
## stdin:6:5 error: 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
#