2014-11-14 19:22:51 +00:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2014 Jeremy Avigad. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
|
|
|
|
|
Module: algebra.ring
|
|
|
|
|
Authors: Jeremy Avigad, Leonardo de Moura
|
|
|
|
|
|
|
|
|
|
Structures with multiplicative and additive components, including semirings, rings, and fields.
|
|
|
|
|
The development is modeled after Isabelle's library.
|
|
|
|
|
-/
|
|
|
|
|
|
2014-12-12 21:20:27 +00:00
|
|
|
|
import logic.eq logic.connectives data.unit data.sigma data.prod
|
2014-11-14 19:22:51 +00:00
|
|
|
|
import algebra.function algebra.binary algebra.group
|
|
|
|
|
open eq eq.ops
|
|
|
|
|
|
|
|
|
|
namespace algebra
|
|
|
|
|
|
|
|
|
|
variable {A : Type}
|
|
|
|
|
|
|
|
|
|
/- auxiliary classes -/
|
|
|
|
|
|
|
|
|
|
structure distrib [class] (A : Type) extends has_mul A, has_add A :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
(left_distrib : ∀a b c, mul a (add b c) = add (mul a b) (mul a c))
|
|
|
|
|
(right_distrib : ∀a b c, mul (add a b) c = add (mul a c) (mul b c))
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem left_distrib [s : distrib A] (a b c : A) : a * (b + c) = a * b + a * c :=
|
|
|
|
|
!distrib.left_distrib
|
|
|
|
|
|
|
|
|
|
theorem right_distrib [s: distrib A] (a b c : A) : (a + b) * c = a * c + b * c :=
|
|
|
|
|
!distrib.right_distrib
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-23 22:34:16 +00:00
|
|
|
|
structure mul_zero_class [class] (A : Type) extends has_mul A, has_zero A :=
|
|
|
|
|
(zero_mul : ∀a, mul zero a = zero)
|
|
|
|
|
(mul_zero : ∀a, mul a zero = zero)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-23 22:34:16 +00:00
|
|
|
|
theorem zero_mul [s : mul_zero_class A] (a : A) : 0 * a = 0 := !mul_zero_class.zero_mul
|
|
|
|
|
theorem mul_zero [s : mul_zero_class A] (a : A) : a * 0 = 0 := !mul_zero_class.mul_zero
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
|
|
|
|
structure zero_ne_one_class [class] (A : Type) extends has_zero A, has_one A :=
|
|
|
|
|
(zero_ne_one : zero ≠ one)
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem zero_ne_one [s: zero_ne_one_class A] : 0 ≠ 1 := @zero_ne_one_class.zero_ne_one A s
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
|
|
|
|
/- semiring -/
|
2014-12-12 23:22:19 +00:00
|
|
|
|
|
2014-12-23 22:34:16 +00:00
|
|
|
|
structure semiring [class] (A : Type) extends add_comm_monoid A, monoid A, distrib A,
|
|
|
|
|
mul_zero_class A, zero_ne_one_class A
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-22 19:21:22 +00:00
|
|
|
|
section semiring
|
|
|
|
|
variables [s : semiring A] (a b c : A)
|
|
|
|
|
include s
|
|
|
|
|
|
|
|
|
|
theorem ne_zero_of_mul_ne_zero_right {a b : A} (H : a * b ≠ 0) : a ≠ 0 :=
|
|
|
|
|
assume H1 : a = 0,
|
2014-12-23 22:34:16 +00:00
|
|
|
|
have H2 : a * b = 0, from H1⁻¹ ▸ zero_mul b,
|
2014-12-22 19:21:22 +00:00
|
|
|
|
H H2
|
|
|
|
|
|
|
|
|
|
theorem ne_zero_of_mul_ne_zero_left {a b : A} (H : a * b ≠ 0) : b ≠ 0 :=
|
|
|
|
|
assume H1 : b = 0,
|
2014-12-23 22:34:16 +00:00
|
|
|
|
have H2 : a * b = 0, from H1⁻¹ ▸ mul_zero a,
|
2014-12-22 19:21:22 +00:00
|
|
|
|
H H2
|
|
|
|
|
end semiring
|
|
|
|
|
|
|
|
|
|
/- comm semiring -/
|
|
|
|
|
|
2014-11-14 19:22:51 +00:00
|
|
|
|
structure comm_semiring [class] (A : Type) extends semiring A, comm_semigroup A
|
2014-12-26 21:25:05 +00:00
|
|
|
|
-- TODO: we could also define a cancelative comm_semiring, i.e. satisfying
|
|
|
|
|
-- c ≠ 0 → c * a = c * b → a = b.
|
2014-12-12 23:22:19 +00:00
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
section comm_semiring
|
|
|
|
|
variables [s : comm_semiring A] (a b c : A)
|
|
|
|
|
include s
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
definition dvd (a b : A) : Prop := ∃c, a * c = b
|
|
|
|
|
infix `|` := dvd
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
theorem dvd.intro {a b c : A} (H : a * b = c) : a | c :=
|
|
|
|
|
exists.intro _ H
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-26 21:25:05 +00:00
|
|
|
|
theorem dvd.intro_right {a b c : A} (H : a * b = c) : b | c :=
|
|
|
|
|
dvd.intro (!mul.comm ▸ H)
|
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
theorem dvd.ex {a b : A} (H : a | b) : ∃c, a * c = b := H
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
theorem dvd.elim {P : Prop} {a b : A} (H₁ : a | b) (H₂ : ∀c, a * c = b → P) : P :=
|
|
|
|
|
exists.elim H₁ H₂
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-24 02:14:19 +00:00
|
|
|
|
theorem dvd.refl : a | a := dvd.intro !mul_one
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd.trans {a b c : A} (H₁ : a | b) (H₂ : b | c) : a | c :=
|
|
|
|
|
dvd.elim H₁
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take d, assume H₃ : a * d = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim H₂
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take e, assume H₄ : b * e = c,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
@dvd.intro _ _ _ (d * e) _
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * (d * e) = (a * d) * e : mul.assoc
|
2014-11-14 19:22:51 +00:00
|
|
|
|
... = b * e : H₃
|
|
|
|
|
... = c : H₄)))
|
|
|
|
|
|
2014-12-24 00:46:48 +00:00
|
|
|
|
theorem eq_zero_of_zero_dvd {a : A} (H : 0 | a) : a = 0 :=
|
2014-12-23 22:34:16 +00:00
|
|
|
|
dvd.elim H (take c, assume H' : 0 * c = a, (H')⁻¹ ⬝ !zero_mul)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-23 22:34:16 +00:00
|
|
|
|
theorem dvd_zero : a | 0 := dvd.intro !mul_zero
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-12-24 02:14:19 +00:00
|
|
|
|
theorem one_dvd : 1 | a := dvd.intro !one_mul
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_mul_right : a | a * b := dvd.intro rfl
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_mul_left : a | b * a := mul.comm a b ▸ dvd_mul_right a b
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_mul_of_dvd_left {a b : A} (H : a | b) (c : A) : a | b * c :=
|
|
|
|
|
dvd.elim H
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take d,
|
|
|
|
|
assume H₁ : a * d = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * (d * c) = a * d * c : (!mul.assoc)⁻¹
|
2014-11-14 19:22:51 +00:00
|
|
|
|
... = b * c : H₁))
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_mul_of_dvd_right {a b : A} (H : a | b) (c : A) : a | c * b :=
|
|
|
|
|
!mul.comm ▸ (dvd_mul_of_dvd_left H _)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_dvd_mul {a b c d : A} (dvd_ab : a | b) (dvd_cd : c | d) : a * c | b * d :=
|
|
|
|
|
dvd.elim dvd_ab
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take e, assume Haeb : a * e = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim dvd_cd
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take f, assume Hcfd : c * f = d,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * c * (e * f) = a * (c * (e * f)) : mul.assoc
|
|
|
|
|
... = a * (e * (c * f)) : mul.left_comm
|
|
|
|
|
... = a * e * (c * f) : (!mul.assoc)⁻¹
|
2014-11-14 19:22:51 +00:00
|
|
|
|
... = b * (c * f) : Haeb
|
|
|
|
|
... = b * d : Hcfd)))
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_of_mul_right_dvd {a b c : A} (H : a * b | c) : a | c :=
|
|
|
|
|
dvd.elim H (take d, assume Habdc : a * b * d = c, dvd.intro (!mul.assoc⁻¹ ⬝ Habdc))
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_of_mul_left_dvd {a b c : A} (H : a * b | c) : b | c :=
|
|
|
|
|
dvd_of_mul_right_dvd (mul.comm a b ▸ H)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
|
|
|
|
theorem dvd_add {a b c : A} (Hab : a | b) (Hac : a | c) : a | b + c :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim Hab
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take d, assume Hadb : a * d = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim Hac
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(take e, assume Haec : a * e = c,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro (show a * (d + e) = b + c, from Hadb ▸ Haec ▸ left_distrib a d e)))
|
2014-12-22 17:21:53 +00:00
|
|
|
|
end comm_semiring
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
|
|
|
|
/- ring -/
|
|
|
|
|
|
|
|
|
|
structure ring [class] (A : Type) extends add_comm_group A, monoid A, distrib A, zero_ne_one_class A
|
|
|
|
|
|
2014-12-26 21:25:05 +00:00
|
|
|
|
definition ring.to_semiring [instance] [coercion] [s : ring A] : semiring A :=
|
2015-01-17 01:42:30 +00:00
|
|
|
|
⦃ semiring,
|
|
|
|
|
mul_zero := take a,
|
2014-11-14 19:22:51 +00:00
|
|
|
|
have H : a * 0 + 0 = a * 0 + a * 0, from
|
|
|
|
|
calc
|
2014-12-24 02:14:19 +00:00
|
|
|
|
a * 0 + 0 = a * 0 : add_zero
|
|
|
|
|
... = a * (0 + 0) : {(add_zero 0)⁻¹}
|
2014-11-30 13:31:34 +00:00
|
|
|
|
... = a * 0 + a * 0 : ring.left_distrib,
|
2015-01-17 01:42:30 +00:00
|
|
|
|
show a * 0 = 0, from (add.left_cancel H)⁻¹,
|
|
|
|
|
zero_mul := take a,
|
|
|
|
|
have H : 0 * a + 0 = 0 * a + 0 * a, from
|
|
|
|
|
calc
|
|
|
|
|
0 * a + 0 = 0 * a : add_zero
|
|
|
|
|
... = (0 + 0) * a : {(add_zero 0)⁻¹}
|
|
|
|
|
... = 0 * a + 0 * a : ring.right_distrib,
|
|
|
|
|
show 0 * a = 0, from (add.left_cancel H)⁻¹,
|
|
|
|
|
using s ⦄
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
|
|
|
|
section
|
2014-11-17 20:19:46 +00:00
|
|
|
|
variables [s : ring A] (a b c d e : A)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
include s
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem neg_mul_eq_neg_mul : -(a * b) = -a * b :=
|
|
|
|
|
neg_eq_of_add_eq_zero
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * b + -a * b = (a + -a) * b : right_distrib
|
|
|
|
|
... = 0 * b : add.right_inv
|
2014-12-23 22:34:16 +00:00
|
|
|
|
... = 0 : zero_mul)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem neg_mul_eq_mul_neg : -(a * b) = a * -b :=
|
|
|
|
|
neg_eq_of_add_eq_zero
|
2014-11-14 19:22:51 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * b + a * -b = a * (b + -b) : left_distrib
|
|
|
|
|
... = a * 0 : add.right_inv
|
2014-12-23 22:34:16 +00:00
|
|
|
|
... = 0 : mul_zero)
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem neg_mul_neg_eq : -a * -b = a * b :=
|
2014-11-14 19:22:51 +00:00
|
|
|
|
calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
-a * -b = -(a * -b) : !neg_mul_eq_neg_mul⁻¹
|
|
|
|
|
... = - -(a * b) : neg_mul_eq_mul_neg
|
2014-12-17 18:32:38 +00:00
|
|
|
|
... = a * b : neg_neg
|
2014-11-14 19:22:51 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem neg_mul_comm : -a * b = a * -b := !neg_mul_eq_neg_mul⁻¹ ⬝ !neg_mul_eq_mul_neg
|
2014-11-17 20:19:46 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_sub_left_distrib : a * (b - c) = a * b - a * c :=
|
2014-11-17 20:19:46 +00:00
|
|
|
|
calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * (b - c) = a * b + a * -c : left_distrib
|
|
|
|
|
... = a * b + - (a * c) : {!neg_mul_eq_mul_neg⁻¹}
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = a * b - a * c : rfl
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_sub_right_distrib : (a - b) * c = a * c - b * c :=
|
2014-11-17 20:19:46 +00:00
|
|
|
|
calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
(a - b) * c = a * c + -b * c : right_distrib
|
|
|
|
|
... = a * c + - (b * c) : {!neg_mul_eq_neg_mul⁻¹}
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = a * c - b * c : rfl
|
|
|
|
|
|
|
|
|
|
-- TODO: can calc mode be improved to make this easier?
|
|
|
|
|
-- TODO: there is also the other direction. It will be easier when we
|
|
|
|
|
-- have the simplifier.
|
2014-11-30 13:31:34 +00:00
|
|
|
|
|
|
|
|
|
theorem mul_add_eq_mul_add_iff_sub_mul_add_eq : a * e + c = b * e + d ↔ (a - b) * e + c = d :=
|
2014-11-17 20:19:46 +00:00
|
|
|
|
calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * e + c = b * e + d ↔ a * e + c = d + b * e : !add.comm ▸ !iff.refl
|
|
|
|
|
... ↔ a * e + c - b * e = d : iff.symm !sub_eq_iff_eq_add
|
|
|
|
|
... ↔ a * e - b * e + c = d : !sub_add_eq_add_sub ▸ !iff.refl
|
|
|
|
|
... ↔ (a - b) * e + c = d : !mul_sub_right_distrib ▸ !iff.refl
|
2014-11-14 19:22:51 +00:00
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
structure comm_ring [class] (A : Type) extends ring A, comm_semigroup A
|
|
|
|
|
|
2014-12-26 21:25:05 +00:00
|
|
|
|
definition comm_ring.to_comm_semiring [instance] [coercion] [s : comm_ring A] : comm_semiring A :=
|
2015-01-17 01:42:30 +00:00
|
|
|
|
⦃ comm_semiring,
|
|
|
|
|
mul_zero := mul_zero,
|
|
|
|
|
zero_mul := zero_mul,
|
|
|
|
|
using s ⦄
|
2014-11-17 20:19:46 +00:00
|
|
|
|
|
|
|
|
|
section
|
|
|
|
|
variables [s : comm_ring A] (a b c d e : A)
|
|
|
|
|
include s
|
|
|
|
|
|
|
|
|
|
-- TODO: wait for the simplifier
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_self_sub_mul_self_eq : a * a - b * b = (a + b) * (a - b) := sorry
|
2014-11-17 20:19:46 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_self_sub_one_eq : a * a - 1 = (a + 1) * (a - 1) :=
|
2014-12-24 02:14:19 +00:00
|
|
|
|
mul_one 1 ▸ mul_self_sub_mul_self_eq a 1
|
2014-11-17 20:19:46 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem dvd_neg_iff_dvd : a | -b ↔ a | b :=
|
2014-11-17 20:19:46 +00:00
|
|
|
|
iff.intro
|
|
|
|
|
(assume H : a | -b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim H
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(take c, assume H' : a * c = -b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * -c = -(a * c) : {!neg_mul_eq_mul_neg⁻¹}
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = -(-b) : H'
|
2014-12-17 18:32:38 +00:00
|
|
|
|
... = b : neg_neg)))
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(assume H : a | b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim H
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(take c, assume H' : a * c = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * -c = -(a * c) : {!neg_mul_eq_mul_neg⁻¹}
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = -b : H')))
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem neg_dvd_iff_dvd : -a | b ↔ a | b :=
|
2014-11-17 20:19:46 +00:00
|
|
|
|
iff.intro
|
|
|
|
|
(assume H : -a | b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim H
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(take c, assume H' : -a * c = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
a * -c = -a * c : !neg_mul_comm⁻¹
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = b : H')))
|
|
|
|
|
(assume H : a | b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim H
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(take c, assume H' : a * c = b,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro
|
2014-11-17 20:19:46 +00:00
|
|
|
|
(calc
|
2014-11-30 13:31:34 +00:00
|
|
|
|
-a * -c = a * c : neg_mul_neg_eq
|
2014-11-17 20:19:46 +00:00
|
|
|
|
... = b : H')))
|
|
|
|
|
|
2014-12-22 19:21:22 +00:00
|
|
|
|
theorem dvd_sub (H₁ : a | b) (H₂ : a | c) : a | (b - c) :=
|
|
|
|
|
dvd_add H₁ (iff.elim_right !dvd_neg_iff_dvd H₂)
|
2014-11-17 20:19:46 +00:00
|
|
|
|
end
|
|
|
|
|
|
2014-11-26 23:08:23 +00:00
|
|
|
|
/- integral domains -/
|
|
|
|
|
|
|
|
|
|
structure no_zero_divisors [class] (A : Type) extends has_mul A, has_zero A :=
|
|
|
|
|
(eq_zero_or_eq_zero_of_mul_eq_zero : ∀a b, mul a b = zero → a = zero ∨ b = zero)
|
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem eq_zero_or_eq_zero_of_mul_eq_zero {A : Type} [s : no_zero_divisors A] {a b : A}
|
|
|
|
|
(H : a * b = 0) :
|
2014-11-26 23:08:23 +00:00
|
|
|
|
a = 0 ∨ b = 0 := !no_zero_divisors.eq_zero_or_eq_zero_of_mul_eq_zero H
|
|
|
|
|
|
2014-12-22 17:21:53 +00:00
|
|
|
|
structure integral_domain [class] (A : Type) extends comm_ring A, no_zero_divisors A
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
|
|
|
|
section
|
|
|
|
|
|
|
|
|
|
variables [s : integral_domain A] (a b c d e : A)
|
|
|
|
|
include s
|
|
|
|
|
|
2014-12-22 19:21:22 +00:00
|
|
|
|
theorem mul_ne_zero {a b : A} (H1 : a ≠ 0) (H2 : b ≠ 0) : a * b ≠ 0 :=
|
2014-11-26 23:08:23 +00:00
|
|
|
|
assume H : a * b = 0,
|
|
|
|
|
or.elim (eq_zero_or_eq_zero_of_mul_eq_zero H) (assume H3, H1 H3) (assume H4, H2 H4)
|
|
|
|
|
|
|
|
|
|
theorem mul.cancel_right {a b c : A} (Ha : a ≠ 0) (H : b * a = c * a) : b = c :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
have H1 : b * a - c * a = 0, from iff.mp !eq_iff_sub_eq_zero H,
|
|
|
|
|
have H2 : (b - c) * a = 0, from eq.trans !mul_sub_right_distrib H1,
|
2014-12-15 20:05:44 +00:00
|
|
|
|
have H3 : b - c = 0, from or_resolve_left (eq_zero_or_eq_zero_of_mul_eq_zero H2) Ha,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
iff.elim_right !eq_iff_sub_eq_zero H3
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
|
|
|
|
theorem mul.cancel_left {a b c : A} (Ha : a ≠ 0) (H : a * b = a * c) : b = c :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
have H1 : a * b - a * c = 0, from iff.mp !eq_iff_sub_eq_zero H,
|
|
|
|
|
have H2 : a * (b - c) = 0, from eq.trans !mul_sub_left_distrib H1,
|
2014-12-15 20:05:44 +00:00
|
|
|
|
have H3 : b - c = 0, from or_resolve_right (eq_zero_or_eq_zero_of_mul_eq_zero H2) Ha,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
iff.elim_right !eq_iff_sub_eq_zero H3
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
|
|
|
|
-- TODO: do we want the iff versions?
|
|
|
|
|
|
|
|
|
|
-- TODO: wait for simplifier
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_self_eq_mul_self_iff (a b : A) : a * a = b * b ↔ a = b ∨ a = -b := sorry
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
2014-11-30 13:31:34 +00:00
|
|
|
|
theorem mul_self_eq_one_iff (a : A) : a * a = 1 ↔ a = 1 ∨ a = -1 := sorry
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
|
|
|
|
-- TODO: c - b * c → c = 0 ∨ b = 1 and variants
|
|
|
|
|
|
|
|
|
|
theorem dvd_of_mul_dvd_mul_left {a b c : A} (Ha : a ≠ 0) (Hdvd : a * b | a * c) : b | c :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim Hdvd
|
2014-11-26 23:08:23 +00:00
|
|
|
|
(take d,
|
|
|
|
|
assume H : a * b * d = a * c,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
have H1 : b * d = c, from mul.cancel_left Ha (mul.assoc a b d ▸ H),
|
|
|
|
|
dvd.intro H1)
|
2014-11-26 23:08:23 +00:00
|
|
|
|
|
|
|
|
|
theorem dvd_of_mul_dvd_mul_right {a b c : A} (Ha : a ≠ 0) (Hdvd : b * a | c * a) : b | c :=
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.elim Hdvd
|
2014-11-26 23:08:23 +00:00
|
|
|
|
(take d,
|
|
|
|
|
assume H : b * a * d = c * a,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
have H1 : b * d * a = c * a, from eq.trans !mul.right_comm H,
|
2014-11-26 23:08:23 +00:00
|
|
|
|
have H2 : b * d = c, from mul.cancel_right Ha H1,
|
2014-11-30 13:31:34 +00:00
|
|
|
|
dvd.intro H2)
|
2014-11-26 23:08:23 +00:00
|
|
|
|
end
|
2014-11-17 20:19:46 +00:00
|
|
|
|
|
2014-11-14 19:22:51 +00:00
|
|
|
|
end algebra
|