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
Goalforall A B C D E F : Prop, A -> B -> C -> D -> E -> F -> A.
Proof.
intros A B C D E F.
intros HA; intros HB; intros HC; intros HD; intros HE; intros HF; exact HA.
Qed.
if I execute everything
if I try to break the line after HE;
The interface goes into an inconsistent state
The text was updated successfully, but these errors were encountered:
I think the range stuff was not invalidated since the document is not.
The code did detect that the texts parses to the same token list, so no need to recompute.
But since the new text is different in length/number-of-lines, the highlighting state needs to be invalidated hence recomputed.
Here is my example
if I execute everything
if I try to break the line after
HE;
The interface goes into an inconsistent state
The text was updated successfully, but these errors were encountered: