Documentation

Lean.Server.InfoUtils

structure String.Range:
Type
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.InfoTree.visitM {m : TypeType u_1} {α : Type} [inst : Monad m] [inst : Inhabited α] (preNode : optParam (Lean.Elab.ContextInfoLean.Elab.InfoStd.PersistentArray Lean.Elab.InfoTreem Unit) fun x x x => pure ()) (postNode : Lean.Elab.ContextInfoLean.Elab.InfoStd.PersistentArray Lean.Elab.InfoTreeList (Option α)m α) :

Visit nodes, passing in a surrounding context (the innermost one) and accumulating results on the way back up.

Equations

Visit nodes bottom-up, passing in a surrounding context (the innermost one) and the union of nested results (empty at leaves).

Equations

For every branch of the InfoTree, find the deepest node in that branch for which p returns some _ and return the union of all such nodes. The visitor p is given a node together with its innermost surrounding ContextInfo.

Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.InfoTree.foldInfo {α : Type u_1} (f : Lean.Elab.ContextInfoLean.Elab.Infoαα) (init : α) :
Equations
partial def Lean.Elab.InfoTree.foldInfo.go {α : Type u_1} (f : Lean.Elab.ContextInfoLean.Elab.Infoαα) (ctx? : Option Lean.Elab.ContextInfo) (a : α) :
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.

Find an info node, if any, which should be shown on hover/cursor at position hoverPos.

Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.

Construct a hover popup, if any, from an info node in a context.

Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.