/- 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 <|

Bookshelf

A study of the books listed below. Most proofs are conducted in LaTeX. Where feasible, theorems are also formally proven in Lean.

In Progress

Complete

Pending

Legend

A color/symbol code is used on generated PDF headers to indicate their status:

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

end Output end DocGen4