Lean (proof assistant)

Print Print
Reading time 3:31

Lean (proof assistant)
Developer(s)Microsoft Research
Initial release2013; 8 years ago (2013)
Stable release
4.0.0-m2 / 2 March 2021; 3 months ago (2021-03-02)
Repositorygithub.com/leanprover/lean
Written inC++
Operating systemCross-platform
Available inEnglish
TypeProof assistant
LicenseApache License 2.0
Websiteleanprover.github.io

Lean is a theorem prover and programming language. It is based on the calculus of constructions with inductive types.

The Lean project is an open source project, hosted on GitHub. It was launched by Leonardo de Moura at Microsoft Research in 2013.[1]

Lean has an interface that differentiates it from other interactive theorem provers. Lean can be compiled to JavaScript and accessed in a web browser. It has native support for Unicode symbols. (These can be typed using LaTeX-like sequences, such as "\times" for "×".) Lean also has an extensive support for meta-programming.

Lean has gotten attention from mathematicians Thomas Hales[2] and Kevin Buzzard.[3] Hales is using it for his project, Formal Abstracts. Buzzard uses it for the Xena project. One of the Xena Project's goals is to rewrite every theorem and proof in the undergraduate math curriculum of Imperial College London in Lean.

Examples

Here is how the natural numbers are defined in Lean.

inductive nat : Type
| zero : nat
| succ : nat  nat

Here is the addition operation defined for natural numbers.

definition add : nat  nat  nat
| n zero     := n
| n (succ m) := succ(add n m)

This is a simple proof in lean in term mode.

theorem and_swap : p  q  q  p :=
    assume h1 : p  q,
    h1.right, h1.left

This same proof can be accomplished using tactics.

theorem and_swap (p q : Prop) : p  q  q  p :=
begin
    assume h : (p  q), -- assume p ∧ q is true
    cases h, -- extract the individual propositions from the conjunction
    split, -- split the goal conjunction into two cases: prove p and prove q separately
    repeat { assumption }
end

See also

  • Proof assistant
  • mimalloc

References

  1. ^ https://leanprover.github.io/about/
  2. ^ Hales, Thomas. "A Review of the Lean Theorem Prover". Retrieved 6 October 2020.
  3. ^ Buzzard, Kevin. "The Future of Mathematics?" (PDF). Retrieved 6 October 2020.

By: Wikipedia.org
Edited: 2021-06-18 18:14:12
Source: Wikipedia.org