Documentation

Lean.DeclarationRange

structure Lean.DeclarationRange:
Type
  • A precomputed UTF-16 character field as in Lean.Lsp.Position. We need to store this because LSP clients want us to report the range in terms of UTF-16, but converting a Unicode codepoint stored in Lean.Position to UTF-16 requires loading and mapping the target source file, which is IO-heavy.

    charUtf16 : Nat
  • endPos : Lean.Position
  • See charUtf16.

    endCharUtf16 : Nat
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.
def Lean.addDeclarationRanges {m : TypeType} [inst : Lean.MonadEnv m] (declName : Lean.Name) (declRanges : Lean.DeclarationRanges) :
Equations
def Lean.findDeclarationRangesCore? {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] (declName : Lean.Name) :
Equations
def Lean.findDeclarationRanges? {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : MonadLiftT IO m] (declName : Lean.Name) :
Equations
  • One or more equations did not get rendered due to their size.