-
Zulip https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/sqrt.204.20.3D.202
-
例が Zulip に載っている。現在は全ビルダーを網羅できていないので追加したい
Zulip: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/lattice.20tactics
-
Report by the Lean FRO:
I am observing a possible bug with lean4web: If I am open, for example, https://lean.math.hhu.de/#project=nightly&codez=M4EwZkA
and look at the network tab of the Firefox d…
-
```
example (h : z = 42) (x y : Nat) : y + 0 = y := by
conv =>
lhs
tactic => clear h -- tactic 'clear' failed, target depends on 'h'
simp
```
This showed up when trying to make …
bollu updated
1 month ago
-
Zulip: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Should.20these.20surds.20be.20simplified.20with.20norm_num.3F
-
https://leanprover-community.github.io/index.html
- https://github.com/leanprover-community/lean-client-python
- https://github.com/leanprover-community/mathlib/blob/master/scripts/polyrith_sage.p…
-
ほしい
-
I would like to do the "Robo" section, which is in German.
I tried Google Chrome's Translate feature as well as [Google Translate](https://translate.google.com/?sl=de&tl=en&op=websites) and [Yandex](…
-
It would be good to forward-port the features from:
* [x] https://github.com/leanprover-community/doc-gen/pull/172
Instance lists for builtin types, like we already have for inductive types
* [ ]…
-
Classifies porting notes claiming `was simp`.
### Examples
https://github.com/leanprover-community/mathlib4/blob/21472664c54bb6e7fe4a120aefa52cf212be8d7c/Mathlib/Algebra/Lie/Engel.lean#L175-L18…