/- 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.Output.ToHtmlFormat import DocGen4.Output.Template namespace DocGen4 namespace Output open scoped DocGen4.Jsx def index : BaseHtmlM Html := do templateExtends (baseHtml "Index") <| pure <|

Welcome to the documentation page

-- Temporary comment until the lake issue is resolved -- for commit {s!"{← getProjectCommit} "}

This was built using Lean 4 at commit {Lean.githash}

end Output end DocGen4