Skip to content

Commit

Permalink
better
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Oct 25, 2024
1 parent 9b4f485 commit 7f79ab6
Show file tree
Hide file tree
Showing 2 changed files with 7 additions and 2 deletions.
7 changes: 6 additions & 1 deletion FltRegular/NumberTheory/Different.lean
Original file line number Diff line number Diff line change
@@ -1,6 +1,5 @@
import Mathlib.RingTheory.DedekindDomain.Different
import Mathlib.RingTheory.DedekindDomain.Ideal
import Mathlib.RingTheory.DedekindDomain.Different
import Mathlib.RingTheory.Localization.FractionRing
import Mathlib.RingTheory.Trace.Quotient
import Mathlib.NumberTheory.KummerDedekind
Expand Down Expand Up @@ -36,6 +35,12 @@ open nonZeroDivisors IsLocalization Matrix Algebra

variable [IsDedekindDomain B]

noncomputable
example : InvolutiveInv (FractionalIdeal B⁰ L) := by
exact DivisionMonoid.toInvolutiveInv

#synth DivisionMonoid (FractionalIdeal B⁰ L)

include K L in
lemma pow_sub_one_dvd_differentIdeal_aux [IsDedekindDomain A]
[NoZeroSMulDivisors A B] [Module.Finite A B]
Expand Down
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/KummersLemma/Field.lean
Original file line number Diff line number Diff line change
Expand Up @@ -272,7 +272,7 @@ lemma separable_poly (I : Ideal (𝓞 K)) [I.IsMaximal] :
rw [ne_eq, Ideal.map_eq_top_iff]; exact Ideal.IsMaximal.ne_top ‹_›
· intros x y e; ext; exact (algebraMap K L).injective (congr_arg Subtype.val e)
· intros x; exact IsIntegral.tower_top (IsIntegralClosure.isIntegral ℤ L x)
rw [← Polynomial.separable_map i, map_map, Ideal.quotientMap_comp_mk, ← map_map]
rw [← Polynomial.separable_map' i, map_map, Ideal.quotientMap_comp_mk, ← map_map]
apply Separable.map
apply separable_poly_aux hp hζ u hcong
exact root_X_pow_sub_C_pow _ _
Expand Down

0 comments on commit 7f79ab6

Please sign in to comment.