Reading/writing LSP messages from/to IO handles.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
IO.FS.Stream.readLspRequestAs
(h : IO.FS.Stream)
(expectedMethod : String)
(α : Type)
[Lean.FromJson α]
:
Instances For
def
IO.FS.Stream.readLspNotificationAs
(h : IO.FS.Stream)
(expectedMethod : String)
(α : Type)
[Lean.FromJson α]
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
IO.FS.Stream.readLspResponseAs
(h : IO.FS.Stream)
(expectedID : Lean.JsonRpc.RequestID)
(α : Type)
[Lean.FromJson α]
:
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
def
IO.FS.Stream.writeLspRequest
{α : Type u_1}
[Lean.ToJson α]
(h : IO.FS.Stream)
(r : Lean.JsonRpc.Request α)
:
Equations
- h.writeLspRequest r = h.writeLspMessage (Lean.JsonRpc.Message.request r.id r.method (Lean.Json.toStructured? r.param).toOption)
Instances For
def
IO.FS.Stream.writeLspNotification
{α : Type u_1}
[Lean.ToJson α]
(h : IO.FS.Stream)
(n : Lean.JsonRpc.Notification α)
:
Instances For
def
IO.FS.Stream.writeLspResponse
{α : Type u_1}
[Lean.ToJson α]
(h : IO.FS.Stream)
(r : Lean.JsonRpc.Response α)
:
Instances For
Instances For
def
IO.FS.Stream.writeLspResponseErrorWithData
{α : Type u_1}
[Lean.ToJson α]
(h : IO.FS.Stream)
(e : Lean.JsonRpc.ResponseError α)
: