/- Copyright (c) 2021 Henrik Böving. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Henrik Böving -/ import DocGen4.ToHtmlFormat import DocGen4.Output.Navbar namespace DocGen4 namespace Output open scoped DocGen4.Jsx def baseHtmlArray (title : String) (site : Array Html) : HtmlM Html := do pure {title}

Documentation

{title}

-- TODO: Replace this form with our own search
[site] {←navbar} -- Lean in JS in HTML in Lean...very meta -- TODO Add more js stuff -- mathjax def baseHtml (title : String) (site : Html) : HtmlM Html := baseHtmlArray title #[site] end Output end DocGen4