Skip to content

Commit

Permalink
chore(ring_theory/localization) weaken hypothesis from field to comm_…
Browse files Browse the repository at this point in the history
…ring (#11713)

also making `B` an explicit argument





Co-authored-by: chughes <christopher.hughes@inria.fr>
  • Loading branch information
ChrisHughes24 and chughes committed Jan 30, 2022
1 parent 1ea49d0 commit dde904e
Show file tree
Hide file tree
Showing 3 changed files with 15 additions and 10 deletions.
2 changes: 1 addition & 1 deletion src/number_theory/class_number/finite.lean
Expand Up @@ -391,7 +391,7 @@ begin
(is_integral_closure.range_le_span_dual_basis S b hb_int),
let bS := b.map ((linear_map.quot_ker_equiv_range _).symm ≪≫ₗ _),
refine fintype_of_admissible_of_algebraic L bS adm
(λ x, (is_fraction_ring.is_algebraic_iff R K).mpr (algebra.is_algebraic_of_finite x)),
(λ x, (is_fraction_ring.is_algebraic_iff R K L).mpr (algebra.is_algebraic_of_finite x)),
{ rw linear_map.ker_eq_bot.mpr,
{ exact submodule.quot_equiv_of_eq_bot _ rfl },
{ exact is_integral_closure.algebra_map_injective _ R _ } },
Expand Down
2 changes: 1 addition & 1 deletion src/ring_theory/dedekind_domain.lean
Expand Up @@ -826,7 +826,7 @@ begin
rintros x ⟨⟩ },
{ rintros x s hx ⟨y, hy, hs⟩,
obtain ⟨x', y', hy', hx'⟩ := exists_integral_multiple
((is_fraction_ring.is_algebraic_iff A K).mpr (algebra.is_algebraic_of_finite x))
((is_fraction_ring.is_algebraic_iff A K L).mpr (algebra.is_algebraic_of_finite x))
((algebra_map A L).injective_iff.mp _),
refine ⟨y * y', mul_ne_zero hy hy', λ x'' hx'', _⟩,
rcases finset.mem_insert.mp hx'' with (rfl | hx''),
Expand Down
21 changes: 13 additions & 8 deletions src/ring_theory/localization.lean
Expand Up @@ -2283,12 +2283,15 @@ begin
exact to_map_eq_zero_iff.mp h }
end

variables (A K)
section

variables (A K) (C : Type*)
variables [comm_ring C]

/-- An element of a field is algebraic over the ring `A` iff it is algebraic
/-- An element of a ring is algebraic over the ring `A` iff it is algebraic
over the field of fractions of `A`.
-/
lemma is_algebraic_iff [algebra A L] [algebra K L] [is_scalar_tower A K L] {x : L} :
lemma is_algebraic_iff [algebra A C] [algebra K C] [is_scalar_tower A K C] {x : C} :
is_algebraic A x ↔ is_algebraic K x :=
begin
split; rintros ⟨p, hp, px⟩,
Expand All @@ -2301,13 +2304,15 @@ begin
integer_normalization_aeval_eq_zero _ p px⟩ },
end

variables {A K}
variables {A K C}

/-- A field is algebraic over the ring `A` iff it is algebraic over the field of fractions of `A`.
/-- A ring is algebraic over the ring `A` iff it is algebraic over the field of fractions of `A`.
-/
lemma comap_is_algebraic_iff [algebra A L] [algebra K L] [is_scalar_tower A K L] :
algebra.is_algebraic A L ↔ algebra.is_algebraic K L :=
⟨λ h x, (is_algebraic_iff A K).mp (h x), λ h x, (is_algebraic_iff A K).mpr (h x)⟩
lemma comap_is_algebraic_iff [algebra A C] [algebra K C] [is_scalar_tower A K C] :
algebra.is_algebraic A C ↔ algebra.is_algebraic K C :=
⟨λ h x, (is_algebraic_iff A K C).mp (h x), λ h x, (is_algebraic_iff A K C).mpr (h x)⟩

end

section num_denom

Expand Down

0 comments on commit dde904e

Please sign in to comment.