Skip to content

Commit

Permalink
feat(field_theory/is_alg_closed/algebraic_closure): add instances no…
Browse files Browse the repository at this point in the history
…rmal and is_galois for algebraic closure (#18730)
  • Loading branch information
xroblot committed Apr 5, 2023
1 parent b2a5f0d commit 0ac3057
Show file tree
Hide file tree
Showing 3 changed files with 24 additions and 4 deletions.
10 changes: 9 additions & 1 deletion src/field_theory/galois.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Thomas Browning, Patrick Lutz
-/

import field_theory.normal
import field_theory.is_alg_closed.algebraic_closure
import field_theory.primitive_element
import field_theory.fixed
import group_theory.group_action.fixing_subgroup
Expand Down Expand Up @@ -424,3 +424,11 @@ end
end is_galois

end galois_equivalent_definitions

section is_alg_closure

@[priority 100]
instance is_alg_closure.is_galois (k K : Type*) [field k] [field K] [algebra k K]
[is_alg_closure k K] [char_zero k] : is_galois k K := { }

end is_alg_closure
2 changes: 1 addition & 1 deletion src/field_theory/is_alg_closed/algebraic_closure.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Kenny Lau
-/
import algebra.direct_limit
import field_theory.is_alg_closed.basic
import field_theory.splitting_field

/-!
# Algebraic Closure
Expand Down
16 changes: 14 additions & 2 deletions src/field_theory/is_alg_closed/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,9 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau
-/

import field_theory.normal
import field_theory.perfect_closure
import field_theory.separable
import ring_theory.adjoin.field
import ring_theory.localization.integral

/-!
Expand Down Expand Up @@ -170,6 +169,19 @@ theorem is_alg_closure_iff (K : Type v) [field K] [algebra k K] :
is_alg_closure k K ↔ is_alg_closed K ∧ algebra.is_algebraic k K :=
⟨λ h, ⟨h.1, h.2⟩, λ h, ⟨h.1, h.2⟩⟩

@[priority 100]
instance is_alg_closure.normal (R K : Type*) [field R] [field K] [algebra R K] [is_alg_closure R K]:
normal R K :=
⟨is_alg_closure.algebraic, λ _,
@is_alg_closed.splits_codomain _ _ _ (is_alg_closure.alg_closed R) _ _ _⟩

@[priority 100]
instance is_alg_closure.separable (R K : Type*) [field R] [field K] [algebra R K]
[is_alg_closure R K] [char_zero R] :
is_separable R K :=
⟨λ _, is_algebraic_iff_is_integral.mp (is_alg_closure.algebraic _), λ _, (minpoly.irreducible
(is_algebraic_iff_is_integral.mp (is_alg_closure.algebraic _))).separable⟩

namespace lift

/- In this section, the homomorphism from any algebraic extension into an algebraically
Expand Down

0 comments on commit 0ac3057

Please sign in to comment.