Skip to content

Commit

Permalink
useless
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Jul 3, 2024
1 parent a43940b commit 2e4d37d
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 4 deletions.
1 change: 0 additions & 1 deletion FltRegular/CaseII/AuxLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ import FltRegular.NumberTheory.Cyclotomic.UnitLemmas
import Mathlib.RingTheory.Ideal.Norm
import Mathlib.RingTheory.ClassGroup
import FltRegular.NumberTheory.Cyclotomic.MoreLemmas
import FltRegular.ReadyForMathlib.PowerBasis

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

Expand Down
3 changes: 0 additions & 3 deletions FltRegular/ReadyForMathlib/PowerBasis.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,6 @@ open RingOfIntegers Ideal Finset Nat FiniteDimensional

variable {K : Type _} [Field K] (pb : PowerBasis ℤ (𝓞 K))

instance instModuleSubtypeMemSubalgebraIntRingOfIntegers_fltRegular_bis :
Module (𝓞 K) (𝓞 K) := Semiring.toModule

theorem exists_int_sModEq (x : 𝓞 K) :
∃ (n : ℤ), SModEq (span ({ pb.gen } : Set (𝓞 K))) x n := by
refine' ⟨(pb.basis.repr x) ⟨0, pb.dim_pos⟩, _⟩
Expand Down

0 comments on commit 2e4d37d

Please sign in to comment.