- timeout : ActionKind
- mousedown : ActionKind
- mouseup : ActionKind
- mousemove : ActionKind
Instances For
Equations
Equations
- ProofWidgets.Svg.instFromJsonActionKind = { fromJson? := ProofWidgets.Svg.fromJsonActionKind✝ }
Equations
- ProofWidgets.Svg.instDecidableEqActionKind x✝ y✝ = if h : x✝.toCtorIdx = y✝.toCtorIdx then isTrue ⋯ else isFalse ⋯
- kind : ActionKind
Instances For
Equations
- ProofWidgets.Svg.instToJsonAction = { toJson := ProofWidgets.Svg.toJsonAction✝ }
Equations
- ProofWidgets.Svg.instFromJsonAction = { fromJson? := ProofWidgets.Svg.fromJsonAction✝ }
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
instance
ProofWidgets.Svg.instFromJsonSvgState
{State✝ : Type}
[Lean.FromJson State✝]
:
Lean.FromJson (SvgState State✝)
Equations
- ProofWidgets.Svg.instFromJsonSvgState = { fromJson? := ProofWidgets.Svg.fromJsonSvgState✝ }
instance
ProofWidgets.Svg.instRpcEncodableSvgState
{State : Type}
[Lean.Server.RpcEncodable State]
:
Lean.Server.RpcEncodable (SvgState State)
Equations
- ProofWidgets.Svg.instRpcEncodableSvgState = { rpcEncode := ProofWidgets.Svg.instRpcEncodableSvgState.enc✝, rpcDecode := ProofWidgets.Svg.instRpcEncodableSvgState.dec✝ }
instance
ProofWidgets.Svg.instToJsonUpdateParams
{State✝ : Type}
[Lean.ToJson State✝]
:
Lean.ToJson (UpdateParams State✝)
Equations
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.