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

Originally from `module.cpp` (RIP) ---- - Persistent `set_option`. We want to be able to store the option settings in .olean files. The main issue is conflict between imported modules. That...

enhancement
nice to have

@Kha when `panic` is evaluated by the interpreter, the execution is interrupted as expected. However, all trace messages produced using `dbgTrace` are lost because the `#eval` command implementation redirects stdout...

enhancement

Consider the following variants of a `cache` function ```lean import Lean set_option trace.compiler.ir.result true open Lean structure State where keys : Array Expr results : Array Expr abbrev M :=...

enhancement
depends on new code generator

### Prerequisites * [x] Put an X between the brackets on this line if you have done all of the following: * Checked that your issue isn't already [filed](https://github.com/leanprover/lean4/issues). *...

enhancement
low priority

We store the Lean wrappers of stdin/stdout/stderr in thread-local variables to support redirection as in `withStdin/...`. New threads spawned within these functions should inherit these variables. Note that if a...

enhancement

### Prerequisites * [x] Put an X between the brackets on this line if you have done all of the following: * Checked that your issue isn't already [filed](https://github.com/leanprover/lean4/issues). *...

enhancement
low priority

The current standard library in the Lean core is lacking many common utility functions. One way to go about fleshing it out is to allow the community to contributed useful...

nice to have
community effort

### Prerequisites * [x] Put an X between the brackets on this line if you have done all of the following: * Checked that your issue isn't already [filed](https://github.com/leanprover/lean4/issues). *...

bug
low priority

As some of the Lean 3 widget features are [rolling in](https://github.com/leanprover/vscode-lean4/pull/37), we should decide on the next step. I think a good one would be to provide a typeclass which...

enhancement

We had this option in Lean 3.

enhancement
lean4_release