Documentation

ProofWidgets.Data.Svg

Instances For
    Equations
    • frame.ySize = frame.height.toFloat * (frame.xSize / frame.width.toFloat)
    Instances For
      Equations
      • frame.xmax = frame.xmin + frame.xSize
      Instances For
        Equations
        • frame.ymax = frame.ymin + frame.ySize
        Instances For
          Equations
          • frame.pixelSize = frame.xSize / frame.width.toFloat
          Instances For
            Instances For
              Equations

              Returns string "rgb(r, g, b)" with r,g,b ∈ [0,...,256)

              Equations
              Instances For
                Instances For
                  Equations
                  Equations
                  Instances For
                    Equations
                    Instances For
                      Instances For
                        Equations
                        Instances For
                          Instances For
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              Instances For
                                def ProofWidgets.Svg.Element.setStroke {f : Frame} (elem : Element f) (color : Color) (width : Size f) :
                                Equations
                                • elem.setStroke color width = { shape := elem.shape, strokeColor := some color, strokeWidth := some width, fillColor := elem.fillColor, id := elem.id, data := elem.data }
                                Instances For
                                  def ProofWidgets.Svg.Element.setFill {f : Frame} (elem : Element f) (color : Color) :
                                  Equations
                                  • elem.setFill color = { shape := elem.shape, strokeColor := elem.strokeColor, strokeWidth := elem.strokeWidth, fillColor := some color, id := elem.id, data := elem.data }
                                  Instances For
                                    Equations
                                    • elem.setId id = { shape := elem.shape, strokeColor := elem.strokeColor, strokeWidth := elem.strokeWidth, fillColor := elem.fillColor, id := some id, data := elem.data }
                                    Instances For
                                      def ProofWidgets.Svg.Element.setData {α : Type} {f : Frame} (elem : Element f) (a : α) [Lean.ToJson α] :
                                      Equations
                                      • elem.setData a = { shape := elem.shape, strokeColor := elem.strokeColor, strokeWidth := elem.strokeWidth, fillColor := elem.fillColor, id := elem.id, data := some (Lean.toJson a) }
                                      Instances For
                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For
                                          def ProofWidgets.Svg.line {f : Frame} (p q : Point f) :
                                          Equations
                                          Instances For
                                            def ProofWidgets.Svg.circle {f : Frame} (c : Point f) (r : Size f) :
                                            Equations
                                            Instances For
                                              Equations
                                              Instances For
                                                Equations
                                                Instances For
                                                  def ProofWidgets.mkIdToIdx {f : Svg.Frame} (elements : Array (Svg.Element f)) :
                                                  Std.HashMap String (Fin elements.size)
                                                  Equations
                                                  • One or more equations did not get rendered due to their size.
                                                  Instances For
                                                    Instances For
                                                      def ProofWidgets.Svg.toHtml {f : Frame} (svg : Svg f) :
                                                      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
                                                          Equations
                                                          Instances For
                                                            instance ProofWidgets.Svg.instGetElemNatElementLtSizeElements {f : Frame} :
                                                            GetElem (Svg f) Nat (Element f) fun (svg : Svg f) (idx : Nat) => idx < svg.elements.size
                                                            Equations
                                                            Equations
                                                            • One or more equations did not get rendered due to their size.
                                                            Equations
                                                            • svg.getData id = match svg[id] with | none => none | some elem => elem.data
                                                            Instances For