Embeddings of number fields #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. This file defines the embeddings of a number field into an algebraic closed field.
Main Results #
number_field.embeddings.range_eval_eq_root_set_minpoly: letx ∈ KwithKnumber field and letAbe an algebraic closed field of char. 0, then the images ofxby the embeddings ofKinAare exactly the roots inAof the minimal polynomial ofxoverℚ.number_field.embeddings.pow_eq_one_of_norm_eq_one: an algebraic integer whose conjugates are all of norm one is a root of unity.
Tags #
number field, embeddings, places, infinite places
There are finitely many embeddings of a number field.
Equations
The number of embeddings of a number field is equal to its finrank.
Let A be an algebraically closed field and let x ∈ K, with K a number field.
The images of x by the embeddings of K in A are exactly the roots in A of
the minimal polynomial of x over ℚ.
Let B be a real number. The set of algebraic integers in K whose conjugates are all
smaller in norm than B is finite.
An algebraic integer whose conjugates are all of norm one is a root of unity.
An embedding into a normed division ring defines a place of K
Equations
The conjugate of a complex embedding as a complex embedding.
Equations
A embedding into ℂ is real if it is fixed by complex conjugation.
Equations
A real embedding as a ring homomorphism from K to ℝ .
An infinite place of a number field K is a place associated to a complex embedding.
Equations
- number_field.infinite_place K = {w // ∃ (φ : K →+* ℂ), number_field.place φ = w}
Return the infinite place defined by a complex embedding φ.
Equations
Equations
- number_field.infinite_place.has_coe_to_fun = {coe := λ (w : number_field.infinite_place K), ⇑(w.val)}
Equations
- number_field.infinite_place.real.monoid_with_zero_hom_class = {coe := λ (w : number_field.infinite_place K) (x : K), ⇑(w.val) x, coe_injective' := _, map_mul := _, map_one := _, map_zero := _}
Equations
- number_field.infinite_place.real.nonneg_hom_class = {coe := λ (w : number_field.infinite_place K) (x : K), ⇑w x, coe_injective' := _, map_nonneg := _}
For an infinite place w, return an embedding φ such that w = infinite_place φ .
Equations
- w.embedding = Exists.some _
An infinite place is real if it is defined by a real embedding.
Equations
- w.is_real = ∃ (φ : K →+* ℂ), number_field.complex_embedding.is_real φ ∧ number_field.infinite_place.mk φ = w
An infinite place is complex if it is defined by a complex (ie. not real) embedding.
Equations
- w.is_complex = ∃ (φ : K →+* ℂ), ¬number_field.complex_embedding.is_real φ ∧ number_field.infinite_place.mk φ = w
The map from real embeddings to real infinite places as an equiv
Equations
- number_field.infinite_place.mk_real K = {to_fun := subtype.map number_field.infinite_place.mk _, inv_fun := λ (w : {w // w.is_real}), ⟨w.val.embedding, _⟩, left_inv := _, right_inv := _}
The map from nonreal embeddings to complex infinite places
Equations
The infinite part of the product formula : for x ∈ K, we have Π_w ‖x‖_w = |norm(x)| where
‖·‖_w is the normalized absolute value for w.