-
Many of the theorem statements does not have formal proofs(they have the sorry tags). If I have a generated proof for a theorem how should I evaluate it, even if we have a predicted proof and ground t…
-
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 the MWE:
```lean
def fails : MetaM Unit := do
let mut val : Bool ← do
pure true
-- unknown identifier val
val := Bool.not val -- FAILS! expected to succeed.
return ()
…
bollu updated
1 month ago
-
Discussed in https://leanprover.zulipchat.com/#narrow/stream/458659-Equational/topic/visualization.20of.20graph.20closure . Let k denote the number of variables in a law. As discussed above, the k=1…
-
Zulip https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Why.20can't.20.60rw.60.20rewrite.20under.20binders.3F
-
See https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Dynamics/Minimal.lean
Our minimal sets need to be extended to action and topological spaces
mseri updated
5 months ago
-
Egg can generate dot/svg/png-files for its e-graphs. Try using the `proofwidgets` package to display this in the info-view.
-
### 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
* …
-
### Prerequisites
Please put an X between the brackets as you perform the following steps:
* [ ] Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues
* …
-
I want to set the option `autoImplicit` to false in a project on my self host server. My `mathlib-demo/lakefile.lean` is as follows:
```
import Lake
open Lake DSL
package "MathlibLatest" where
…