mathlib3 documentation

data.rat.cast

Casts for Rational Numbers #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Summary #

We define the canonical injection from ℚ into an arbitrary division ring and prove various casting lemmas showing the well-behavedness of this injection.

Notations #

Tags #

rat, rationals, field, ℚ, numerator, denominator, num, denom, cast, coercion, casting

@[simp, norm_cast]
theorem rat.cast_coe_int {α : Type u_3} [division_ring α] (n : ) :
@[simp, norm_cast]
theorem rat.cast_coe_nat {α : Type u_3} [division_ring α] (n : ) :
@[simp, norm_cast]
theorem rat.cast_zero {α : Type u_3} [division_ring α] :
0 = 0
@[simp, norm_cast]
theorem rat.cast_one {α : Type u_3} [division_ring α] :
1 = 1
theorem rat.cast_commute {α : Type u_3} [division_ring α] (r : ) (a : α) :
theorem rat.cast_comm {α : Type u_3} [division_ring α] (r : ) (a : α) :
r * a = a * r
theorem rat.commute_cast {α : Type u_3} [division_ring α] (a : α) (r : ) :
@[norm_cast]
theorem rat.cast_mk_of_ne_zero {α : Type u_3} [division_ring α] (a b : ) (b0 : b 0) :
(rat.mk a b) = a / b
@[norm_cast]
theorem rat.cast_add_of_ne_zero {α : Type u_3} [division_ring α] {m n : } :
(m.denom) 0 (n.denom) 0 (m + n) = m + n
@[simp, norm_cast]
theorem rat.cast_neg {α : Type u_3} [division_ring α] (n : ) :
@[norm_cast]
theorem rat.cast_sub_of_ne_zero {α : Type u_3} [division_ring α] {m n : } (m0 : (m.denom) 0) (n0 : (n.denom) 0) :
(m - n) = m - n
@[norm_cast]
theorem rat.cast_mul_of_ne_zero {α : Type u_3} [division_ring α] {m n : } :
(m.denom) 0 (n.denom) 0 (m * n) = m * n
@[simp]
theorem rat.cast_inv_nat {α : Type u_3} [division_ring α] (n : ) :
@[simp]
theorem rat.cast_inv_int {α : Type u_3} [division_ring α] (n : ) :
@[norm_cast]
theorem rat.cast_inv_of_ne_zero {α : Type u_3} [division_ring α] {n : } :
@[norm_cast]
theorem rat.cast_div_of_ne_zero {α : Type u_3} [division_ring α] {m n : } (md : (m.denom) 0) (nn : (n.num) 0) (nd : (n.denom) 0) :
(m / n) = m / n
@[simp, norm_cast]
theorem rat.cast_inj {α : Type u_3} [division_ring α] [char_zero α] {m n : } :
m = n m = n
@[simp]
theorem rat.cast_eq_zero {α : Type u_3} [division_ring α] [char_zero α] {n : } :
n = 0 n = 0
theorem rat.cast_ne_zero {α : Type u_3} [division_ring α] [char_zero α] {n : } :
n 0 n 0
@[simp, norm_cast]
theorem rat.cast_add {α : Type u_3} [division_ring α] [char_zero α] (m n : ) :
(m + n) = m + n
@[simp, norm_cast]
theorem rat.cast_sub {α : Type u_3} [division_ring α] [char_zero α] (m n : ) :
(m - n) = m - n
@[simp, norm_cast]
theorem rat.cast_mul {α : Type u_3} [division_ring α] [char_zero α] (m n : ) :
(m * n) = m * n
@[simp, norm_cast]
theorem rat.cast_bit0 {α : Type u_3} [division_ring α] [char_zero α] (n : ) :
@[simp, norm_cast]
theorem rat.cast_bit1 {α : Type u_3} [division_ring α] [char_zero α] (n : ) :
def rat.cast_hom (α : Type u_3) [division_ring α] [char_zero α] :

Coercion ℚ → α as a ring_hom.

