2015-04-14 15:56:59 +00:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2015 Microsoft Corporation. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
2015-05-14 04:48:32 +00:00
|
|
|
|
Authors: Leonardo de Moura, Jeremy Avigad
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
2015-05-14 04:48:32 +00:00
|
|
|
|
The power function on the natural numbers.
|
2015-04-14 15:56:59 +00:00
|
|
|
|
-/
|
2015-07-08 01:27:55 +00:00
|
|
|
|
import data.nat.basic data.nat.order data.nat.div data.nat.gcd algebra.ring_power
|
2015-10-08 18:01:57 +00:00
|
|
|
|
open - [notations] algebra
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
|
|
|
|
namespace nat
|
|
|
|
|
|
2015-10-09 19:47:55 +00:00
|
|
|
|
definition nat_has_pow_nat [instance] [reducible] [priority nat.prio] : has_pow_nat nat :=
|
|
|
|
|
has_pow_nat.mk has_pow_nat.pow_nat
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
2015-10-08 18:01:57 +00:00
|
|
|
|
theorem pow_le_pow_of_le {x y : ℕ} (i : ℕ) (H : x ≤ y) : x^i ≤ y^i :=
|
|
|
|
|
algebra.pow_le_pow_of_le i !zero_le H
|
2015-05-23 05:38:42 +00:00
|
|
|
|
|
2015-08-17 03:23:03 +00:00
|
|
|
|
theorem eq_zero_of_pow_eq_zero {a m : ℕ} (H : a^m = 0) : a = 0 :=
|
|
|
|
|
or.elim (eq_zero_or_pos m)
|
|
|
|
|
(suppose m = 0,
|
2015-10-09 19:47:55 +00:00
|
|
|
|
by krewrite [`m = 0` at H, pow_zero at H]; contradiction)
|
2015-08-17 03:23:03 +00:00
|
|
|
|
(suppose m > 0,
|
|
|
|
|
have h₁ : ∀ m, a^succ m = 0 → a = 0,
|
|
|
|
|
begin
|
|
|
|
|
intro m,
|
|
|
|
|
induction m with m ih,
|
2015-10-09 19:47:55 +00:00
|
|
|
|
{krewrite pow_one; intros; assumption},
|
2015-08-17 03:23:03 +00:00
|
|
|
|
rewrite pow_succ,
|
|
|
|
|
intro H,
|
|
|
|
|
cases eq_zero_or_eq_zero_of_mul_eq_zero H with h₃ h₄,
|
|
|
|
|
assumption,
|
|
|
|
|
exact ih h₄
|
|
|
|
|
end,
|
|
|
|
|
obtain m' (h₂ : m = succ m'), from exists_eq_succ_of_pos `m > 0`,
|
|
|
|
|
show a = 0, by rewrite h₂ at H; apply h₁ m' H)
|
|
|
|
|
|
2015-07-08 01:27:55 +00:00
|
|
|
|
-- generalize to semirings?
|
|
|
|
|
theorem le_pow_self {x : ℕ} (H : x > 1) : ∀ i, i ≤ x^i
|
|
|
|
|
| 0 := !zero_le
|
2015-10-08 18:01:57 +00:00
|
|
|
|
| (succ j) := have x > 0, from lt.trans zero_lt_one H,
|
|
|
|
|
have h₁ : x^j ≥ 1, from succ_le_of_lt (pow_pos_of_pos _ this),
|
|
|
|
|
have x ≥ 2, from succ_le_of_lt H,
|
2015-07-08 01:27:55 +00:00
|
|
|
|
calc
|
|
|
|
|
succ j = j + 1 : rfl
|
|
|
|
|
... ≤ x^j + 1 : add_le_add_right (le_pow_self j)
|
2015-10-08 18:01:57 +00:00
|
|
|
|
... ≤ x^j + x^j : add_le_add_left h₁
|
2015-07-08 01:27:55 +00:00
|
|
|
|
... = x^j * (1 + 1) : by rewrite [mul.left_distrib, *mul_one]
|
|
|
|
|
... = x^j * 2 : rfl
|
2015-07-22 20:41:50 +00:00
|
|
|
|
... ≤ x^j * x : mul_le_mul_left _ `x ≥ 2`
|
2015-08-14 15:00:16 +00:00
|
|
|
|
... = x^(succ j) : pow_succ'
|
2015-07-08 01:27:55 +00:00
|
|
|
|
|
2015-05-14 04:48:32 +00:00
|
|
|
|
-- TODO: eventually this will be subsumed under the algebraic theorems
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
2015-10-08 18:01:57 +00:00
|
|
|
|
theorem mul_self_eq_pow_2 (a : nat) : a * a = a ^ 2 :=
|
|
|
|
|
show a * a = a ^ (succ (succ zero)), from
|
|
|
|
|
by krewrite [*pow_succ, *pow_zero, mul_one] -- TODO(Leo): krewrite -> rewrite after new numeral encoding
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
2015-10-08 18:01:57 +00:00
|
|
|
|
theorem pow_cancel_left : ∀ {a b c : nat}, a > 1 → a^b = a^c → b = c
|
2015-04-14 15:56:59 +00:00
|
|
|
|
| a 0 0 h₁ h₂ := rfl
|
|
|
|
|
| a (succ b) 0 h₁ h₂ :=
|
2015-08-14 15:00:16 +00:00
|
|
|
|
assert a = 1, by rewrite [pow_succ at h₂, pow_zero at h₂]; exact (eq_one_of_mul_eq_one_right h₂),
|
2015-07-22 20:41:50 +00:00
|
|
|
|
assert 1 < 1, by rewrite [this at h₁]; exact h₁,
|
|
|
|
|
absurd `1 < 1` !lt.irrefl
|
2015-04-14 15:56:59 +00:00
|
|
|
|
| a 0 (succ c) h₁ h₂ :=
|
2015-08-14 15:00:16 +00:00
|
|
|
|
assert a = 1, by rewrite [pow_succ at h₂, pow_zero at h₂]; exact (eq_one_of_mul_eq_one_right (eq.symm h₂)),
|
2015-07-22 20:41:50 +00:00
|
|
|
|
assert 1 < 1, by rewrite [this at h₁]; exact h₁,
|
|
|
|
|
absurd `1 < 1` !lt.irrefl
|
2015-04-14 15:56:59 +00:00
|
|
|
|
| a (succ b) (succ c) h₁ h₂ :=
|
2015-07-22 20:41:50 +00:00
|
|
|
|
assert a ≠ 0, from assume aeq0, by rewrite [aeq0 at h₁]; exact (absurd h₁ dec_trivial),
|
2015-10-08 18:01:57 +00:00
|
|
|
|
assert a^b = a^c, by rewrite [*pow_succ at h₂]; exact (eq_of_mul_eq_mul_left (pos_of_ne_zero this) h₂),
|
2015-07-22 20:41:50 +00:00
|
|
|
|
by rewrite [pow_cancel_left h₁ this]
|
2015-04-14 15:56:59 +00:00
|
|
|
|
|
2015-10-08 18:01:57 +00:00
|
|
|
|
theorem pow_div_cancel : ∀ {a b : nat}, a ≠ 0 → (a ^ succ b) div a = a ^ b
|
|
|
|
|
-- TODO(Leo): krewrite -> rewrite after new numeral encoding
|
|
|
|
|
| a 0 h := by krewrite [pow_succ, pow_zero, mul_one, div_self (pos_of_ne_zero h)]
|
2015-08-14 15:00:16 +00:00
|
|
|
|
| a (succ b) h := by rewrite [pow_succ, mul_div_cancel_left _ (pos_of_ne_zero h)]
|
2015-07-03 05:27:21 +00:00
|
|
|
|
|
|
|
|
|
lemma dvd_pow : ∀ (i : nat) {n : nat}, n > 0 → i ∣ i^n
|
|
|
|
|
| i 0 h := absurd h !lt.irrefl
|
2015-08-14 15:00:16 +00:00
|
|
|
|
| i (succ n) h := by rewrite [pow_succ']; apply dvd_mul_left
|
2015-07-03 05:27:21 +00:00
|
|
|
|
|
|
|
|
|
lemma dvd_pow_of_dvd_of_pos : ∀ {i j n : nat}, i ∣ j → n > 0 → i ∣ j^n
|
|
|
|
|
| i j 0 h₁ h₂ := absurd h₂ !lt.irrefl
|
2015-08-14 15:00:16 +00:00
|
|
|
|
| i j (succ n) h₁ h₂ := by rewrite [pow_succ']; apply dvd_mul_of_dvd_right h₁
|
2015-07-03 05:27:21 +00:00
|
|
|
|
|
|
|
|
|
lemma pow_mod_eq_zero (i : nat) {n : nat} (h : n > 0) : (i^n) mod i = 0 :=
|
|
|
|
|
iff.mp !dvd_iff_mod_eq_zero (dvd_pow i h)
|
|
|
|
|
|
2015-07-13 21:51:35 +00:00
|
|
|
|
lemma pow_dvd_of_pow_succ_dvd {p i n : nat} : p^(succ i) ∣ n → p^i ∣ n :=
|
2015-07-22 20:41:50 +00:00
|
|
|
|
suppose p^(succ i) ∣ n,
|
2015-08-14 15:00:16 +00:00
|
|
|
|
assert p^i ∣ p^(succ i), from by rewrite [pow_succ']; apply dvd_of_eq_mul; apply rfl,
|
2015-07-22 20:41:50 +00:00
|
|
|
|
dvd.trans `p^i ∣ p^(succ i)` `p^(succ i) ∣ n`
|
2015-07-13 21:51:35 +00:00
|
|
|
|
|
|
|
|
|
lemma dvd_of_pow_succ_dvd_mul_pow {p i n : nat} (Ppos : p > 0) :
|
|
|
|
|
p^(succ i) ∣ (n * p^i) → p ∣ n :=
|
2015-08-14 15:00:16 +00:00
|
|
|
|
by rewrite [pow_succ]; apply dvd_of_mul_dvd_mul_right; apply pow_pos_of_pos _ Ppos
|
2015-07-13 21:51:35 +00:00
|
|
|
|
|
2015-07-04 07:37:09 +00:00
|
|
|
|
lemma coprime_pow_right {a b} : ∀ n, coprime b a → coprime b (a^n)
|
|
|
|
|
| 0 h := !comprime_one_right
|
|
|
|
|
| (succ n) h :=
|
|
|
|
|
begin
|
2015-08-14 15:00:16 +00:00
|
|
|
|
rewrite [pow_succ'],
|
2015-07-04 07:37:09 +00:00
|
|
|
|
apply coprime_mul_right,
|
|
|
|
|
exact coprime_pow_right n h,
|
|
|
|
|
exact h
|
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
lemma coprime_pow_left {a b} : ∀ n, coprime b a → coprime (b^n) a :=
|
2015-07-22 20:41:50 +00:00
|
|
|
|
take n, suppose coprime b a,
|
|
|
|
|
coprime_swap (coprime_pow_right n (coprime_swap this))
|
2015-04-14 15:56:59 +00:00
|
|
|
|
end nat
|