Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- text : CompletionItemKind
- method : CompletionItemKind
- function : CompletionItemKind
- constructor : CompletionItemKind
- field : CompletionItemKind
- variable : CompletionItemKind
- class : CompletionItemKind
- interface : CompletionItemKind
- module : CompletionItemKind
- property : CompletionItemKind
- unit : CompletionItemKind
- value : CompletionItemKind
- enum : CompletionItemKind
- keyword : CompletionItemKind
- snippet : CompletionItemKind
- color : CompletionItemKind
- file : CompletionItemKind
- reference : CompletionItemKind
- folder : CompletionItemKind
- enumMember : CompletionItemKind
- constant : CompletionItemKind
- struct : CompletionItemKind
- event : CompletionItemKind
- operator : CompletionItemKind
- typeParameter : CompletionItemKind
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.text = 0
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.method = 1
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.function = 2
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.constructor = 3
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.field = 4
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.variable = 5
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.class = 6
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.interface = 7
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.module = 8
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.property = 9
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.unit = 10
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.value = 11
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.enum = 12
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.keyword = 13
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.snippet = 14
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.color = 15
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.file = 16
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.reference = 17
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.folder = 18
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.enumMember = 19
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.constant = 20
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.struct = 21
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.event = 22
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.operator = 23
- Lean.Lsp.instHashableCompletionItemKind.hash Lean.Lsp.CompletionItemKind.typeParameter = 24
Instances For
Equations
- Lean.Lsp.instToJsonCompletionItemKind = { toJson := fun (a : Lean.Lsp.CompletionItemKind) => Lean.toJson (a.ctorIdx + 1) }
Equations
- Lean.Lsp.instFromJsonCompletionItemKind = { fromJson? := fun (v : Lean.Json) => do let i ← Lean.fromJson? v pure (Lean.Lsp.CompletionItemKind.ofNat (i - 1)) }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Lsp.instToJsonCompletionItemTag = { toJson := fun (t : Lean.Lsp.CompletionItemTag) => Lean.toJson (t.ctorIdx + 1) }
Equations
- Lean.Lsp.instFromJsonCompletionItemTag = { fromJson? := fun (v : Lean.Json) => do let i ← Lean.fromJson? v pure (Lean.Lsp.CompletionItemTag.ofNat (i - 1)) }
- label : String
- documentation? : Option MarkupContent
- kind? : Option CompletionItemKind
- textEdit? : Option InsertReplaceEdit
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Lsp.instBEqCompletionItem.beq x✝¹ x✝ = false
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
- isIncomplete : Bool
- items : Array CompletionItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Lsp.instToJsonCompletionList.toJson x✝ = Lean.Json.mkObj [[("isIncomplete", Lean.toJson x✝.isIncomplete)], [("items", Lean.toJson x✝.items)]].flatten
Instances For
Equations
Identifier that is sent from the server to the client as part of the CompletionItem.data?
field.
Needed to resolve the CompletionItem
when the client sends a completionItem/resolve
request
for that item, again containing the data?
field provided by the server.
- const (declName : Name) : CompletionIdentifier
- fvar (id : FVarId) : CompletionIdentifier
Instances For
Equations
- Lean.Lsp.instBEqCompletionIdentifier.beq (Lean.Lsp.CompletionIdentifier.const a) (Lean.Lsp.CompletionIdentifier.const b) = (a == b)
- Lean.Lsp.instBEqCompletionIdentifier.beq (Lean.Lsp.CompletionIdentifier.fvar a) (Lean.Lsp.CompletionIdentifier.fvar b) = (a == b)
- Lean.Lsp.instBEqCompletionIdentifier.beq x✝¹ x✝ = false
Instances For
Equations
Instances For
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.
- mod : Name
- pos : Position
Position of the completion info that this completion item was created from.
- id? : Option CompletionIdentifier
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Lsp.instBEqResolvableCompletionItemData.beq x✝¹ x✝ = false
Instances For
Equations
Instances For
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.
- label : String
- documentation? : Option MarkupContent
- kind? : Option CompletionItemKind
- textEdit? : Option InsertReplaceEdit
- data? : Option ResolvableCompletionItemData
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Lsp.instBEqResolvableCompletionItem.beq x✝¹ x✝ = false
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- isIncomplete : Bool
- items : Array ResolvableCompletionItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonResolvableCompletionList.toJson x✝ = Lean.Json.mkObj [[("isIncomplete", Lean.toJson x✝.isIncomplete)], [("items", Lean.toJson x✝.items)]].flatten
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonCompletionParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
Equations
- Lean.Lsp.instToJsonHover.toJson x✝ = Lean.Json.mkObj [[("contents", Lean.toJson x✝.contents)], Lean.Json.opt "range" x✝.range?].flatten
Instances For
Equations
Equations
- Lean.Lsp.instFromJsonHover = { fromJson? := Lean.Lsp.instFromJsonHover.fromJson }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Lsp.instToJsonHoverParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonDeclarationParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonDefinitionParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonTypeDefinitionParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonReferenceContext.toJson x✝ = Lean.Json.mkObj [[("includeDeclaration", Lean.toJson x✝.includeDeclaration)]].flatten
Instances For
- context : ReferenceContext
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonDocumentHighlightParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
- text : DocumentHighlightKind
- read : DocumentHighlightKind
- write : DocumentHighlightKind
Instances For
Equations
- One or more equations did not get rendered due to their size.
- range : Range
- kind? : Option DocumentHighlightKind
Instances For
Equations
- Lean.Lsp.instToJsonDocumentHighlight.toJson x✝ = Lean.Json.mkObj [[("range", Lean.toJson x✝.range)], Lean.Json.opt "kind" x✝.kind?].flatten
Instances For
@[reducible, inline]
Instances For
- textDocument : TextDocumentIdentifier
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonDocumentSymbolParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)]].flatten
Instances For
- file : SymbolKind
- module : SymbolKind
- namespace : SymbolKind
- package : SymbolKind
- class : SymbolKind
- method : SymbolKind
- property : SymbolKind
- field : SymbolKind
- constructor : SymbolKind
- enum : SymbolKind
- interface : SymbolKind
- function : SymbolKind
- variable : SymbolKind
- constant : SymbolKind
- string : SymbolKind
- number : SymbolKind
- boolean : SymbolKind
- array : SymbolKind
- object : SymbolKind
- key : SymbolKind
- null : SymbolKind
- enumMember : SymbolKind
- struct : SymbolKind
- event : SymbolKind
- operator : SymbolKind
- typeParameter : SymbolKind
Instances For
Equations
Equations
- Lean.Lsp.instBEqSymbolKind.beq x✝ y✝ = (x✝.ctorIdx == y✝.ctorIdx)
Instances For
Equations
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.file = 0
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.module = 1
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.namespace = 2
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.package = 3
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.class = 4
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.method = 5
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.property = 6
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.field = 7
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.constructor = 8
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.enum = 9
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.interface = 10
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.function = 11
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.variable = 12
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.constant = 13
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.string = 14
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.number = 15
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.boolean = 16
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.array = 17
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.object = 18
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.key = 19
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.null = 20
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.enumMember = 21
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.struct = 22
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.event = 23
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.operator = 24
- Lean.Lsp.instHashableSymbolKind.hash Lean.Lsp.SymbolKind.typeParameter = 25
Instances For
Equations
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.
instance
Lean.Lsp.instFromJsonDocumentSymbolAux
{Self✝ : Type}
[FromJson Self✝]
:
FromJson (DocumentSymbolAux Self✝)
Equations
def
Lean.Lsp.instFromJsonDocumentSymbolAux.fromJson
{Self✝ : Type}
[FromJson Self✝]
:
Json → Except String (DocumentSymbolAux Self✝)
Equations
- One or more equations did not get rendered due to their size.
Instances For
instance
Lean.Lsp.instToJsonDocumentSymbolAux
{Self✝ : Type}
[ToJson Self✝]
:
ToJson (DocumentSymbolAux Self✝)
Equations
def
Lean.Lsp.instToJsonDocumentSymbolAux.toJson
{Self✝ : Type}
[ToJson Self✝]
:
DocumentSymbolAux Self✝ → Json
Equations
- One or more equations did not get rendered due to their size.
Instances For
- mk (sym : DocumentSymbolAux DocumentSymbol) : DocumentSymbol
Instances For
Equations
Equations
- Lean.Lsp.instToJsonDocumentSymbolResult = { toJson := fun (dsr : Lean.Lsp.DocumentSymbolResult) => Lean.toJson dsr.syms }
Equations
Equations
- Lean.Lsp.instBEqSymbolTag.beq x✝ y✝ = (x✝.ctorIdx == y✝.ctorIdx)
Instances For
Equations
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Lsp.instToJsonSymbolTag = { toJson := fun (x : Lean.Lsp.SymbolTag) => match x with | Lean.Lsp.SymbolTag.deprecated => 1 }
- name : String
- kind : SymbolKind
- location : Location
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonCallHierarchyPrepareParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
- name : String
- kind : SymbolKind
- uri : DocumentUri
- range : Range
- selectionRange : Range
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Lsp.instBEqCallHierarchyItem.beq x✝¹ x✝ = false
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- item : CallHierarchyItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- from : CallHierarchyItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonCallHierarchyIncomingCall.toJson x✝ = Lean.Json.mkObj [[("from", Lean.toJson x✝.from)], [("fromRanges", Lean.toJson x✝.fromRanges)]].flatten
Instances For
Equations
Instances For
- item : CallHierarchyItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- to : CallHierarchyItem
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonCallHierarchyOutgoingCall.toJson x✝ = Lean.Json.mkObj [[("to", Lean.toJson x✝.to)], [("fromRanges", Lean.toJson x✝.fromRanges)]].flatten
Instances For
Equations
Instances For
- keyword : SemanticTokenType
- variable : SemanticTokenType
- property : SemanticTokenType
- function : SemanticTokenType
- namespace : SemanticTokenType
- type : SemanticTokenType
- class : SemanticTokenType
- enum : SemanticTokenType
- interface : SemanticTokenType
- struct : SemanticTokenType
- typeParameter : SemanticTokenType
- parameter : SemanticTokenType
- enumMember : SemanticTokenType
- event : SemanticTokenType
- method : SemanticTokenType
- macro : SemanticTokenType
- modifier : SemanticTokenType
- comment : SemanticTokenType
- string : SemanticTokenType
- number : SemanticTokenType
- regexp : SemanticTokenType
- operator : SemanticTokenType
- decorator : SemanticTokenType
- leanSorryLike : SemanticTokenType
Instances For
Equations
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.keyword = Lean.toJson "keyword"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.variable = Lean.toJson "variable"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.property = Lean.toJson "property"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.function = Lean.toJson "function"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.namespace = Lean.toJson "namespace"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.type = Lean.toJson "type"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.class = Lean.toJson "class"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.enum = Lean.toJson "enum"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.interface = Lean.toJson "interface"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.struct = Lean.toJson "struct"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.typeParameter = Lean.toJson "typeParameter"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.parameter = Lean.toJson "parameter"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.enumMember = Lean.toJson "enumMember"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.event = Lean.toJson "event"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.method = Lean.toJson "method"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.macro = Lean.toJson "macro"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.modifier = Lean.toJson "modifier"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.comment = Lean.toJson "comment"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.string = Lean.toJson "string"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.number = Lean.toJson "number"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.regexp = Lean.toJson "regexp"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.operator = Lean.toJson "operator"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.decorator = Lean.toJson "decorator"
- Lean.Lsp.instToJsonSemanticTokenType.toJson Lean.Lsp.SemanticTokenType.leanSorryLike = Lean.toJson "leanSorryLike"
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instBEqSemanticTokenType.beq x✝ y✝ = (x✝.ctorIdx == y✝.ctorIdx)
Instances For
Equations
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.keyword = 0
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.variable = 1
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.property = 2
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.function = 3
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.namespace = 4
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.type = 5
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.class = 6
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.enum = 7
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.interface = 8
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.struct = 9
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.typeParameter = 10
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.parameter = 11
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.enumMember = 12
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.event = 13
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.method = 14
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.macro = 15
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.modifier = 16
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.comment = 17
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.string = 18
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.number = 19
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.regexp = 20
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.operator = 21
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.decorator = 22
- Lean.Lsp.instHashableSemanticTokenType.hash Lean.Lsp.SemanticTokenType.leanSorryLike = 23
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
The semantic token modifiers included by default in the LSP specification. Not used by the Lean core, but implementing them here allows them to be utilized by users extending the Lean server.
- declaration : SemanticTokenModifier
- definition : SemanticTokenModifier
- readonly : SemanticTokenModifier
- static : SemanticTokenModifier
- deprecated : SemanticTokenModifier
- abstract : SemanticTokenModifier
- async : SemanticTokenModifier
- modification : SemanticTokenModifier
- documentation : SemanticTokenModifier
- defaultLibrary : SemanticTokenModifier
Instances For
Equations
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.declaration = Lean.toJson "declaration"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.definition = Lean.toJson "definition"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.readonly = Lean.toJson "readonly"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.static = Lean.toJson "static"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.deprecated = Lean.toJson "deprecated"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.abstract = Lean.toJson "abstract"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.async = Lean.toJson "async"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.modification = Lean.toJson "modification"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.documentation = Lean.toJson "documentation"
- Lean.Lsp.instToJsonSemanticTokenModifier.toJson Lean.Lsp.SemanticTokenModifier.defaultLibrary = Lean.toJson "defaultLibrary"
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonSemanticTokensLegend.toJson x✝ = Lean.Json.mkObj [[("tokenTypes", Lean.toJson x✝.tokenTypes)], [("tokenModifiers", Lean.toJson x✝.tokenModifiers)]].flatten
Instances For
- legend : SemanticTokensLegend
- range : Bool
- full : Bool
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
- textDocument : TextDocumentIdentifier
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonSemanticTokensParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)]].flatten
Instances For
- textDocument : TextDocumentIdentifier
- range : Range
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonSemanticTokensRangeParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("range", Lean.toJson x✝.range)]].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
Equations
- Lean.Lsp.instToJsonSemanticTokens.toJson x✝ = Lean.Json.mkObj [Lean.Json.opt "resultId" x✝.resultId?, [("data", Lean.toJson x✝.data)]].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonFoldingRangeParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)]].flatten
Instances For
- comment : FoldingRangeKind
- imports : FoldingRangeKind
- region : FoldingRangeKind
Instances For
Equations
- One or more equations did not get rendered due to their size.
- startLine : Nat
- endLine : Nat
- kind? : Option FoldingRangeKind
Instances For
Equations
- Lean.Lsp.instToJsonFoldingRange.toJson x✝ = Lean.Json.mkObj [[("startLine", Lean.toJson x✝.startLine)], [("endLine", Lean.toJson x✝.endLine)], Lean.Json.opt "kind" x✝.kind?].flatten
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
Equations
- Lean.Lsp.instToJsonRenameOptions.toJson x✝ = Lean.Json.mkObj [[("prepareProvider", Lean.toJson x✝.prepareProvider)]].flatten
Instances For
- newName : String
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonPrepareRenameParams.toJson x✝ = Lean.Json.mkObj [[("textDocument", Lean.toJson x✝.textDocument)], [("position", Lean.toJson x✝.position)]].flatten
Instances For
- textDocument : TextDocumentIdentifier
- range : Range
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- plaintext (text : String) : InlayHintTooltip
- markdown (markup : MarkupContent) : InlayHintTooltip
Instances For
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.
- value : String
- tooltip? : Option InlayHintTooltip
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- name (n : String) : InlayHintLabel
- parts (p : Array InlayHintLabelPart) : InlayHintLabel
Instances For
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.
- type : InlayHintKind
- parameter : InlayHintKind
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Lsp.instToJsonInlayHintKind = { toJson := fun (x : Lean.Lsp.InlayHintKind) => match x with | Lean.Lsp.InlayHintKind.type => 1 | Lean.Lsp.InlayHintKind.parameter => 2 }
- position : Position
- label : InlayHintLabel
- kind? : Option InlayHintKind
- tooltip? : Option InlayHintTooltip
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- resolveSupport? : Option ResolveSupport
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonInlayHintOptions.toJson x✝ = Lean.Json.mkObj [[("workDoneProgress", Lean.toJson x✝.workDoneProgress)], Lean.Json.opt "resolveProvider" x✝.resolveProvider?].flatten
Instances For
- name (name : String) : ParameterInformationLabel
- range (startUtf16Offset endUtf16Offset : Nat) : ParameterInformationLabel
Instances For
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.
- label : ParameterInformationLabel
- documentation? : Option MarkupContent
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Lsp.instToJsonParameterInformation.toJson x✝ = Lean.Json.mkObj [[("label", Lean.toJson x✝.label)], Lean.Json.opt "documentation" x✝.documentation?].flatten
Instances For
- label : String
- documentation? : Option MarkupContent
- parameters? : Option (Array ParameterInformation)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- signatures : Array SignatureInformation
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- invoked : SignatureHelpTriggerKind
- triggerCharacter : SignatureHelpTriggerKind
- contentChange : SignatureHelpTriggerKind
Instances For
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.
- triggerKind : SignatureHelpTriggerKind
- isRetrigger : Bool
- activeSignatureHelp? : Option SignatureHelp
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
structure
Lean.Lsp.SignatureHelpParamsextends Lean.Lsp.TextDocumentPositionParams, Lean.Lsp.WorkDoneProgressParams :
- context? : Option SignatureHelpContext
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.