Skip to content

Commit

Permalink
bump
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Jul 19, 2024
1 parent 079cac5 commit bc83c2e
Show file tree
Hide file tree
Showing 4 changed files with 2 additions and 48 deletions.
1 change: 0 additions & 1 deletion FltRegular.lean
Original file line number Diff line number Diff line change
Expand Up @@ -29,4 +29,3 @@ import FltRegular.NumberTheory.RegularPrimes
import FltRegular.NumberTheory.SystemOfUnits
import FltRegular.NumberTheory.Unramified
import FltRegular.ReadyForMathlib.Homogenization
import FltRegular.ReadyForMathlib.PowerBasis
6 changes: 1 addition & 5 deletions FltRegular/NumberTheory/Cyclotomic/MoreLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ import FltRegular.NumberTheory.Cyclotomic.UnitLemmas
import FltRegular.NumberTheory.Cyclotomic.CyclRat
import Mathlib.RingTheory.Ideal.Norm
import Mathlib.RingTheory.NormTrace
import FltRegular.ReadyForMathlib.PowerBasis

variable {K : Type*} {p : ℕ+} [hpri : Fact p.Prime] [Field K] [CharZero K] [IsCyclotomicExtension {p} ℚ K]

Expand Down Expand Up @@ -90,10 +89,7 @@ lemma exists_zeta_sub_one_dvd_sub_Int (a : 𝓞 K) : ∃ b : ℤ, (hζ.unit' - 1
letI : Fact (Nat.Prime p) := hpri
simp_rw [← Ideal.Quotient.eq_zero_iff_dvd, ← Ideal.Quotient.mk_eq_mk, Submodule.Quotient.mk_sub,
sub_eq_zero, ← SModEq.def]
convert exists_int_sModEq hζ.subOneIntegralPowerBasis' a
rw [hζ.subOneIntegralPowerBasis'_gen]
rw [Subtype.ext_iff, AddSubgroupClass.coe_sub, IsPrimitiveRoot.val_unit'_coe, OneMemClass.coe_one]
rfl
exact hζ.subOneIntegralPowerBasis'_gen ▸ hζ.subOneIntegralPowerBasis'.exists_smodEq a

lemma exists_dvd_pow_sub_Int_pow (a : 𝓞 K) : ∃ b : ℤ, ↑p ∣ a ^ (p : ℕ) - (b : 𝓞 K) ^ (p : ℕ) := by
obtain ⟨ζ, hζ⟩ := IsCyclotomicExtension.exists_prim_root ℚ (B := K) (Set.mem_singleton p)
Expand Down
41 changes: 0 additions & 41 deletions FltRegular/ReadyForMathlib/PowerBasis.lean

This file was deleted.

2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -65,7 +65,7 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "84542b3e09d0b491b76dc7b4eed87729001ca714",
"rev": "bb5c2ab8b54104352d8aaec9a606f327e5976028",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit bc83c2e

Please sign in to comment.