Skip to content

Commit 54cef9c

Browse files
those are useless
1 parent df804cb commit 54cef9c

File tree

3 files changed

+0
-59
lines changed

3 files changed

+0
-59
lines changed

FltRegular/NumberTheory/GaloisPrime.lean

-13
Original file line numberDiff line numberDiff line change
@@ -50,11 +50,6 @@ lemma primesOver_bot [Nontrivial R] [IsDomain S] [NoZeroSMulDivisors R S]
5050

5151
variable (S)
5252

53-
lemma primesOverFinset_bot [IsDedekindDomain S] : primesOverFinset S (⊥ : Ideal R) = ∅ := by
54-
classical
55-
rw [primesOverFinset, Ideal.map_bot, ← Ideal.zero_eq_bot, factors_zero]
56-
rfl
57-
5853
lemma coe_primesOverFinset [Ring.DimensionLEOne R] [IsDedekindDomain S]
5954
[NoZeroSMulDivisors R S] (p : Ideal R) (hp : p ≠ ⊥) [hp' : p.IsPrime] :
6055
primesOverFinset S p = primesOver S p := by
@@ -82,14 +77,6 @@ lemma primesOver_finite [Ring.DimensionLEOne R] [IsDedekindDomain S] [NoZeroSMul
8277
· rw [primesOver_eq_empty_of_not_isPrime S p h]
8378
exact Set.finite_empty
8479

85-
lemma primesOver_nonempty [IsDomain S] [NoZeroSMulDivisors R S] [Algebra.IsIntegral R S]
86-
(p : Ideal R) [p.IsPrime] : (primesOver S p).Nonempty := by
87-
have := Ideal.bot_prime (α := S)
88-
obtain ⟨Q, _, hQ⟩ := Ideal.exists_ideal_over_prime_of_isIntegral p ⊥
89-
(by rw [Ideal.comap_bot_of_injective _
90-
(NoZeroSMulDivisors.algebraMap_injective R S)]; exact bot_le)
91-
exact ⟨Q, hQ⟩
92-
9380
variable {S}
9481

9582
lemma ne_bot_of_mem_primesOver [IsDedekindDomain S] [NoZeroSMulDivisors R S] {p : Ideal R}

FltRegular/NumberTheory/Hilbert92.lean

-9
Original file line numberDiff line numberDiff line change
@@ -53,15 +53,6 @@ lemma systemOfUnits.IsFundamental.maximal' [Module A G] (S : systemOfUnits p G r
5353
letI := hs.choose
5454
convert hs.choose_spec a ‹_› <;> symm <;> exact Nat.card_eq_fintype_card.symm
5555

56-
@[to_additive]
57-
theorem Finsupp.prod_congr' {α M N} [Zero M] [CommMonoid N] {f₁ f₂ : α →₀ M} {g1 g2 : α → M → N}
58-
(h : ∀ x, g1 x (f₁ x) = g2 x (f₂ x)) (hg1 : ∀ i, g1 i 0 = 1) (hg2 : ∀ i, g2 i 0 = 1) :
59-
f₁.prod g1 = f₂.prod g2 := by
60-
classical
61-
rw [f₁.prod_of_support_subset Finset.subset_union_left _ (fun i _ ↦ hg1 i),
62-
f₂.prod_of_support_subset Finset.subset_union_right _ (fun i _ ↦ hg2 i)]
63-
exact Finset.prod_congr rfl (fun x _ ↦ h x)
64-
6556
@[simps]
6657
noncomputable
6758
def Finsupp.ltotal (α M R) [CommSemiring R] [AddCommMonoid M] [Module R M] :

FltRegular/NumberTheory/Unramified.lean

-37
Original file line numberDiff line numberDiff line change
@@ -120,47 +120,10 @@ lemma comap_map_eq_of_isUnramified [IsGalois K L] [IsUnramified R S] (I : Ideal
120120
Ideal.mem_normalizedFactors_iff hIbot']
121121
exact ⟨hP.1.comap _, Ideal.comap_mono hP.2
122122

123-
open scoped Classical in
124-
lemma isUnramifiedAt_iff_normalizedFactors_nodup [NoZeroSMulDivisors R S] [IsDedekindDomain S]
125-
(p : Ideal R) [p.IsPrime] (hp : p ≠ ⊥) :
126-
IsUnramifiedAt S p ↔ (normalizedFactors (p.map (algebraMap R S))).Nodup := by
127-
simp_rw [Multiset.nodup_iff_count_eq_one, ← Multiset.mem_toFinset,
128-
← factors_eq_normalizedFactors]
129-
show _ ↔ ∀ P ∈ (primesOverFinset S p : Set (Ideal S)), _
130-
simp_rw [IsUnramifiedAt, coe_primesOverFinset S p hp]
131-
refine forall₂_congr (fun P hP ↦ ?_)
132-
rw [Ideal.IsDedekindDomain.ramificationIdx_eq_factors_count]
133-
· exact (Ideal.map_eq_bot_iff_of_injective
134-
(NoZeroSMulDivisors.algebraMap_injective R S)).not.mpr hp
135-
· exact hP.1
136-
· exact ne_bot_of_mem_primesOver hp hP
137-
138123
section KummerDedekind
139124

140125
end KummerDedekind
141126

142-
attribute [local instance] Ideal.Quotient.field in
143-
lemma isUnramifiedAt_iff_SquareFree_minpoly [NoZeroSMulDivisors R S] [IsDedekindDomain S]
144-
(p : Ideal R) [hp : p.IsPrime] (hpbot : p ≠ ⊥) (x : S)
145-
(hx : (conductor R x).comap (algebraMap R S) ⊔ p = ⊤) (hx' : IsIntegral R x) :
146-
IsUnramifiedAt S p ↔ Squarefree ((minpoly R x).map (Ideal.Quotient.mk p)) := by
147-
classical
148-
have := hp.isMaximal hpbot
149-
rw [isUnramifiedAt_iff_normalizedFactors_nodup p hpbot,
150-
KummerDedekind.normalizedFactors_ideal_map_eq_normalizedFactors_min_poly_mk_map
151-
this hpbot hx hx', Multiset.nodup_map_iff_of_injective, Multiset.nodup_attach,
152-
← squarefree_iff_nodup_normalizedFactors (Polynomial.map_monic_ne_zero (minpoly.monic hx'))]
153-
exact Subtype.val_injective.comp
154-
(KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk
155-
this hpbot hx hx').symm.injective
156-
157-
lemma isUnramifiedAt_iff_SquareFree_minpoly_powerBasis [NoZeroSMulDivisors R S] [IsDedekindDomain S]
158-
[Algebra.IsIntegral R S] (pb : PowerBasis R S)
159-
(p : Ideal R) [p.IsPrime] (hpbot : p ≠ ⊥) :
160-
IsUnramifiedAt S p ↔ Squarefree ((minpoly R pb.gen).map (Ideal.Quotient.mk p)) := by
161-
rw [isUnramifiedAt_iff_SquareFree_minpoly p hpbot pb.gen _ _]
162-
rw [conductor_eq_top_of_powerBasis, Ideal.comap_top, top_sup_eq]
163-
exact PowerBasis.isIntegral_gen pb
164127

165128
open nonZeroDivisors Polynomial
166129

0 commit comments

Comments
 (0)