As a step towards computer-formalizing the classification of low-dimensional Lie algebras, we finally formalized our first non-boring theorem in #Lean4 !
If L is a 3-dimensional Lie algebra (over any field) with a one-dimensional commutator subalgebra which is contained in the center of L, then L is isomorphic to the 3D Heisenberg algebra - that is, it has a basis (𝑒₀, 𝑒₁, 𝑒₂) such that the bracket is determined by
[𝑒₁,𝑒₂]=𝑒₀,
[𝑒₀,𝑒₁]=0,
[𝑒₀,𝑒₂]=0.
Now we're working on the analogous results for higher dimensional commutator subalgebras. These are going to be harder because
a) there's no one-size-fits-all classification statement for arbitrary fields, and
b) they rely on certain normal forms of matrices which aren't yet implemented in #mathlib .
The Matrix Cookbook, using Lean's mathlib. ~ Eric Wieser. https://github.com/eric-wieser/lean-matrix-cookbook #ITP #LeanProver #Lean4 #Mathlib #Math
Readings shared September 21, 2024. https://jaalonso.github.io/vestigium/posts/2024/09/21-readings_shared_09-21-24 #ITP #IsabelleHOL #LeanProver #Lean3 #Lean4 #Mathlib #Logic #Math #AI #LLMs #DeepLearning
Finding lemmas in Mathlib. ~ Damiano Testa. https://github.com/adomani/MA4N1_Theorem_proving_with_Lean/blob/master/MA4N1_2023/L17_navigating_Mathlib.lean #ITP #LeanProver #Mathlib
Lecturas compartidas el 1 de agosto de 2024. https://jaalonso.github.io/vestigium/posts/2024/08/02-lecturas_compartidas_el_01-ago-24 #ITP #Lean4 #Mathlib #Coq #Math #Haskell #FunctionalProgramming
Search Mathlib: A webpage that searches for Mathlib theorems. ~ Deming Xu. https://huggingface.co/spaces/dx2102/search-mathlib #ITP #Lean4 #Mathlib
LeanSearch: Find theorems in Mathlib4 using natural language query. https://leansearch.net #ITP #Lean4 #Mathlib
This month in Mathlib (May 2024). https://leanprover-community.github.io/blog/posts/month-in-mathlib/2024/month-in-mathlib-may-2024/ #ITP #Lean4 #Mathlib #Math
All tactics in mathlib4. ~ Haruhisa Enomoto. https://github.com/haruhisa-enomoto/mathlib4-all-tactics/blob/main/all-tactics.md #ITP #LeanProver #Mathlib