mathlib4

The math library of Lean 4 (by leanprover-community)

Mathlib4 Alternatives

Similar projects and alternatives to mathlib4

  1. learnxinyminutes-docs

    Code documentation written as code! How novel and totally my idea!

  2. 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.

    CodeRabbit logo
  3. lean4

    62 mathlib4 VS lean4

    Lean 4 programming language and theorem prover

  4. gmp-wasm

    Fork of the GNU Multiple Precision Arithmetic Library (GMP), suitable for compilation into WebAssembly.

  5. mathlib3

    Discontinued Lean 3's obsolete mathematical components library: please use mathlib4

  6. P

    11 mathlib4 VS P

    The P programming language.

  7. topos

    Topos theory in lean (by b-mehta)

  8. TypeTopology

    Logical manifestations of topological concepts, and other things, via the univalent point of view.

  9. SaaSHub

    SaaSHub - Software Alternatives and Reviews. SaaSHub helps you find the best software and product alternatives

    SaaSHub logo
  10. UniMath

    This coq library aims to formalize a substantial body of mathematics using the univalent point of view.

  11. logical_verification_2023

    Hitchhiker's Guide to Logical Verification (2023 Edition)

  12. turing

    A reference implementation of Alan Turing's 1936 paper, On Computable Numbers (by planetlambert)

  13. lean4-raytracer

    A simple raytracer written in Lean 4

  14. lean4-mode

    2 mathlib4 VS lean4-mode

    Emacs major mode for Lean 4

  15. math-comp

    Mathematical Components

  16. fib-bench

    Benchmark of a few Ruby implementations of Fibonacci

  17. SaaSHub

    SaaSHub - Software Alternatives and Reviews. SaaSHub helps you find the best software and product alternatives

    SaaSHub logo
NOTE: The number of mentions on this list indicates mentions on common posts plus user suggested alternatives. Hence, a higher number means a better mathlib4 alternative or higher similarity.

mathlib4 discussion

Log in or Post with

mathlib4 reviews and mentions

Posts with mentions or reviews of mathlib4. We have used some of these posts to build our list of alternatives and similar projects. The last one was on 2024-12-12.
  • Fermat's Last Theorem – how it's going
    2 projects | news.ycombinator.com | 12 Dec 2024
    > 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]
    2 projects | news.ycombinator.com | 28 Aug 2024
  • How to choose a textbook that is pedagogically optimal for oneself?
    2 projects | news.ycombinator.com | 20 Jul 2024
    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
    3 projects | news.ycombinator.com | 6 Nov 2023
    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
    2 projects | news.ycombinator.com | 17 Sep 2023
    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
    10 projects | news.ycombinator.com | 7 Sep 2023
    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?
    3 projects | /r/berlinsocialclub | 13 Jun 2023
    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?
    1 project | /r/askmath | 10 Jun 2023
    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
    2 projects | news.ycombinator.com | 29 May 2023
    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`?
    1 project | /r/math | 16 May 2023
    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
    SaaSHub helps you find the best software and product alternatives Learn more →

Stats

Basic mathlib4 repo stats
14
1,791
10.0
4 days ago

Sponsored
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.
coderabbit.ai