-
### Description
In a configuration with multiple libraries, "go to definition" fails in some circumstances.
### Context
I had noticed intermittent failures of "go to definition" while working…
-
I have the Chrome Gitpod extension installed, and when I click on the Gitpod button
that appears on the page, it opens up a VSCode environment, showing the following
messages in the terminal window:…
-
It would be great to be able to run LEAN from Proof-General
https://github.com/leanprover/lean
https://leanprover.github.io/tutorial/
-
### Proposal
There's a few places in Std and Mathlib where there is a desire to filter out auto-generated and other stable names (e.g., leanprover/std4#347 and leanprover/std4#355).
I think this…
-
Zulip: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Deprecation.20and.20time.20out
MWE reported by @AntoineChambert-Loir :
```lean
import Mathlib.RingTheory.TensorProduct…
-
Classifies porting notes claiming anything semantically equivalent to
- "`simp` can prove this"
- "`simp` can simplify this`"
- "was `@[simp]`, now can be proved by `simp`"
- "was `@[simp]`, but …
-
### 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
* …
-
I'm encountering an error while trying to install a specific lean toolchain with elan. I'm not sure what could be happening, if this is a problem with elan, or if this is a user-error (and perhaps in …
-
As an experiment, I created a `lakefile.lean` as follows
```lean
import Lake
open Lake DSL
package "benchmark" where
-- add package configuration options here
@[default_target]
lean_exe…
-
Many of the theorem statements does not have formal proofs(they have the sorry tags). If I have a generated proof for a theorem how should I evaluate it, even if we have a predicted proof and ground t…