Skip to content

Commit

Permalink
chore: rm @[simp] from factorial_succ (#6840)
Browse files Browse the repository at this point in the history
Co-authored-by: Moritz Firsching <firsching@google.com>
  • Loading branch information
mo271 and mo271 committed Aug 30, 2023
1 parent c83178f commit e8477a9
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 2 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Complex/Exponential.lean
Expand Up @@ -1596,7 +1596,7 @@ theorem sum_div_factorial_le {α : Type*} [LinearOrderedField α] (n j : ℕ) (h
· rw [← Nat.cast_pow, ← Nat.cast_mul, Nat.cast_le, add_comm]
exact Nat.factorial_mul_pow_le_factorial
_ = (n.factorial : α)⁻¹ * ∑ m in range (j - n), (n.succ : α)⁻¹ ^ m := by
simp [mul_inv, mul_sum.symm, sum_mul.symm, -Nat.factorial_succ, mul_comm, inv_pow]
simp [mul_inv, mul_sum.symm, sum_mul.symm, mul_comm, inv_pow]
_ = ((n.succ : α) - n.succ * (n.succ : α)⁻¹ ^ (j - n)) / (n.factorial * n) := by
have h₁ : (n.succ : α) ≠ 1 :=
@Nat.cast_one α _ ▸ mt Nat.cast_inj.1 (mt Nat.succ.inj (pos_iff_ne_zero.1 hn))
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/Nat/Factorial/Basic.lean
Expand Up @@ -44,7 +44,6 @@ theorem factorial_zero : 0! = 1 :=
rfl
#align nat.factorial_zero Nat.factorial_zero

@[simp]
theorem factorial_succ (n : ℕ) : n.succ ! = (n + 1) * n ! :=
rfl
#align nat.factorial_succ Nat.factorial_succ
Expand Down

0 comments on commit e8477a9

Please sign in to comment.