You cannot select more than 25 topics Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
lean4game/server/testgame/TestGame/Levels/Induction/L10_Bernoulli.lean

47 lines
764 B
Plaintext

2 years ago
import TestGame.Metadata
import Mathlib.Tactic.Ring
import Mathlib
2 years ago
import TestGame.ToBePorted
2 years ago
Game "TestGame"
World "Induction"
2 years ago
Level 5
2 years ago
2 years ago
Title "Bernoulli Ungleichung"
2 years ago
Introduction
"
TODO: Induktion (& induktion vs rcases)
"
2 years ago
example (x : ) (n : ) : 1 + n * x ≤ (x + 1) ^ n := by
induction' n with n hn
simp
rw [Nat.succ_mul]
rw [Nat.pow_succ]
sorry
2 years ago
2 years ago
example (n : ) : (∑ i : Fin (n + 1), ↑(2 * i - 1)) = n ^ 2 := by
induction' n with n hn
2 years ago
simp
2 years ago
2 years ago
Statement
"Zeige $\\sum_{i = 0}^n i = \\frac{n ⬝ (n + 1)}{2}$."
(n : ) : (∑ i : Fin (n + 1), ↑i) = n * (n + 1) / 2 := by
apply hh1
induction' n with n hn
simp
sorry
-- rw [Fin.sum_univ_castSucc]
-- simp [nat_succ]
-- rw [mul_add, hn]
-- ring
Tactics ring