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
I have vscoqtop version 2.2.3 with coq version 8.20.1 installed with the vscoq extension version 2.2.3.
When running in continous mode I can evaluate a proof. However, when I try to step through a proof with my cursor it vscoqtop crashes with the following error:
[top , 466313, 1739460348.381356] ==========================================================
[top , 466313, 1739460348.381404] Uncaught exception Failure("tag not closed").
[top , 466313, 1739460348.381408] ==========================================================
[Error - 16:25:48] Server process exited with code 0.
An example short script which causes this for me is:
Lemma test : False = True -> True.
Proof.
intros H.
Admitted.
Where moving the cursor from before intros H. to after it crashes vscoqtop.
Strangely when the lemma is Lemma test : True -> True., this does work.
The same problem also occurs in manual mode when evaluating the intros tactic.
The text was updated successfully, but these errors were encountered:
lukovdm
changed the title
vscoqtop crashes when showing proof state after a tactic
vscoqtop crashes when showing proof state after certain tactics
Feb 13, 2025
I have vscoqtop version 2.2.3 with coq version 8.20.1 installed with the vscoq extension version 2.2.3.
When running in continous mode I can evaluate a proof. However, when I try to step through a proof with my cursor it vscoqtop crashes with the following error:
An example short script which causes this for me is:
Where moving the cursor from before
intros H.
to after it crashes vscoqtop.Strangely when the lemma is
Lemma test : True -> True.
, this does work.The same problem also occurs in manual mode when evaluating the intros tactic.
The text was updated successfully, but these errors were encountered: