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

### 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 * [x] Reduce the...

bug
depends on new code generator
P-medium

We currently have to manually write `DecidableEq` instances for nested and mutual inductive datatypes. Here is an example. ```lean namespace Example inductive Min where | Base | Const (a :...

feature
P-medium

### Proposal #### Multiple edits I would be able to address #4546 in maybe the most preferable way if the the “Try this” functionality would allow multiple simultaneous replacements. In...

RFC
P-low

### 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 * [x] Reduce the...

bug
depends on new code generator
P-medium

``` import Lean example (range : String.Range) : String.Pos := ⟨range.stop.b⟩ example (p : String.Pos) : String.Pos := ⟨p.b⟩ ``` Both `b`s complete to very different lists, but neither contains...

bug
server
P-medium

### 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 * [x] Reduce the...

bug
P-medium

### Proposal Add a built in option to disable compilation. [Here](https://github.com/leanprover/lean4/commit/c02bcb6b679eed0f7a7c2f812d63ac3b06a15ed6) is one possibility. (Edit: this is too naive.) - **User Experience**: Currently, Lean attempts to compile declarations in `noncomputable...

RFC
Mathlib4 high prio
P-high

Here is an example failing build of Mathport due to a moved upstream file: ``` $ lake build ✖ [63/1717] Running Mathlib.Init.ZeroOne error: no such file or directory (error code:...

bug
Lake
P-medium

### 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 * [x] Reduce the...

bug
P-low

### 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 * [x] Reduce the...

bug
P-medium