Equations
@[simp]
theorem rat.coe_cast_hom {α : Type u_3} [division_ring α] [char_zero α] :
@[simp, norm_cast]
theorem rat.cast_inv {α : Type u_3} [division_ring α] [char_zero α] (n : ) :
@[simp, norm_cast]
theorem rat.cast_div {α : Type u_3} [division_ring α] [char_zero α] (m n : ) :
(m / n) = m / n
@[simp, norm_cast]
theorem rat.cast_zpow {α : Type u_3} [division_ring α] [char_zero α] (q : ) (n : ) :
(q ^ n) = q ^ n
@[norm_cast]
theorem rat.cast_mk {α : Type u_3} [division_ring α] [char_zero α] (a b : ) :
(rat.mk a b) = a / b
@[simp, norm_cast]
theorem rat.cast_pow {α : Type u_3} [division_ring α] [char_zero α] (q : ) (k : ) :
(q ^ k) = q ^ k
theorem rat.cast_pos_of_pos {K : Type u_5} [linear_ordered_field K] {r : } (hr : 0 < r) :
0 < r
@[simp, norm_cast]
theorem rat.cast_le {K : Type u_5} [linear_ordered_field K] {m n : } :
m n m n
@[simp, norm_cast]
theorem rat.cast_lt {K : Type u_5} [linear_ordered_field K] {m n : } :
m < n m < n
@[simp]
theorem rat.cast_nonneg {K : Type u_5} [linear_ordered_field K] {n : } :
0 n 0 n
@[simp]
theorem rat.cast_nonpos {K : Type u_5} [linear_ordered_field K] {n : } :
n 0 n 0
@[simp]
theorem rat.cast_pos {K : Type u_5} [linear_ordered_field K] {n : } :
0 < n 0 < n
@[simp]
theorem rat.cast_lt_zero {K : Type u_5} [linear_ordered_field K] {n : } :
n < 0 n < 0
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
theorem rat.cast_abs {K : Type u_5} [linear_ordered_field K] {q : } :
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[norm_cast]
theorem rat.cast_id (n : ) :
n = n
@[simp]
theorem rat.cast_eq_id  :
@[simp]
theorem map_rat_cast {F : Type u_1} {α : Type u_3} {β : Type u_4} [division_ring α] [division_ring β] [ring_hom_class F α β] (f : F) (q : ) :
@[simp]
theorem eq_rat_cast {F : Type u_1} {k : Type u_2} [division_ring k] [ring_hom_class F k] (f : F) (r : ) :
f r = r
theorem monoid_with_zero_hom.ext_rat' {F : Type u_1} {M₀ : Type u_5} [monoid_with_zero M₀] [monoid_with_zero_hom_class F M₀] {f g : F} (h : (m : ), f m = g m) :
f = g

If f and g agree on the integers then they are equal φ.

@[ext]
theorem monoid_with_zero_hom.ext_rat {M₀ : Type u_5} [monoid_with_zero M₀] {f g : →*₀ M₀} (h : f.comp (int.cast_ring_hom ) = g.comp (int.cast_ring_hom )) :
f = g

If f and g agree on the integers then they are equal φ.

See note [partially-applied ext lemmas] for why comp is used here.

theorem monoid_with_zero_hom.ext_rat_on_pnat {F : Type u_1} {M₀ : Type u_5} [monoid_with_zero M₀] [monoid_with_zero_hom_class F M₀] {f g : F} (same_on_neg_one : f (-1) = g (-1)) (same_on_pnat : (n : ), 0 < n f n = g n) :
f = g

Positive integer values of a morphism φ and its value on -1 completely determine φ.

theorem ring_hom.ext_rat {F : Type u_1} {R : Type u_2} [semiring R] [ring_hom_class F R] (f g : F) :
f = g

Any two ring homomorphisms from to a semiring are equal. If the codomain is a division ring, then this lemma follows from eq_rat_cast.

@[protected, instance]
@[protected, instance]