Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 700effa

Browse files
committed
feat(ring_theory/localization): the algebraic elements over Frac(R) are those over R (#8826)
We had this lemma for `L / K` is algebraic iff `L / A` is, but now we also have it elementwise!
1 parent 2a69dc2 commit 700effa

File tree

1 file changed

+18
-7
lines changed

1 file changed

+18
-7
lines changed

src/ring_theory/localization.lean

Lines changed: 18 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -1590,21 +1590,32 @@ begin
15901590
exact to_map_eq_zero_iff.mp h }
15911591
end
15921592

1593-
/-- A field is algebraic over the ring `A` iff it is algebraic over the field of fractions of `A`.
1593+
variables (A K)
1594+
1595+
/-- An element of a field is algebraic over the ring `A` iff it is algebraic
1596+
over the field of fractions of `A`.
15941597
-/
1595-
lemma comap_is_algebraic_iff [algebra A L] [algebra K L] [is_scalar_tower A K L] :
1596-
algebra.is_algebraic A Lalgebra.is_algebraic K L :=
1598+
lemma is_algebraic_iff [algebra A L] [algebra K L] [is_scalar_tower A K L] {x : L} :
1599+
is_algebraic A x ↔ is_algebraic K x :=
15971600
begin
1598-
split; intros h x; obtain ⟨p, hp, px⟩ := h x,
1601+
split; rintros ⟨p, hp, px⟩,
15991602
{ refine ⟨p.map (algebra_map A K), λ h, hp (polynomial.ext (λ i, _)), _⟩,
1600-
{ have : algebra_map A K (p.coeff i) = 0 := trans (polynomial.coeff_map _ _).symm (by simp [h]),
1601-
exact to_map_eq_zero_iff.mp this },
1602-
{ rwa is_scalar_tower.aeval_apply _ K at px } },
1603+
{ have : algebra_map A K (p.coeff i) = 0 := trans (polynomial.coeff_map _ _).symm (by simp [h]),
1604+
exact to_map_eq_zero_iff.mp this },
1605+
{ rwa is_scalar_tower.aeval_apply _ K at px } },
16031606
{ exact ⟨integer_normalization _ p,
16041607
mt integer_normalization_eq_zero_iff.mp hp,
16051608
integer_normalization_aeval_eq_zero _ p px⟩ },
16061609
end
16071610

1611+
variables {A K}
1612+
1613+
/-- A field is algebraic over the ring `A` iff it is algebraic over the field of fractions of `A`.
1614+
-/
1615+
lemma comap_is_algebraic_iff [algebra A L] [algebra K L] [is_scalar_tower A K L] :
1616+
algebra.is_algebraic A L ↔ algebra.is_algebraic K L :=
1617+
⟨λ h x, (is_algebraic_iff A K).mp (h x), λ h x, (is_algebraic_iff A K).mpr (h x)⟩
1618+
16081619
section num_denom
16091620

16101621
variables (A) [unique_factorization_monoid A]

0 commit comments

Comments
 (0)