OrderPQ
This is an open-source project that formalises in the Lean theorem prover the classification of the groups of order p * q
where p
and q
are prime numbers, using mathlib.
The main theorems are in Main.lean.
Also formalised as part of the project are some key properties of semidirect products of groups and a number of other group-theoretic results.
The authors are
Upstream PRs
The following pull requests (PRs) to mathlib and its dependencies were necessitated or inspired by this project. Further PRs will be made in due course.
- leanprover/lean4#4037: Added
dite_some_none_eq_none
anddite_some_none_eq_some
to the moduleInit.ByCases
. - leanprover-community/mathlib4#14097: Added
toAdd_eq_zero
andtoMul_eq_one
to the moduleMathlib.Algebra.Group.TypeTags
. - leanprover-community/mathlib4#14104 and leanprover-community/mathlib4#14154: Added
Prod.orderOf_mk
to the moduleMathlib.GroupTheory.OrderOfElement
. - leanprover-community/mathlib4#14365: Added lemmas on sufficient conditions for two
Set
s orSubgroup
s to be equal.
License
The source code of this project is distributed under the terms of the Apache License 2.0. See LICENSE for more details.