We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 3c14836 commit a098d27Copy full SHA for a098d27
Mathlib/Data/Nat/Pow.lean
@@ -71,6 +71,10 @@ theorem one_lt_pow (n m : ℕ) (h₀ : 0 < n) (h₁ : 1 < m) : 1 < m ^ n := by
71
exact pow_lt_pow_of_lt_left h₁ h₀
72
#align nat.one_lt_pow Nat.one_lt_pow
73
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
78
theorem one_lt_pow' (n m : ℕ) : 1 < (m + 2) ^ (n + 1) :=
79
one_lt_pow (n + 1) (m + 2) (succ_pos n) (Nat.lt_of_sub_eq_succ rfl)
80
#align nat.one_lt_pow' Nat.one_lt_pow'
0 commit comments