import DocGen4.Output.Template import DocGen4.Output.DocString import DocGen4.Process namespace DocGen4 namespace Output open scoped DocGen4.Jsx open Lean def instancesForToHtml (typeName : Name) : BaseHtmlM Html := do pure
Instances For
def ctorToHtml (c : Process.NameInfo) : HtmlM Html := do let shortName := c.name.componentsRev.head!.toString let name := c.name.toString if let some doc := c.doc then let renderedDoc ← docStringToHtml doc pure
  • {shortName} : [← infoFormatToHtml c.type]
    [renderedDoc]
  • else pure
  • {shortName} : [← infoFormatToHtml c.type]
  • def inductiveToHtml (i : Process.InductiveInfo) : HtmlM (Array Html) := do let constructorsHtml := return #[constructorsHtml] end Output end DocGen4