Skip to content

Commit

Permalink
feat(FieldTheory/IsAlgClosed/Basic): add IsAlgClosed.perfectField i…
Browse files Browse the repository at this point in the history
…nstance (#9710)

Co-authored-by: Junyan Xu <junyanxu.math@gmail.com>
  • Loading branch information
2 people authored and riccardobrasca committed Jan 19, 2024
1 parent 5f1151c commit 07a9af9
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/FieldTheory/IsAlgClosed/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -283,6 +283,10 @@ noncomputable instance (priority := 100) perfectRing (p : ℕ) [Fact p.Prime] [C
PerfectRing.ofSurjective k p fun _ => IsAlgClosed.exists_pow_nat_eq _ <| NeZero.pos p
#align is_alg_closed.perfect_ring IsAlgClosed.perfectRing

noncomputable instance (priority := 100) perfectField [IsAlgClosed k] : PerfectField k := by
obtain _ | ⟨p, _, _⟩ := CharP.exists' k
exacts [.ofCharZero k, PerfectRing.toPerfectField k p]

/-- Algebraically closed fields are infinite since `Xⁿ⁺¹ - 1` is separable when `#K = n` -/
instance (priority := 500) {K : Type*} [Field K] [IsAlgClosed K] : Infinite K := by
apply Infinite.of_not_fintype
Expand Down

0 comments on commit 07a9af9

Please sign in to comment.