Open
Description
In a proof of example (a b : Nat) (_ : a ≤ b ∧ b ≤ c) (_ : 0 < a) (_ : c < 3) : 0 < a ∧ a < 3
I have to use apply And.intro
and then apply linarith
separately to both goals. I think we could consider automatically splitting And with linarith
.
One problem I can see, is that linarith
is able to prove one part of And, and not the other, it would still fail. It might be a good idea to also report in the error which parts it managed to solve.
Metadata
Metadata
Assignees
Labels
No labels