Documentation

Lean.Data.JsonRpc

Implementation of JSON-RPC 2.0 (https://www.jsonrpc.org/specification) for use in the LSP server.

Equations
Equations
  • One or more equations did not get rendered due to their size.
inductive Lean.JsonRpc.ErrorCode:
Type

Error codes defined by JSON-RPC and LSP.

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.
structure Lean.JsonRpc.Request (α : Type u) :
Type u
instance Lean.JsonRpc.instInhabitedRequest:
{a : Type u_1} → [inst : Inhabited a] → Inhabited (Lean.JsonRpc.Request a)
Equations
  • Lean.JsonRpc.instInhabitedRequest = { default := { id := default, method := default, param := default } }
instance Lean.JsonRpc.instBEqRequest:
{α : Type u_1} → [inst : BEq α] → BEq (Lean.JsonRpc.Request α)
Equations
  • Lean.JsonRpc.instBEqRequest = { beq := [anonymous] }
Equations
structure Lean.JsonRpc.Notification (α : Type u) :
Type u
Equations
  • Lean.JsonRpc.instInhabitedNotification = { default := { method := default, param := default } }
instance Lean.JsonRpc.instBEqNotification:
{α : Type u_1} → [inst : BEq α] → BEq (Lean.JsonRpc.Notification α)
Equations
  • Lean.JsonRpc.instBEqNotification = { beq := [anonymous] }
Equations
structure Lean.JsonRpc.Response (α : Type u) :
Type u
instance Lean.JsonRpc.instInhabitedResponse:
{a : Type u_1} → [inst : Inhabited a] → Inhabited (Lean.JsonRpc.Response a)
Equations
  • Lean.JsonRpc.instInhabitedResponse = { default := { id := default, result := default } }
instance Lean.JsonRpc.instBEqResponse:
{α : Type u_1} → [inst : BEq α] → BEq (Lean.JsonRpc.Response α)
Equations
  • Lean.JsonRpc.instBEqResponse = { beq := [anonymous] }
Equations
structure Lean.JsonRpc.ResponseError (α : Type u) :
Type u
Equations
  • Lean.JsonRpc.instInhabitedResponseError = { default := { id := default, code := default, message := default, data? := default } }
instance Lean.JsonRpc.instBEqResponseError:
{α : Type u_1} → [inst : BEq α] → BEq (Lean.JsonRpc.ResponseError α)
Equations
  • Lean.JsonRpc.instBEqResponseError = { beq := [anonymous] }
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.
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.
def IO.FS.Stream.readRequestAs (h : IO.FS.Stream) (nBytes : Nat) (expectedMethod : String) (α : Type) [inst : Lean.FromJson α] :
Equations
  • One or more equations did not get rendered due to their size.
def IO.FS.Stream.readNotificationAs (h : IO.FS.Stream) (nBytes : Nat) (expectedMethod : String) (α : Type) [inst : Lean.FromJson α] :
Equations
  • One or more equations did not get rendered due to their size.
partial def IO.FS.Stream.readResponseAs (h : IO.FS.Stream) (nBytes : Nat) (expectedID : Lean.JsonRpc.RequestID) (α : Type) [inst : Lean.FromJson α] :