Skip to content

Commit 7f79ab6

Browse files
better
1 parent 9b4f485 commit 7f79ab6

File tree

2 files changed

+7
-2
lines changed

2 files changed

+7
-2
lines changed

FltRegular/NumberTheory/Different.lean

+6-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,5 @@
11
import Mathlib.RingTheory.DedekindDomain.Different
22
import Mathlib.RingTheory.DedekindDomain.Ideal
3-
import Mathlib.RingTheory.DedekindDomain.Different
43
import Mathlib.RingTheory.Localization.FractionRing
54
import Mathlib.RingTheory.Trace.Quotient
65
import Mathlib.NumberTheory.KummerDedekind
@@ -36,6 +35,12 @@ open nonZeroDivisors IsLocalization Matrix Algebra
3635

3736
variable [IsDedekindDomain B]
3837

38+
noncomputable
39+
example : InvolutiveInv (FractionalIdeal B⁰ L) := by
40+
exact DivisionMonoid.toInvolutiveInv
41+
42+
#synth DivisionMonoid (FractionalIdeal B⁰ L)
43+
3944
include K L in
4045
lemma pow_sub_one_dvd_differentIdeal_aux [IsDedekindDomain A]
4146
[NoZeroSMulDivisors A B] [Module.Finite A B]

FltRegular/NumberTheory/KummersLemma/Field.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -272,7 +272,7 @@ lemma separable_poly (I : Ideal (𝓞 K)) [I.IsMaximal] :
272272
rw [ne_eq, Ideal.map_eq_top_iff]; exact Ideal.IsMaximal.ne_top ‹_›
273273
· intros x y e; ext; exact (algebraMap K L).injective (congr_arg Subtype.val e)
274274
· intros x; exact IsIntegral.tower_top (IsIntegralClosure.isIntegral ℤ L x)
275-
rw [← Polynomial.separable_map i, map_map, Ideal.quotientMap_comp_mk, ← map_map]
275+
rw [← Polynomial.separable_map' i, map_map, Ideal.quotientMap_comp_mk, ← map_map]
276276
apply Separable.map
277277
apply separable_poly_aux hp hζ u hcong
278278
exact root_X_pow_sub_C_pow _ _

0 commit comments

Comments
 (0)