The inequality p⁻¹ + q⁻¹ + r⁻¹ > 1 #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we classify solutions to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1, for positive natural numbers p, q, and r.
The solutions are exactly of the form.
- A' q r := {1,q,r}
- D' r := {2,2,r}
- E6 := {2,3,3}, or- E7 := {2,3,4}, or- E8 := {2,3,5}
This inequality shows up in Lie theory, in the classification of Dynkin diagrams, root systems, and semisimple Lie algebras.
Main declarations #
- pqr.A' q r, the multiset- {1,q,r}
- pqr.D' r, the multiset- {2,2,r}
- pqr.E6, the multiset- {2,3,3}
- pqr.E7, the multiset- {2,3,4}
- pqr.E8, the multiset- {2,3,5}
- pqr.classification, the classification of solutions to- p⁻¹ + q⁻¹ + r⁻¹ > 1
A' q r := {1,q,r} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
Equations
- ADE_inequality.A' q r = {1, q, r}
A r := {1,1,r} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
These solutions are related to the Dynkin diagrams $A_r$.
Equations
D' r := {2,2,r} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
These solutions are related to the Dynkin diagrams $D_{r+2}$.
Equations
- ADE_inequality.D' r = {2, 2, r}
E' r := {2,3,r} is a multiset ℕ+.
For r ∈ {3,4,5} is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
These solutions are related to the Dynkin diagrams $E_{r+3}$.
Equations
- ADE_inequality.E' r = {2, 3, r}
E6 := {2,3,3} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
This solution is related to the Dynkin diagrams $E_6$.
Equations
E7 := {2,3,4} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
This solution is related to the Dynkin diagrams $E_7$.
Equations
E8 := {2,3,5} is a multiset ℕ+
that is a solution to the inequality
(p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1.
This solution is related to the Dynkin diagrams $E_8$.
Equations
sum_inv pqr for a pqr : multiset ℕ+ is the sum of the inverses
of the elements of pqr, as rational number.
The intended argument is a multiset {p,q,r} of cardinality 3.
Equations
- ADE_inequality.sum_inv pqr = (multiset.map (λ (x : ℕ+), (↑x)⁻¹) pqr).sum
A multiset pqr of positive natural numbers is admissible
if it is equal to A' q r, or D' r, or one of E6, E7, or E8.
Equations
- ADE_inequality.admissible pqr = ((∃ (q r : ℕ+), ADE_inequality.A' q r = pqr) ∨ (∃ (r : ℕ+), ADE_inequality.D' r = pqr) ∨ ADE_inequality.E' 3 = pqr ∨ ADE_inequality.E' 4 = pqr ∨ ADE_inequality.E' 5 = pqr)
A multiset {p,q,r} of positive natural numbers
is a solution to (p⁻¹ + q⁻¹ + r⁻¹ : ℚ) > 1 if and only if
it is admissible which means it is one of:
- A' q r := {1,q,r}
- D' r := {2,2,r}
- E6 := {2,3,3}, or- E7 := {2,3,4}, or- E8 := {2,3,5}