-
Guys, I read the guide to contribute to the mathlib, https://leanprover-community.github.io/contribute/index.html
And in summary, here is what we need to do :
- [ ] discuss on Zulip chat : https://l…
-
### 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
* …
-
LeanInk is sensitive to Lean versions and expected to be installed locally, it's useful to support specifying the LeanInk path via a flag like `--leanink=` in such scenarios.
A similar flag (but as…
-
-
`decidable.to_bool` is `export`ed out of `decidable` [here](https://github.com/leanprover-community/lean/blob/4c40c41/library/init/logic.lean#L597), however, https://leanprover-community.github.io/mat…
-
```lean
open Lean Elab Command
elab "private section" ppLine cmd:command* ppLine "end private section": command => do
let old ← get
try
for cmd in cmd do
elabCommandTopLevel cmd
…
-
Could someone point me to the code that is responsible for generating https://leanprover-community.github.io/archive/ ?
srid updated
7 months ago
-
ただし,Lean by Example でいま紹介している例は `priority` を指定してもなぜかエラーになる
```lean
-- 排他的論理和の記号を定義
infix:60 (priority := high) " ⊕ " => xor
#check_failure true ⊕ true = false
```
-
see: https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/what.20is.20.60class.60.20attribute/near/445581181
MIL の7章に記述があるものの,ただの構造体との違いがわからない
-
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…