Functionality to do with initializing and shutting down the server ("General Messages" section of LSP spec).
Equations
Equations
- Lean.Lsp.instToJsonClientInfo.toJson x✝ = Lean.Json.mkObj [[("name", Lean.toJson x✝.name)], Lean.Json.opt "version" x✝.version?].flatten
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.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Lsp.instToJsonHashSet
{α : Type u_1}
[BEq α]
[Hashable α]
[ToJson α]
:
ToJson (Std.HashSet α)
Equations
- Lean.Lsp.instToJsonHashSet = { toJson := fun (s : Std.HashSet α) => Lean.Json.arr (Array.map Lean.toJson s.toArray) }
Instances For
def
Lean.Lsp.instFromJsonHashSet
{α : Type u_1}
[BEq α]
[Hashable α]
[FromJson α]
:
FromJson (Std.HashSet α)
Equations
- One or more equations did not get rendered due to their size.
Instances For
- logDir? : Option System.FilePath
- allowedMethods? : Option (Std.HashSet String)
- disallowedMethods? : Option (Std.HashSet String)
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Lean-specific initialization options.
Whether the client supports interactive widgets. When true, in order to improve performance the server may cease including information which can be retrieved interactively in some standard LSP messages. Defaults to false.
Instances For
Equations
- Lean.Lsp.instToJsonInitializationOptions.toJson x✝ = Lean.Json.mkObj [Lean.Json.opt "hasWidgets" x✝.hasWidgets?, Lean.Json.opt "logCfg" x✝.logCfg?].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- clientInfo? : Option ClientInfo
Not used by the language server. We use the cwd of the server process instead.
- initializationOptions? : Option InitializationOptions
- capabilities : ClientCapabilities
- trace : Trace
If omitted, we default to off.
- workspaceFolders? : Option (Array WorkspaceFolder)
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.
Equations
- Lean.Lsp.instFromJsonInitializedParams = { fromJson? := fun (x : Lean.Json) => pure Lean.Lsp.InitializedParams.mk }
Equations
- Lean.Lsp.instToJsonInitializedParams = { toJson := fun (x : Lean.Lsp.InitializedParams) => Lean.Json.null }
Equations
- Lean.Lsp.instToJsonServerInfo.toJson x✝ = Lean.Json.mkObj [[("name", Lean.toJson x✝.name)], Lean.Json.opt "version" x✝.version?].flatten
Instances For
Equations
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
- capabilities : ServerCapabilities
- serverInfo? : Option ServerInfo
Instances For
Equations
- Lean.Lsp.instToJsonInitializeResult.toJson x✝ = Lean.Json.mkObj [[("capabilities", Lean.toJson x✝.capabilities)], Lean.Json.opt "serverInfo" x✝.serverInfo?].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.