Skip to content

Commit 33953c1

Browse files
ops
1 parent 7f79ab6 commit 33953c1

File tree

2 files changed

+1
-7
lines changed

2 files changed

+1
-7
lines changed

FltRegular/NumberTheory/Different.lean

-6
Original file line numberDiff line numberDiff line change
@@ -35,12 +35,6 @@ open nonZeroDivisors IsLocalization Matrix Algebra
3535

3636
variable [IsDedekindDomain B]
3737

38-
noncomputable
39-
example : InvolutiveInv (FractionalIdeal B⁰ L) := by
40-
exact DivisionMonoid.toInvolutiveInv
41-
42-
#synth DivisionMonoid (FractionalIdeal B⁰ L)
43-
4438
include K L in
4539
lemma pow_sub_one_dvd_differentIdeal_aux [IsDedekindDomain A]
4640
[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)