Zulip Chat Archive

Stream: Is there code for X?

Topic: Algebraic closure is normal


Xavier Roblot (Apr 04 2023 at 06:56):

Is it true that these results are missing?

import field_theory.is_alg_closed.algebraic_closure
import field_theory.normal

variables {R K : Type*} [field R] [field K] [algebra R K]

lemma is_alg_closure.normal (h : is_alg_closure R K) : normal R K :=
h.algebraic, λ _, @is_alg_closed.splits_codomain _ _ _ h.alg_closed _ _ _

instance : normal K (algebraic_closure K) :=
  is_alg_closure.normal (algebraic_closure.is_alg_closure _)

Ruben Van de Velde (Apr 04 2023 at 06:58):

is_alg_closed only seems used in three files under src/field_theory/is_alg_closed/, so if it's not there, it's not in mathlib

Xavier Roblot (Apr 04 2023 at 09:58):

#18730


Last updated: Dec 20 2023 at 11:08 UTC