CoCalc Logo Icon
StoreFeaturesDocsShareSupportNewsAboutSign UpSign In

Real-time collaboration for Jupyter Notebooks, Linux Terminals, LaTeX, VS Code, R IDE, and more,
all in one place.

| Download

Try doing some basic maths questions in the Lean Theorem Prover. Functions, real numbers, equivalence relations and groups. Click on README.md and then on "Open in CoCalc with one click".

Project: Xena
Views: 18536
License: APACHE

Documentation style

We are in the process of implementing new documentation requirements for mathlib. All future pull requests must meet the following standards.

Header comment

Each mathlib file should start with:

  • a header comment with copyright information;

  • the list of imports;

  • a module docstring containing general documentation, written using Markdown.

(See the example below.)

Headers use atx-style headers (with hash signs, no underlying dash). The open and close delimiters /-! and -/ should appear on their own lines.

The mandatory title of the file is a first level header. It is followed by a summary of the content of the file.

The other sections, with second level headers are (in this order):

  • Main definitions (optional, can be covered in the summary)

  • Main statements (optional, can be covered in the summary)

  • Notations (omitted only if no notation is introduced in this file)

  • Implementation notes (description of important design decisions or interface features, including use of type classes and simp canonical form for new definitions)

  • References (references to textbooks or papers, or Wikipedia pages)

  • Tags (a list of keywords that could be useful when doing text search in mathlib to find where something is covered)

References should refer to bibtex entries in the mathlib citations file.

The following code block is an example of a file header.

/- Copyright (c) 2018 Robert Y. Lewis. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Robert Y. Lewis -/ import data.rat algebra.gcd_domain algebra.field_power import ring_theory.multiplicity tactic.ring import data.real.cau_seq import tactic.norm_cast /-! # p-adic norm This file defines the p-adic valuation and the p-adic norm on . The p-adic valuation on is the difference of the multiplicities of `p` in the numerator and denominator of `q`. This function obeys the standard properties of a valuation, with the appropriate assumptions on p. The valuation induces a norm on . This norm is a nonarchimedean absolute value. It takes values in {0} {1/p^k | k }. ## Notations This file uses the local notation `/.` for `rat.mk`. ## Implementation notes Much, but not all, of this file assumes that `p` is prime. This assumption is inferred automatically by taking (prime p) as a type class argument. ## References * [F. Q. Gouêva, *p-adic numbers*][gouvea1997] * https://en.wikipedia.org/wiki/P-adic_number ## Tags p-adic, p adic, padic, norm, valuation -/

Docstrings

Every definition and major theorem is required to have a doc string. (Doc strings on lemmas are also encouraged, particularly if the lemma has any mathematical content or might be useful in another file.) These are introduced using /-- and closed by -/ above the definition. They can contain some markdown, e.g. backtick quotes. They should convey the mathematical meaning of the definition. It is allowed to lie slightly about the actual implementation. The following is a docstring example:

/-- If `q ≠ 0`, the p-adic norm of a rational `q` is `p ^ (-(padic_val_rat p q))`. If `q = 0`, the p-adic norm of `q` is 0. -/ def padic_norm (p : ) (q : ) : := if q = 0 then 0 else (p : ) ^ (-(padic_val_rat p q))

An example that is slightly lying but still describes the mathematical content would be:

/-- For `p ≠ 1`, the p-adic valuation of an integer `z ≠ 0` is the largest natural number `n` such that p^n divides z. `padic_val_rat` defines the valuation of a rational `q` to be the valuation of `q.num` minus the valuation of `q.denom`. If `q = 0` or `p = 1`, then `padic_val_rat p q` defaults to 0. -/ def padic_val_rat (p : ) (q : ) : := if h : q 0 p 1 then (multiplicity (p : ) q.num).get (multiplicity.finite_int_iff.2 h.2, rat.num_ne_zero_of_ne_zero h.1) - (multiplicity (p : ) q.denom).get (multiplicity.finite_int_iff.2 h.2, by exact_mod_cast rat.denom_ne_zero _) else 0

The #doc_blame command can be run at the bottom of a file to list all definitions that do not have doc strings. #doc_blame! will also list theorems and lemmas.

Sectioning comments

It is common to structure a file in sections, where each section contains related declarations. By describing the sections with module documentation /-! ... -/ at the beginning, these sections can be seen in the documentation.

While these sectioning comments will often correspond to section or namespace commands, this is not required. You can use sectioning comments inside of a section or namespace, and you can have multiple sections or namespaces following one sectioning comment.

Sectioning comments are for display and readability only. They have no semantic meaning.

Third-level headers ### should be used for titles inside sectioning comments.

If the comment is more than one line long, the delimiters /-! and -/ should appear on their own lines.

See meta/expr.lean for an example in practice.

namespace binder_info /-! ### Declarations about `binder_info` This section develops an extended API for the type `binder_info`. -/ instance : inhabited binder_info := binder_info.default /-- The brackets corresponding to a given binder_info. -/ def brackets : binder_info string × string | binder_info.implicit := ("{", "}") | binder_info.strict_implicit := ("{{", "}}") | binder_info.inst_implicit := ("[", "]") | _ := ("(", ")") end binder_info namespace name /-! ### Declarations about `name` -/ /-- Find the largest prefix `n` of a `name` such that `f n ≠ none`, then replace this prefix with the value of `f n`. -/ def map_prefix (f : name option name) : name name | anonymous := anonymous | (mk_string s n') := (f (mk_string s n')).get_or_else (mk_string s $ map_prefix n') | (mk_numeral d n') := (f (mk_numeral d n')).get_or_else (mk_numeral d $ map_prefix n')

Theories documentation

In addition to documentation living in Lean file, we have tactic documentation in docs/tactics, and theory documentation in docs/theories where we give overviews spanning several Lean files, and more mathematical explanations in cases where formalization requires slightly exotic points of view, see for instance the topology documentation.

Examples

The following files are maintained as examples of good documentation style: