leanprover-community / lean4web

The Lean 4 web editor
https://live.lean-lang.org/
Apache License 2.0
52 stars 14 forks source link

infoview "copy message to comment" looses stuff #13

Closed joneugster closed 6 months ago

joneugster commented 7 months ago

See Zulip.

In the following example, the infoview button "copy message to comment" copies an incomplete error message to context.

import Mathlib

example : 1 + 1 = 2 := Nat.add_one
joneugster commented 7 months ago

Seems to be specific to error messages.

In the following, it works fine:

import Mathlib

example : 1 + 1 = 2 := Nat.add_one _
abentkamp commented 7 months ago

We'll need a new release of the @leanprover/infoview npm package. I have written to Wojciech about this.