-
See https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Dynamics/Minimal.lean
Our minimal sets need to be extended to action and topological spaces
mseri updated
4 months ago
-
### Prerequisites
Please put an X between the brackets as you perform the following steps:
* [x] Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues
* …
TwoFX updated
1 month ago
-
- [x] Most of the statements work for `UniqueFactorizationMonoid` with normalization (or even without normalization, up to unit), so we may upgrade them first by replacing `k[X]` with general `UniqueF…
-
### Prerequisites
Please put an X between the brackets as you perform the following steps:
* [x] Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues
* …
TwoFX updated
1 month ago
-
### Prerequisites
Please put an X between the brackets as you perform the following steps:
* [X] Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues
* …
-
### Proposal
Add a `-j` option to `lake build` to only spawn `N` compilation threads, similar to tools like `make` or `cargo build`.
If this is difficult to implement, it might be good enough to…
-
## The problem
The present set of prompts, extracted from `mathlib`, has the following known limitations:
* __LaTeX formulas__ : Docstrings contain formulas as Lean code in backticks so example …
-
A long standing issue is that the kernel will happily try to reduce functions defined by well-founded recursion (#2171), and then this often fails with `(kernel) deep recursion detected`.
This lead…
-
```lean
import Mathlib.Data.Int.Cast.Defs
variable {R : Type _} [AddGroupWithOne R]
namespace Int
@[norm_cast] -- Removing this attribute fixes the issue
theorem cast_negSucc (n : ℕ) : (-[n…
-
```lean
import Mathlib.Data.Nat.Factorial.Basic
open Nat
example (n : ℕ) : ∃ m : ℕ, 0 + n ! = m := by
use n !
simp
```
The code above parses incorrectly. Replacing line 5 with `use (n !)`…