@@ -4,6 +4,8 @@ import Mathlib.RingTheory.Valuation.ValuationRing
4
4
import Mathlib.FieldTheory.Separable
5
5
import Mathlib.RingTheory.Trace.Defs
6
6
7
+ import Mathlib
8
+
7
9
/-!
8
10
9
11
This file contains lemmas that should go somewhere in a file in mathlib.
@@ -132,10 +134,6 @@ lemma IsSeparable_of_isLocalization (R S Rₚ Sₚ) [CommRing R] [CommRing S] [F
132
134
[IsScalarTower R S Sₚ] [IsScalarTower R Rₚ Sₚ] (M : Submonoid R) [IsLocalization M Rₚ]
133
135
[IsLocalization (Algebra.algebraMapSubmonoid S M) Sₚ] [hRS : Algebra.IsSeparable R S] :
134
136
Algebra.IsSeparable Rₚ Sₚ := by
135
- have : algebraMap Rₚ Sₚ = IsLocalization.map (T := Algebra.algebraMapSubmonoid S M) Sₚ
136
- (algebraMap R S) (Submonoid.le_comap_map M) := by
137
- apply IsLocalization.ringHom_ext M
138
- simp only [IsLocalization.map_comp, ← IsScalarTower.algebraMap_eq]
139
137
refine ⟨fun x ↦ ?_⟩
140
138
obtain ⟨x, s, rfl⟩ := IsLocalization.mk'_surjective (Algebra.algebraMapSubmonoid S M) x
141
139
obtain ⟨t, ht, e⟩ := s.prop
@@ -145,8 +143,8 @@ lemma IsSeparable_of_isLocalization (R S Rₚ Sₚ) [CommRing R] [CommRing S] [F
145
143
exact isUnit_of_invertible _
146
144
· rw [aeval_def]
147
145
convert scaleRoots_eval₂_eq_zero _ (r := algebraMap S Sₚ x) _
148
- · rw [this, IsLocalization.map_mk', _root_.map_one , IsLocalization.mk'_eq_mul_mk'_one ,
149
- mul_comm]
146
+ · rw [IsLocalization.algebraMap_eq_map_map_submonoid M S , IsLocalization.map_mk' ,
147
+ _root_.map_one, IsLocalization.mk'_eq_mul_mk'_one, mul_comm]
150
148
congr; ext; exact e.symm
151
149
· rw [← aeval_def, ← map_aeval_eq_aeval_map, minpoly.aeval, map_zero]
152
150
rw [← IsScalarTower.algebraMap_eq, ← IsScalarTower.algebraMap_eq]
0 commit comments