lean4 icon indicating copy to clipboard operation
lean4 copied to clipboard

Lean 4 programming language and theorem prover

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

Since `nightly-2025-06-21` the file `CoreM.lean` changed line `670` to `defValue := true`. The new code generator does not want to generate code any more for the some of my code....

bug
P-low

### Description Ambiguous name errors while pattern matching in `do`-notation are swallowed and replaced by an unrelated message about syntax pattern matching. ### Context This occurred while migrating Verso code...

bug
P-medium

Consider ``` -- import Lean set_option linter.unusedSimpArgs false example : True := by simp [BitVec.reduceEq] ``` hovering over the simproc it just says ``` A simp lemma specification is: optional...

bug
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

Consider this ``` /-- error: Tactic `split` failed: Could not split an `if` or `match` expression in the goal n : Nat ⊢ Fin.last n = match id n with...

bug
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 We should support attribute declaration modifiers on inductive constructors. This would allow the following example from mathlib [here](https://github.com/leanprover-community/mathlib4/blob/f0e5f810b831671addae1078f6e05fb3697276ab/Mathlib/Logic/Relation.lean#L256-L262): ```lean @[mk_iff ReflTransGen.cases_tail_iff] inductive ReflTransGen (r : α → α...

RFC
P-medium

This is split out of #371. I would like to see support for match guards: some sort of boolean clause attached to a match branch which must return true if...

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
P-high

### 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...

P-low