You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
In Propositions and Proofs, when the suffices keyword is introduced, the text reads, "Writing suffices hq : q leaves us with two goals.". I was expecting, in the style of using Coq, to see those two goals explicitly shown in the context window/infoview. However, the incomplete example does not do so: there is still only one goal, and it appears to be unchanged from the previous line.
variable (p q : Prop)
example (h : p ∧ q) : q ∧ p :=
have hp : p := h.left
suffices hq : q
Expected type
pq: Prop
h: p ∧ q
⊢ q ∧ p
Is there a different infoview that I should be using that the text doesn't explicitly call out? Or, has this behaviour since changed?
Dear all,
In Propositions and Proofs, when the
suffices
keyword is introduced, the text reads, "Writingsuffices hq : q
leaves us with two goals.". I was expecting, in the style of using Coq, to see those two goals explicitly shown in the context window/infoview. However, the incomplete example does not do so: there is still only one goal, and it appears to be unchanged from the previous line.Is there a different infoview that I should be using that the text doesn't explicitly call out? Or, has this behaviour since changed?
Version
#eval Lean.versionString:
4.0.0, commit 96de208a6b1a575b3f07d978965573d5b6fad454
The text was updated successfully, but these errors were encountered: