-
Getting this error when trying to load this library on Android (Termux). This doesn't appear to be a problem on any other targets. Builds for macos, windows & linux all work as expected.
Is there …
-
Hi everyone,
This is Rex, and I have been exploring this fantastic project. It's a great starting point for newcomers to get an introduction to Lean! And I think it could be even more engaging and …
-
**What question should the reference manual answer?**
One of the [most common tactic bugs](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/weird.20tactic.20bug/near/370576262…
-
Maybe you're already aware or don't want to constantly update how Mathlib is used, but some of the things in your repo are already in Mathlib. For example some of the things here:
https://github.co…
-
Report by the Lean FRO:
I am observing a possible bug with lean4web: If I am open, for example, https://lean.math.hhu.de/#project=nightly&codez=M4EwZkA
and look at the network tab of the Firefox d…
-
# To-Do List
- [ ] Port `IsInvariant` and `inv_def'` from InvariantSubset.lean (needs to be harmonized/unified with IsInvariant under Flow in mathlib)
- [ ] Move results on invariance and orbits f…
mseri updated
4 months ago
-
As already issued here: https://github.com/leanprover-community/mathlib4/issues/15415
It seems that the documentation assumes `x.abs` to be the polymorphic version, but doesn't see that there is al…
-
I am not sure if Bell numbers are currently supported in Mathlib, so this may require also creating some API for Bell numbers in /forMathlib.
When done, update Lemma 1.8 in the blueprint with \leanok…
-
Updating to the new Mathlib version (2024-09-26) broke AliveStatement `bv_AddSub_1556`:
```lean
theorem broken {x y : BitVec 1} : y - x = y ^^^ x := by
bv_automata
```
The offending commit…
-
These involve counting the number of equations up to relabeling and relabeling + symmetry, they involve the Catalan numbers and the [Bell numbers](https://en.wikipedia.org/wiki/Bell_number) which AFAI…