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

Commit 3148cfe

Browse files
committed
feat(field_theory/algebraic_closure): polynomials in an algebraically closed fields have roots (#9037)
1 parent 3a62419 commit 3148cfe

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/field_theory/algebraic_closure.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -69,6 +69,9 @@ polynomial.splits_of_splits_id _ $ is_alg_closed.splits _
6969

7070
namespace is_alg_closed
7171

72+
theorem exists_root [is_alg_closed k] (p : polynomial k) (hp : p.degree ≠ 0) : ∃ x, is_root p x :=
73+
exists_root_of_splits _ (is_alg_closed.splits p) hp
74+
7275
theorem of_exists_root (H : ∀ p : polynomial k, p.monic → irreducible p → ∃ x, p.eval x = 0) :
7376
is_alg_closed k :=
7477
⟨λ p, or.inr $ λ q hq hqp,

0 commit comments

Comments
 (0)