lean4 icon indicating copy to clipboard operation
lean4 copied to clipboard

Lean 4 programming language and theorem prover

Results 621 lean4 issues
Sort by recently updated
recently updated
newest added

awaiting-author
builds-mathlib
toolchain-available

The current `Classical.em` proof isn't that easy to follow. Since Lean has quotients, we can take a two-element type like `Bool`, and quotient it by `x = y ∨ P`....

low priority
P-low

This fixes indentation before `|` in places where the amount of spaces was not 0 or 2. I suppose this is the non-controversial part of #2580. Deciding for either 0...

Fixes #2483

low priority
awaiting-review
builds-mathlib
toolchain-available
P-low

* [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/memory.20model.20of.20natural.20numbers/near/387485542) Documentation regarding the borrowing convention of arguments and return values for C functions in `lean.h` and related files is very important for FFI writers to be able...

low priority
P-low

implementation based on: https://ieeexplore.ieee.org/stamp/stamp.jsp?tp=&arnumber=987767 co-authored by @bollu

builds-mathlib
toolchain-available

This PR adds a small docstring to `Simp.Methods.discharge?` - (this is what I *think* it does, so any corrections are appreciated:)) This was suggested in the review of [this mathlib...

toolchain-available
P-low

This PR provides functions to merge and split vectors of bitvectors, taking up the abandoned #3727.

WIP
toolchain-available
P-medium
changelog-library

This PR ensures that `libuv` objects are cleaned up by `finalize_runtime_module()`. Closes #7753

toolchain-available
release-ci

This PR adds a bitblasting cache for the boolean substructure of problems that bv_decide works on in addition to the one used for bvexpr. Unfortunately this is currently causing a...

toolchain-available
changelog-language