- paramsRange : String.Range
- diagRange : String.Range
Instances For
def
Lean.Server.FileWorker.waitUnknownIdentifierRanges
(doc : EditableDocument)
(requestedRange : String.Range)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
- fullName : Name
- edit : Lsp.TextEdit
Instances For
- env : Environment
Instances For
def
Lean.Server.FileWorker.collectOpenNamespaces
(currentNamespace : Name)
(openDecls : List OpenDecl)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.computeFallbackQuery?
(doc : EditableDocument)
(requestedRange unknownIdentifierRange : String.Range)
(infoTree : Elab.InfoTree)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.computeIdQuery?
(doc : EditableDocument)
(ctx : Elab.ContextInfo)
(stx : Syntax)
(id : Name)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.computeDotQuery?
(doc : EditableDocument)
(ctx : Elab.ContextInfo)
(ti : Elab.TermInfo)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.computeDotIdQuery?
(doc : EditableDocument)
(ctx : Elab.ContextInfo)
(stx : Syntax)
(id : Name)
(lctx : LocalContext)
(expectedType? : Option Expr)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.computeQuery?
(doc : EditableDocument)
(requestedRange unknownIdentifierRange : String.Range)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Server.FileWorker.importAllUnknownIdentifiersProvider = `unknownIdentifiers
Instances For
def
Lean.Server.FileWorker.importAllUnknownIdentifiersCodeAction
(params : Lsp.CodeActionParams)
(kind : String)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.handleUnknownIdentifierCodeAction
(id : JsonRpc.RequestID)
(params : Lsp.CodeActionParams)
(requestedRange : String.Range)
(unknownIdentifierRanges : Array String.Range)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.handleResolveImportAllUnknownIdentifiersCodeAction?
(id : JsonRpc.RequestID)
(action : Lsp.CodeAction)
(unknownIdentifierRanges : Array String.Range)
:
Equations
- One or more equations did not get rendered due to their size.