-
Amazing library, thanks so much for the amazing work.
We are just attempting to update and we are having a problem:
In https://github.com/leanprover-community/quote4/pull/49 the option was added…
-
Consider
```lean
@[reducible] def g (x : α) := x
-- def foo := @g.eq_def
example (P : Nat → Prop) : P (id (g 42)) := by
simp only [g.eq_def]
```
and hover over the `g.eq_def` in the las…
-
1. I would like to use the ideas from https://homepages.inf.ed.ac.uk/wadler/papers/prettier/prettier.pdf implemented in Lean as Format type.
2. I would like to follow the idea of codecs from https:…
-
The [Shapley-Folkman lemma](https://eml.berkeley.edu/~anderson/Econ201B/NonconvexHandout.pdf) is a convex analysis result standard in the economics literature. In contrast, it is basically unheard of …
-
### 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
* …
-
The middle `String` in the signature of "String.append : String → String → String" doesn't have a hover.
-
Twice now, I've run into situations where the maximum resident set size has spiked due to increased compilation of one declaration.
#6998 and #6499 with Zulip threads
https://leanprover.zulipchat.…
-
-
The `lakefile.lean` currently links against hardcoded system libraries. This works fine for examples and tests, but only when they are executed with `lake exe `.
Libraries depending on `CTypes` als…
-
### 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
* …