vscode-lean4
vscode-lean4 copied to clipboard
Popups for huge expressions are shown outside of viewport
def N : Nat := Nat.add 37 50
example : N ≠ N := by
simp (config := {decide := false}) only [N, Nat.add]
/- Put cursor on `≠` in infoview -/
sorry
When highlighting a subterm that is multiple pages long, the popup gets shown at the beginning of the subterm, which is outside of the viewport.
