/- Modified from: https://github.com/leanprover/doc-gen4/blob/main/DocGen4/Output/Template.lean 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 Modifications include: Style changes. Test these changes with: - cp ./scripts/Template.lean .lake/packages/doc-gen4/DocGen4/Output/Template.lean - lake -Kenv=dev build Batteries:docs; rm -rf ./docs/docs; mv .lake/build/doc docs/docs - cd ./docs - bundle exec jekyll serve -/ import DocGen4.Output.ToHtmlFormat import DocGen4.Output.Navbar namespace DocGen4 namespace Output open scoped DocGen4.Jsx /-- The HTML template used for all pages. -/ def baseHtmlGenerator (title : String) (site : Array Html) : BaseHtmlM Html := do let moduleConstant := if let some module := ← getCurrentName then #[] else #[] pure
[← baseHtmlHeadDeclarations]