Skip to content

Commit a098d27

Browse files
committed
feat: theorems about power of twos (#8547)
These were factored out of #5920 as they seem generally useful.
1 parent 3c14836 commit a098d27

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

Mathlib/Data/Nat/Pow.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -71,6 +71,10 @@ theorem one_lt_pow (n m : ℕ) (h₀ : 0 < n) (h₁ : 1 < m) : 1 < m ^ n := by
7171
exact pow_lt_pow_of_lt_left h₁ h₀
7272
#align nat.one_lt_pow Nat.one_lt_pow
7373

74+
theorem two_pow_pos (n : ℕ) : 0 < 2^n := Nat.pos_pow_of_pos _ (by decide)
75+
76+
theorem two_pow_succ (n : ℕ) : 2^(n + 1) = 2^n + 2^n := by simp [pow_succ, mul_two]
77+
7478
theorem one_lt_pow' (n m : ℕ) : 1 < (m + 2) ^ (n + 1) :=
7579
one_lt_pow (n + 1) (m + 2) (succ_pos n) (Nat.lt_of_sub_eq_succ rfl)
7680
#align nat.one_lt_pow' Nat.one_lt_pow'

0 commit comments

Comments
 (0)