lean4
lean4 copied to clipboard
Lean 4 programming language and theorem prover
I expected to see that on this page/section of the doc https://leanprover.github.io/lean4/doc/organization.html but it isn't listed there
### 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). *...
```lean import Lean syntax "foo " str : tactic open Lean Elab elab_rules : tactic | `(foo $x:str) => logInfo x.getString example : True := by foo "hello" -- Error...
We currently use the longest match parser combinator only when processing syntax categories. During the ICERM after-party hackton, users created fake "syntax category" to get the longest match behavior. BTW,...
In Lean 3 we had `by have : stmt := proof; exact term` which added `stmt` to the local context *without leaving any trace behind*. In Lean 4 `have` always...
### 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). *...
@digama0 and I want to make sure tactics such as `Ring` can be invoked from `simp`.
This issue is a placeholder for collecting ideas and features for visualizing and filtering traces. @dselsam @Kha @Vtec234
Continuing discussion from [here](https://github.com/leanprover/lean4/issues/681#issuecomment-922544455) and #1157. There is currently an inconsistency between whether the head symbol in a function application is hoverable/selectable in source code and in the infoview. I...
The formatter in the pretty printer already produces pretty good output for goals and also makes a reasonable attempt at preserving comments and command-level layout: https://github.com/leanprover/lean4/blob/master/tests/lean/Reformat.lean.expected.out. But it is not...