- timeout : ActionKind
- mousedown : ActionKind
- mouseup : ActionKind
- mousemove : ActionKind
Instances For
Equations
- ProofWidgets.Svg.instToJsonActionKind.toJson ProofWidgets.Svg.ActionKind.timeout = Lean.toJson "timeout"
- ProofWidgets.Svg.instToJsonActionKind.toJson ProofWidgets.Svg.ActionKind.mousedown = Lean.toJson "mousedown"
- ProofWidgets.Svg.instToJsonActionKind.toJson ProofWidgets.Svg.ActionKind.mouseup = Lean.toJson "mouseup"
- ProofWidgets.Svg.instToJsonActionKind.toJson ProofWidgets.Svg.ActionKind.mousemove = Lean.toJson "mousemove"
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- kind : ActionKind
Instances For
Equations
Equations
The input type State
is any state the user wants to use and update
SvgState in addition automatically handles tracking of time, selection and custom data
- state : State
- time : Float
time in milliseconds
Instances For
instance
ProofWidgets.Svg.instToJsonSvgState
{State✝ : Type}
[Lean.ToJson State✝]
:
Lean.ToJson (SvgState State✝)
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
instance
ProofWidgets.Svg.instFromJsonSvgState
{State✝ : Type}
[Lean.FromJson State✝]
:
Lean.FromJson (SvgState State✝)
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
instance
ProofWidgets.Svg.instRpcEncodableSvgState
{State : Type}
[Lean.Server.RpcEncodable State]
:
Lean.Server.RpcEncodable (SvgState State)
Equations
instance
ProofWidgets.Svg.instToJsonUpdateParams
{State✝ : Type}
[Lean.ToJson State✝]
:
Lean.ToJson (UpdateParams State✝)
Equations
def
ProofWidgets.Svg.instToJsonUpdateParams.toJson
{State✝ : Type}
[Lean.ToJson State✝]
:
UpdateParams State✝ → Lean.Json
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
ProofWidgets.Svg.instFromJsonUpdateParams.fromJson
{State✝ : Type}
[Lean.FromJson State✝]
:
Lean.Json → Except String (UpdateParams State✝)
Equations
- One or more equations did not get rendered due to their size.
Instances For
instance
ProofWidgets.Svg.instFromJsonUpdateParams
{State✝ : Type}
[Lean.FromJson State✝]
:
Lean.FromJson (UpdateParams State✝)
Equations
instance
ProofWidgets.Svg.instRpcEncodableUpdateResult
{State : Type}
[Lean.Server.RpcEncodable State]
:
Lean.Server.RpcEncodable (UpdateResult State)
Equations
- init : State
- frame : Frame
Instances For
def
ProofWidgets.Svg.InteractiveSvg.serverRpcMethod
{State : Type}
(isvg : InteractiveSvg State)
(params : UpdateParams State)
:
Equations
- One or more equations did not get rendered due to their size.