SaaSHub helps you find the best software and product alternatives Learn more →
Mathlib4 Alternatives
Similar projects and alternatives to mathlib4
-
-
CodeRabbit
CodeRabbit: AI Code Reviews for Developers. Revolutionize your code reviews with AI. CodeRabbit offers PR summaries, code walkthroughs, 1-click suggestions, and AST-based analysis. Boost productivity and code quality across all major languages with each PR.
-
-
gmp-wasm
Fork of the GNU Multiple Precision Arithmetic Library (GMP), suitable for compilation into WebAssembly.
-
-
-
-
TypeTopology
Logical manifestations of topological concepts, and other things, via the univalent point of view.
-
SaaSHub
SaaSHub - Software Alternatives and Reviews. SaaSHub helps you find the best software and product alternatives
-
UniMath
This coq library aims to formalize a substantial body of mathematics using the univalent point of view.
-
-
turing
A reference implementation of Alan Turing's 1936 paper, On Computable Numbers (by planetlambert)
-
-
-
-
-
SaaSHub
SaaSHub - Software Alternatives and Reviews. SaaSHub helps you find the best software and product alternatives
mathlib4 discussion
mathlib4 reviews and mentions
-
Fermat's Last Theorem – how it's going
> shouldn't proof checkers have a database of theorems and be able to fill in the intermediate steps or confirm that it's possible to fill in the missing steps?
This is essentially exactly what Mathlib[1] is, which is Lean's database of mathematics, and which large portions of the FLT project will likely continually contribute into.
(Other theorem provers have similar libraries, e.g. Coq's is called math-comp: https://math-comp.github.io/ )
[1]: https://github.com/leanprover-community/mathlib4/
- The Future of TLA+ [pdf]
-
How to choose a textbook that is pedagogically optimal for oneself?
I am not aware of any good one, but I realized you could probably mechanically extract such a map from Lean's mathlib[0][1].
Since Lean builds everything from scratch, this should be doable, albeit Lean builds everything on top of type theory which is not the only choice possible. Different foundations will result in a different graph.
Also the best way to learn is probably not this sort of graph.
[0] https://leanprover-community.github.io/mathlib4_docs/
-
A Linear Algebra Trick for Computing Fibonacci Numbers Fast
We essentially implemented this matrix version in Lean/mathlib to both compute the fibonacci number and generate an efficient proof for the calculation.
https://github.com/leanprover-community/mathlib4/blob/master...
In practice this isn't very useful (the definition of Nat.fib unfolds quick enough and concrete large fibonacci numbers don't often appear in proofs) but still it shaves a bit of time off the calculation and the proof verification.
-
Show HN: The first complete open source implementation of Turing's famous paper
As an aside, there are a number of Turing machines defined in Lean's mathlib. https://github.com/leanprover-community/mathlib4/blob/2c3ee3...
-
Lean 4.0.0, first official lean4 release
Thanks,
and there is Subobject, which looks like the subobject classifier.
https://github.com/leanprover-community/mathlib4/blob/master...
-
Are There People Doing Formal Math In Berlin?
I just wonder if there are any irl meetups of people involved with formalizing mathematics, I thought that it would be a cool hobby to pick up (with some background in math and programming) but the existing libraries, like MathLib, TypeTopology or UniMath look a bit intimidating...
-
Good First Formal Proof?
What is a good proof in either unimath or mathlib4 or somewhere else to get started with formal proofs? Like some well known result without too many dependencies, but still nothing trivial like propositional logic?
-
Functional Programming in Lean – a book on using Lean 4 to write programs
For searching using search terms for theorems in mathlib, there is the mathlib documentation page (for Lean 3 https://leanprover-community.github.io/mathlib_docs/ and Lean 4 https://leanprover-community.github.io/mathlib4_docs/). To find theorems by type, I find the best way is to use the `library_search` tactic from inside Lean itself.
-
Good Entry Points For `mathlib4`?
Hello, I'd like to start learning Lean 4. I'm already reading the book, but I'm really curious to study real-life parallel. So I looked into mathlib4, but there seem to be a lot of dependencies between the the files. So I wonder the following:
-
A note from our sponsor - SaaSHub
www.saashub.com | 16 Mar 2025
Stats
leanprover-community/mathlib4 is an open source project licensed under Apache License 2.0 which is an OSI approved license.
The primary programming language of mathlib4 is Lean.