Skip to content

Hovering on syntax-less attributes shows no docstring #8432

Open
@nomeata

Description

@nomeata

Attriubutes like elab_as_elim that don't have dedicated : attr syntax don’t show anything useful when hovering on them (they show the generic “declModifiers is the collection of modifiers on a declaration:” docstring):

@[elab_as_elim] theorem subst {p : (b : α) → a = b → Prop} (h₁ : a = b) (h₂ : p a rfl) : p b h₁ := by
  cases h₁
  assumption

This is unfortunate, since these attributes do have an descr passed to registerBuiltinAttribute.

It would be good if that could be surfaced here somehow, and also make Ctrl-Click work.

Versions

Lean 4.21.0-nightly-2025-05-21

Impact

Add 👍 to issues you consider important. If others are impacted by this issue, please ask them to add 👍 to it.

Metadata

Metadata

Assignees

No one assigned

    Labels

    P-mediumWe may work on this issue if we find the timebugSomething isn't working

    Type

    No type

    Projects

    No projects

    Milestone

    No milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions