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.
def
Lean.Server.FileWorker.locationLinksOfInfo
(kind : Lean.Server.GoToKind)
(ci : Lean.Elab.ContextInfo)
(i : Lean.Elab.Info)
(infoTree? : optParam (Option Lean.Elab.InfoTree) none)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Server.FileWorker.handleDefinition
(kind : Lean.Server.GoToKind)
(p : Lean.Lsp.TextDocumentPositionParams)
:
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.
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.
partial def
Lean.Server.FileWorker.handleDocumentHighlight.highlightReturn?
(text : Lean.FileMap)
(pos : String.Pos)
(doRange? : Option Lean.Lsp.Range)
:
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.Server.FileWorker.handleDocumentSymbol.sectionLikeToDocumentSymbols
(text : Lean.FileMap)
(stx : Lean.Syntax)
(stxs : List Lean.Syntax)
(name : String)
(kind : Lean.Lsp.SymbolKind)
(selection : Lean.Syntax)
:
Equations
- Lean.Server.FileWorker.noHighlightKinds = #[`Lean.Parser.Term.sorry, `Lean.Parser.Term.type, `Lean.Parser.Term.prop, `antiquotName, `Lean.Parser.Command.docComment]
- beginPos : String.Pos
- endPos : String.Pos
- text : Lean.FileMap
- lastLspPos : Lean.Lsp.Position
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.
def
Lean.Server.FileWorker.handleSemanticTokens.addToken
(stx : Lean.Syntax)
(type : Lean.Lsp.SemanticTokenType)
:
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.
Equations
- Lean.Server.FileWorker.handleFoldingRange.isImport stx = (Lean.Syntax.isOfKind stx `Lean.Parser.Module.header || Lean.Syntax.isOfKind stx `Lean.Parser.Command.open)
partial def
Lean.Server.FileWorker.handleFoldingRange.addRanges
(text : Lean.FileMap)
(sections : List (Option String.Pos))
:
def
Lean.Server.FileWorker.handleFoldingRange.addCommandRange
(text : Lean.FileMap)
(stx : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Server.FileWorker.handleFoldingRange.addRangeFromSyntax
(text : Lean.FileMap)
(kind : Lean.Lsp.FoldingRangeKind)
(stx : Lean.Syntax)
:
Equations
- Lean.Server.FileWorker.handleFoldingRange.addRangeFromSyntax text kind stx = Lean.Server.FileWorker.handleFoldingRange.addRange text kind (Lean.Syntax.getPos? stx) (Lean.Syntax.getTailPos? stx)
def
Lean.Server.FileWorker.handleFoldingRange.addRange
(text : Lean.FileMap)
(kind : Lean.Lsp.FoldingRangeKind)
(start? : Option String.Pos)
(stop? : Option String.Pos)
:
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.