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

See for example ``` #check List.Sublist.below.cons List.Sublist.below.cons.{u_1} {α : Type u_1} : ∀ {motive : (a a_1 : List α) → a.Sublist a_1 → Prop} {l₁ l₂ : List α}...

RFC
P-low

Without this change, ```lean example : True := by refine' trivial .. . trivial ``` is a parse error. # Read this section before submitting * Ensure your PR follows...

toolchain-available
P-medium

### Description constructor of structure does not accept defalut value of field whose type is not `Prop`. ```lean structure NonEmptyString where value : String another_value : Int := 0 ev...

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

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

MWE: ```lean import Lean elab (ident)? ("Foo") : command => sorry syntax "Fix " colGt ident : tactic example (x : Lean.TSyntax `ident) : Lean.MacroM Lean.Syntax := `(tactic| Fix $x:iden)...

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

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-low

builds-mathlib
toolchain-available
release-ci

breaks-mathlib
toolchain-available