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

Commit dad88d8

Browse files
committed
feat(field_theory/splitting_field): add splits_X theorem (#5343)
This is a handy result and isn't definitionally a special case of splits_X_sub_C
1 parent cf7377a commit dad88d8

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/field_theory/splitting_field.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -101,6 +101,9 @@ splits_of_splits_of_dvd i one_ne_zero (splits_one _) $ is_unit_iff_dvd_one.1 hu
101101
theorem splits_X_sub_C {x : α} : (X - C x).splits i :=
102102
splits_of_degree_eq_one _ $ degree_X_sub_C x
103103

104+
theorem splits_X : X.splits i :=
105+
splits_of_degree_eq_one _ $ degree_X
106+
104107
theorem splits_id_iff_splits {f : polynomial α} :
105108
(f.map i).splits (ring_hom.id β) ↔ f.splits i :=
106109
by rw [splits_map_iff, ring_hom.id_comp]

0 commit comments

Comments
 (0)