- timeout : ProofWidgets.Svg.ActionKind
- mousedown : ProofWidgets.Svg.ActionKind
- mouseup : ProofWidgets.Svg.ActionKind
- mousemove : ProofWidgets.Svg.ActionKind
Instances For
Equations
- ProofWidgets.Svg.instDecidableEqActionKind x✝ y✝ = if h : x✝.toCtorIdx = y✝.toCtorIdx then isTrue ⋯ else isFalse ⋯
- kind : ProofWidgets.Svg.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 (ProofWidgets.Svg.SvgState State✝)
Equations
- ProofWidgets.Svg.instToJsonSvgState = { toJson := ProofWidgets.Svg.toJsonSvgState✝ }
instance
ProofWidgets.Svg.instFromJsonSvgState
{State✝ : Type}
[Lean.FromJson State✝]
:
Lean.FromJson (ProofWidgets.Svg.SvgState State✝)
Equations
- ProofWidgets.Svg.instFromJsonSvgState = { fromJson? := ProofWidgets.Svg.fromJsonSvgState✝ }
instance
ProofWidgets.Svg.instRpcEncodableSvgState
{State : Type}
[Lean.Server.RpcEncodable State]
:
Equations
- ProofWidgets.Svg.instRpcEncodableSvgState = { rpcEncode := ProofWidgets.Svg.instRpcEncodableSvgState.enc✝, rpcDecode := ProofWidgets.Svg.instRpcEncodableSvgState.dec✝ }
- elapsed : Float
- actions : Array ProofWidgets.Svg.Action
- state : ProofWidgets.Svg.SvgState State
Instances For
instance
ProofWidgets.Svg.instToJsonUpdateParams
{State✝ : Type}
[Lean.ToJson State✝]
:
Lean.ToJson (ProofWidgets.Svg.UpdateParams State✝)
Equations
- ProofWidgets.Svg.instToJsonUpdateParams = { toJson := ProofWidgets.Svg.toJsonUpdateParams✝ }
Equations
- ProofWidgets.Svg.instFromJsonUpdateParams = { fromJson? := ProofWidgets.Svg.fromJsonUpdateParams✝ }
- html : ProofWidgets.Html
- state : ProofWidgets.Svg.SvgState State
Approximate number of milliseconds to wait before calling again.
Instances For
instance
ProofWidgets.Svg.instRpcEncodableUpdateResult
{State : Type}
[Lean.Server.RpcEncodable State]
:
Equations
- ProofWidgets.Svg.instRpcEncodableUpdateResult = { rpcEncode := ProofWidgets.Svg.instRpcEncodableUpdateResult.enc✝, rpcDecode := ProofWidgets.Svg.instRpcEncodableUpdateResult.dec✝ }
- init : State
- frame : ProofWidgets.Svg.Frame
- update (time_ms Δt_ms : Float) (action : ProofWidgets.Svg.Action) (mouseStart mouseEnd : Option (ProofWidgets.Svg.Point self.frame)) (selectedId : Option String) (getSelectedData : (α : Type) → [inst : Lean.FromJson α] → Option α) : State → State
- render (time_ms : Float) (mouseStart mouseEnd : Option (ProofWidgets.Svg.Point self.frame)) : State → ProofWidgets.Svg self.frame
Instances For
def
ProofWidgets.Svg.InteractiveSvg.serverRpcMethod
{State : Type}
(isvg : ProofWidgets.Svg.InteractiveSvg State)
(params : ProofWidgets.Svg.UpdateParams State)
:
Equations
- One or more equations did not get rendered due to their size.