This webpage is about Lean 3, which is effectively obsolete; the community has migrated to Lean 4.

100 theorems

Freek Wiedijk maintains a list tracking progress of theorem provers in formalizing 100 classic theorems in mathematics as a way of comparing prominent theorem provers. Currently 76 of them are formalized in Lean. We also have a page with the theorems from the list not yet in mathlib.

1. The Irrationality of the Square Root of 2 #

Author: mathlib

docs, source

2. Fundamental Theorem of Algebra #

Author: Chris Hughes

theorem complex.exists_root {f : polynomial } (hf : 0 < f.degree) :
(z : ), f.is_root z

docs, source

3. The Denumerability of the Rational Numbers #

Author: Chris Hughes

docs, source

4. Pythagorean Theorem #

Author: Joseph Myers

docs, source

7. Law of Quadratic Reciprocity #

Author: Chris Hughes (first) and Michael Stoll (second)

theorem legendre_sym.quadratic_reciprocity {p q : } [fact (nat.prime p)] [fact (nat.prime q)] (hp : p 2) (hq : q 2) (hpq : p q) :
legendre_sym q p * legendre_sym p q = (-1) ^ (p / 2 * (q / 2))

docs, source

theorem jacobi_sym.quadratic_reciprocity {a b : } (ha : odd a) (hb : odd b) :
jacobi_sym a b = (-1) ^ (a / 2 * (b / 2)) * jacobi_sym b a

docs, source

9. The Area of a Circle #

Authors: James Arthur, Benjamin Davidson, and Andrew Souther

mathlib archive

10. Euler’s Generalization of Fermat’s Little Theorem #

Author: Chris Hughes

theorem nat.modeq.pow_totient {x n : } (h : x.coprime n) :
x ^ n.totient 1 [MOD n]

docs, source

11. The Infinitude of Primes #

Author: Jeremy Avigad

theorem nat.exists_infinite_primes (n : ) :
(p : ), n p nat.prime p

docs, source

14. Euler’s Summation of 1 + (1/2)^2 + (1/3)^2 + …. #

Authors: Marc Masdeu, David Loeffler

theorem has_sum_zeta_two  :
has_sum (λ (n : ), 1 / n ^ 2) (real.pi ^ 2 / 6)

docs, source

15. Fundamental Theorem of Integral Calculus #

Author: Yury G. Kudryashov (first) and Benjamin Davidson (second)

docs, source

theorem interval_integral.integral_eq_sub_of_has_deriv_right_of_le {E : Type u_3} [normed_add_comm_group E] [complete_space E] [normed_space E] {f : E} {a b : } {f' : E} (hab : a b) (hcont : continuous_on f (set.Icc a b)) (hderiv : (x : ), x set.Ioo a b has_deriv_within_at f (f' x) (set.Ioi x) x) (f'int : interval_integrable f' measure_theory.measure_space.volume a b) :
(y : ) in a..b, f' y = f b - f a

docs, source

16. Insolvability of General Higher Degree Equations (Abel-Ruffini Theorem) #

Author: Thomas Browning

mathlib archive

17. De Moivre’s Formula #

Author: Abhimanyu Pallavi Sudhir

docs, source

18. Liouville’s Theorem and the Construction of Transcendental Numbers #

Author: Jujian Zhang

docs, source

19. Four Squares Theorem #

Author: Chris Hughes

theorem nat.sum_four_squares (n : ) :
(a b c d : ), a ^ 2 + b ^ 2 + c ^ 2 + d ^ 2 = n

docs, source

20. All Primes (1 mod 4) Equal the Sum of Two Squares #

Author: Chris Hughes

theorem nat.prime.sq_add_sq {p : } [fact (nat.prime p)] (hp : p % 4 3) :
(a b : ), a ^ 2 + b ^ 2 = p

docs, source

22. The Non-Denumerability of the Continuum #

Author: Floris van Doorn

docs, source

23. Formula for Pythagorean Triples #

Author: Paul van Wamelen

theorem pythagorean_triple.classification {x y z : } :
pythagorean_triple x y z (k m n : ), (x = k * (m ^ 2 - n ^ 2) y = k * (2 * m * n) x = k * (2 * m * n) y = k * (m ^ 2 - n ^ 2)) (z = k * (m ^ 2 + n ^ 2) z = -k * (m ^ 2 + n ^ 2))

docs, source

24. The Independence of the Continuum Hypothesis #

Author: Jesse Michael Han and Floris van Doorn

result

website

