import DocGen4.Output.Template import DocGen4.Output.DocString import DocGen4.Process namespace DocGen4 namespace Output open scoped DocGen4.Jsx open Lean Widget /-- This is basically an arbitrary number that seems to work okay. -/ def equationLimit : Nat := 200 def equationToHtml (c : CodeWithInfos) : HtmlM Html := do return
  • [← infoFormatToHtml c]
  • /-- Attempt to render all `simp` equations for this definition. At a size defined in `equationLimit` we stop trying since they: - are too ugly to read most of the time - take too long -/ def equationsToHtml (i : Process.DefinitionInfo) : HtmlM (Array Html) := do if let some eqs := i.equations then let equationsHtml ← eqs.mapM equationToHtml let filteredEquationsHtml := equationsHtml.filter (·.textLength < equationLimit) if equationsHtml.size ≠ filteredEquationsHtml.size then return #[
    Equations
    ] else return #[
    Equations
    ] else return #[] end Output end DocGen4