-
```lean
import Mathlib.Tactic
-- `2 - n < 0` となることはありえないので、この仮定は偽で、
-- 偽の仮定があるから証明が通ってしまう。
theorem Fermat (x y z n : ℕ) (h1 : 2 - n < 0) : (x * y * z ≠ 0) → x ^ n + y ^ n ≠ z ^ n := by
omega
…
-
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
…
-
```lean
import Mathlib.Tactic
example {n : Nat} (h : 3 ∣ n + 4) : 3 ∣ n + 1 := by
norm_num at h
assumption
```
-
Nat.isPrime を Decidableにする
-
你好,首先非常感谢这个非常棒的开源工程的工作!我在按照安装说明安装好依赖和mathlib后,执行quick_start.py,但是并没有得到预期结果,NN模型有正确输出结果,但是lean4的验证有问题。
python quick_start.py
Special tokens have been added in the vocabulary, make sure the associated…
-
```lean
import Mathlib.Tactic
theorem foo (n : ℕ) (h₀ : 0 < n) :
(∏ x ∈ Finset.Ico 1 (n + 1), x * (x + 1) : ℤ) ∣
∏ x ∈ Finset.Ico 1 (n + 1), 1 := by
induction id h₀ with
| refl =…
-
```lean
import Mathlib.Data.Fin.VecNotation
open Lean
partial def matchVecLit (e : Expr) : Option (List Expr) :=
match_expr e with
| Matrix.vecEmpty _ => some []
| Matrix.vecCons _ _ x…
-
```lean
import Mathlib.Tactic.Lift
abbrev MyNat := ℕ
example (n : ℤ) (hn : n ≥ 0) : True := by
lift n to MyNat using hn
-- type of `n` is `ℕ` instead of `MyNat`, in the goal state
triv…
-
I was trying to execute the following theorem via REPL:
```
theorem ftaylorSeriesWithin_univ : ftaylorSeriesWithin 𝕜 f univ = ftaylorSeries 𝕜 f := by sorry
```
.This theorem can be found in Mathli…
-
# Handle
byterocket
# Vulnerability details
## Impact
Issue Information: [G008](https://github.com/byterocket/c4-common-issues/blob/main/0-Gas-Optimizations.md#g008---shift-right-instead-of-divid…