see the README file in the linked repository.

25. Schroeder-Bernstein Theorem #

Author: Mario Carneiro

theorem function.embedding.schroeder_bernstein {α : Type u} {β : Type v} {f : α β} {g : β α} (hf : function.injective f) (hg : function.injective g) :

docs, source

26. Leibniz’s Series for Pi #

Author: Benjamin Davidson

theorem real.tendsto_sum_pi_div_four  :
filter.tendsto (λ (k : ), (finset.range k).sum (λ (i : ), (-1) ^ i / (2 * i + 1))) filter.at_top (nhds (real.pi / 4))

docs, source

27. Sum of the Angles of a Triangle #

Author: Joseph Myers

docs, source

30. The Ballot Problem #

Authors: Bhavik Mehta, Kexing Ying

mathlib archive

31. Ramsey’s Theorem #

Author: Bhavik Mehta

result

34. Divergence of the Harmonic Series #

Authors: Anatole Dedecker, Yury Kudryashov

docs, source

35. Taylor’s Theorem #

Author: Moritz Doll

theorem taylor_mean_remainder_lagrange {f : } {x x₀ : } {n : } (hx : x₀ < x) (hf : cont_diff_on n f (set.Icc x₀ x)) (hf' : differentiable_on (iterated_deriv_within n f (set.Icc x₀ x)) (set.Ioo x₀ x)) :
(x' : ) (hx' : x' set.Ioo x₀ x), f x - taylor_within_eval f n (set.Icc x₀ x) x₀ x = iterated_deriv_within (n + 1) f (set.Icc x₀ x) x' * (x - x₀) ^ (n + 1) / ((n + 1).factorial)

docs, source

theorem taylor_mean_remainder_cauchy {f : } {x x₀ : } {n : } (hx : x₀ < x) (hf : cont_diff_on n f (set.Icc x₀ x)) (hf' : differentiable_on (iterated_deriv_within n f (set.Icc x₀ x)) (set.Ioo x₀ x)) :
(x' : ) (hx' : x' set.Ioo x₀ x), f x - taylor_within_eval f n (set.Icc x₀ x) x₀ x = iterated_deriv_within (n + 1) f (set.Icc x₀ x) x' * (x - x') ^ n / (n.factorial) * (x - x₀)

docs, source

36. Brouwer Fixed Point Theorem #

Author: Brendan Seamas Murphy

result

37. The Solution of a Cubic #

Author: Jeoff Lee

mathlib archive

38. Arithmetic Mean/Geometric Mean #

Author: Yury G. Kudryashov

theorem real.geom_mean_le_arith_mean_weighted {ι : Type u} (s : finset ι) (w z : ι ) (hw : (i : ι), i s 0 w i) (hw' : s.sum (λ (i : ι), w i) = 1) (hz : (i : ι), i s 0 z i) :
s.prod (λ (i : ι), z i ^ w i) s.sum (λ (i : ι), w i * z i)

docs, source

39. Solutions to Pell’s Equation #

Authors: Mario Carneiro (first), Michael Stoll (second)

theorem pell.eq_pell {a : } (a1 : 1 < a) {x y : } (hp : x * x - d a1 * y * y = 1) :
(n : ), x = pell.xn a1 n y = pell.yn a1 n

docs, source

theorem pell.exists_of_not_is_square {d : } (h₀ : 0 < d) (hd : ¬is_square d) :
(x y : ), x ^ 2 - d * y ^ 2 = 1 y 0

docs, source

In pell.eq_pell, d is defined to be a*a - 1 for an arbitrary a > 1.

40. Minkowski’s Fundamental Theorem #

Authors: Alex J. Best, Yaël Dillies

docs, source

42. Sum of the Reciprocals of the Triangular Numbers #

Authors: Jalex Stark, Yury Kudryashov

mathlib archive

44. The Binomial Theorem #

Author: Chris Hughes

theorem add_pow {R : Type u_1} [comm_semiring R] (x y : R) (n : ) :
(x + y) ^ n = (finset.range (n + 1)).sum (λ (m : ), x ^ m * y ^ (n - m) * (n.choose m))

docs, source

45. The Partition Theorem #

Authors: Bhavik Mehta, Aaron Anderson

mathlib archive

49. The Cayley-Hamilton Theorem #

Author: Scott Morrison

theorem matrix.aeval_self_charpoly {R : Type u} [comm_ring R] {n : Type w} [decidable_eq n] [fintype n] (M : matrix n n R) :

docs, source

51. Wilson’s Lemma #

Author: Chris Hughes

theorem zmod.wilsons_lemma (p : ) [fact (nat.prime p)] :
((p - 1).factorial) = -1

docs, source

52. The Number of Subsets of a Set #

Author: mathlib

theorem finset.card_powerset {α : Type u_1} (s : finset α) :

docs, source

54. Königsberg Bridges Problem #

Author: Kyle Miller

mathlib archive

55. Product of Segments of Chords #

Author: Manuel Candales

docs, source

57. Heron’s Formula #

Author: Matt Kempster

mathlib archive

58. Formula for the Number of Combinations #

Author: mathlib

theorem finset.card_powerset_len {α : Type u_1} (n : ) (s : finset α) :

docs, source

theorem finset.mem_powerset_len {α : Type u_1} {n : } {s t : finset α} :

docs, source

59. The Laws of Large Numbers #

Author: Sébastien Gouëzel

docs, source

60. Bezout’s Theorem #

Author: mathlib

theorem nat.gcd_eq_gcd_ab (x y : ) :
(x.gcd y) = x * x.gcd_a y + y * x.gcd_b y

docs, source

62. Fair Games Theorem #

Author: Kexing Ying

docs, source

63. Cantor’s Theorem #

Author: mathlib

theorem cardinal.cantor (a : cardinal) :
a < 2 ^ a

docs, source

64. L’Hopital’s Rule #

Author: Anatole Dedecker

theorem deriv.lhopital_zero_nhds {a : } {l : filter } {f g : } (hdf : ∀ᶠ (x : ) in nhds a, differentiable_at f x) (hg' : ∀ᶠ (x : ) in nhds a, deriv g x 0) (hfa : filter.tendsto f (nhds a) (nhds 0)) (hga : filter.tendsto g (nhds a) (nhds 0)) (hdiv : filter.tendsto (λ (x : ), deriv f x / deriv g x) (nhds a) l) :
filter.tendsto (λ (x : ), f x / g x) (nhds_within a {a}) l

docs, source

65. Isosceles Triangle Theorem #

Author: Joseph Myers

docs, source

66. Sum of a Geometric Series #

Author: Sander R. Dahmen (finite) and Johannes Hölzl (infinite)

theorem geom_sum_Ico {α : Type u} [division_ring α] {x : α} (hx : x 1) {m n : } (hmn : m n) :
(finset.Ico m n).sum (λ (i : ), x ^ i) = (x ^ n - x ^ m) / (x - 1)

docs, source

theorem nnreal.has_sum_geometric {r : nnreal} (hr : r < 1) :
has_sum (λ (n : ), r ^ n) (1 - r)⁻¹

docs, source

67. e is Transcendental #

Author: Jujian Zhang

result

website

68. Sum of an arithmetic series #

Author: Johannes Hölzl

theorem finset.sum_range_id (n : ) :
(finset.range n).sum (λ (i : ), i) = n * (n - 1) / 2

docs, source

69. Greatest Common Divisor Algorithm #

Author: mathlib

docs, source

docs, source

theorem euclidean_domain.dvd_gcd {R : Type u} [euclidean_domain R] [decidable_eq R] {a b c : R} :

docs, source

70. The Perfect Number Theorem #

Author: Aaron Anderson

mathlib archive

71. Order of a Subgroup #

Author: mathlib

docs, source

72. Sylow’s Theorem #

Author: Chris Hughes

theorem sylow.exists_subgroup_card_pow_prime {G : Type u} [group G] [fintype G] (p : ) {n : } [fact (nat.prime p)] (hdvd : p ^ n fintype.card G) :

docs, source

sylow_conjugate

card_sylow_dvd

card_sylow_modeq_one

73. Ascending or Descending Sequences (Erdős–Szekeres Theorem) #

Author: Bhavik Mehta

mathlib archive

74. The Principle of Mathematical Induction #

Author: Leonardo de Moura

inductive nat  :

docs, source

Automatically generated when defining the natural numbers

75. The Mean Value Theorem #

Author: Yury G. Kudryashov

theorem exists_deriv_eq_slope (f : ) {a b : } (hab : a < b) (hfc : continuous_on f (set.Icc a b)) (hfd : differentiable_on f (set.Ioo a b)) :
(c : ) (H : c set.Ioo a b), deriv f c = (f b - f a) / (b - a)

docs, source

76. Fourier Series #

Author: Heather Macbeth

noncomputable def fourier_coeff {T : } [hT : fact (0 < T)] {E : Type} [normed_add_comm_group E] [normed_space E] [complete_space E] (f : add_circle T E) (n : ) :
E

docs, source

docs, source

77. Sum of kth powers #

Authors: mathlib (Moritz Firsching, Fabian Kruse, Ashvni Narayanan)

theorem sum_range_pow (n p : ) :
(finset.range n).sum (λ (k : ), k ^ p) = (finset.range (p + 1)).sum (λ (i : ), bernoulli i * ((p + 1).choose i) * n ^ (p + 1 - i) / (p + 1))

docs, source

theorem sum_Ico_pow (n p : ) :
(finset.Ico 1 (n + 1)).sum (λ (k : ), k ^ p) = (finset.range (p + 1)).sum (λ (i : ), bernoulli' i * ((p + 1).choose i) * n ^ (p + 1 - i) / (p + 1))

docs, source

78. The Cauchy-Schwarz Inequality #

Author: Zhouhang Zhou

docs, source

theorem norm_inner_le_norm {𝕜 : Type u_1} {E : Type u_2} [is_R_or_C 𝕜] [normed_add_comm_group E] [inner_product_space 𝕜 E] (x y : E) :

docs, source

79. The Intermediate Value Theorem #

Author: mathlib (Rob Lewis and Chris Hughes)

theorem intermediate_value_Icc {α : Type u} [conditionally_complete_linear_order α] [topological_space α] [order_topology α] [densely_ordered α] {δ : Type u_1} [linear_order δ] [topological_space δ] [order_closed_topology δ] {a b : α} (hab : a b) {f : α δ} (hf : continuous_on f (set.Icc a b)) :
set.Icc (f a) (f b) f '' set.Icc a b

docs, source

80. The Fundamental Theorem of Arithmetic #

Author: mathlib (Chris Hughes)

theorem nat.factors_unique {n : } {l : list } (h₁ : l.prod = n) (h₂ : (p : ), p l nat.prime p) :

docs, source

docs, source

docs, source

docs, source

docs, source

it also has a generalized version, by showing that every Euclidean domain is a unique factorization domain, and showing that the integers form a Euclidean domain.

81. Divergence of the Prime Reciprocal Series #

Author: Manuel Candales

mathlib archive

82. Dissection of Cubes (J.E. Littlewood’s ‘elegant’ proof) #

Author: Floris van Doorn

mathlib archive

83. The Friendship Theorem #

Authors: Aaron Anderson, Jalex Stark, Kyle Miller

mathlib archive

85. Divisibility by 3 Rule #

Author: Scott Morrison

theorem nat.three_dvd_iff (n : ) :
3 n 3 (10.digits n).sum

docs, source

86. Lebesgue Measure and Integration #

Author: Johannes Hölzl

noncomputable def measure_theory.lintegral {α : Type u_1} {m : measurable_space α} (μ : measure_theory.measure α) (f : α ennreal) :

docs, source

88. Derangements Formula #

Author: Henry Swanson

docs, source

theorem num_derangements_sum (n : ) :
(num_derangements n) = (finset.range (n + 1)).sum (λ (k : ), (-1) ^ k * (k.asc_factorial (n - k)))

docs, source

89. The Factor and Remainder Theorems #

Author: Chris Hughes

docs, source

docs, source

90. Stirling’s Formula #

Authors: mathlib (Moritz Firsching, Fabian Kruse, Nikolas Kuhn, Heather Macbeth)

docs, source

91. The Triangle Inequality #

Author: Zhouhang Zhou

theorem norm_add_le {E : Type u_6} [seminormed_add_group E] (a b : E) :

docs, source

93. The Birthday Problem #

Author: Eric Rodriguez

mathlib archive

94. The Law of Cosines #

Author: Joseph Myers

docs, source

95. Ptolemy’s Theorem #

Author: Manuel Candales

docs, source

96. Principle of Inclusion/Exclusion #

Author: Neil Strickland

github

97. Cramer’s Rule #

Author: Anne Baanen

theorem matrix.mul_vec_cramer {n : Type v} {α : Type w} [decidable_eq n] [fintype n] [comm_ring α] (A : matrix n n α) (b : n α) :
A.mul_vec ((A.cramer) b) = A.det b

docs, source

98. Bertrand’s Postulate #

Authors: Bolton Bailey, Patrick Stevens

theorem nat.bertrand (n : ) (hn0 : n 0) :
(p : ), nat.prime p n < p p 2 * n

docs, source