Skip to content

Commit

Permalink
move files
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Nov 6, 2023
1 parent e8ea484 commit a68ed38
Show file tree
Hide file tree
Showing 5 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion FltRegular/CaseII/AuxLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ import FltRegular.NumberTheory.Cyclotomic.Factoring
import FltRegular.NumberTheory.Cyclotomic.UnitLemmas
import Mathlib.RingTheory.Ideal.Norm
import Mathlib.RingTheory.ClassGroup
import FltRegular.Norm.NormPrime
import FltRegular.ReadyForMathlib.PowerBasis

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

Expand Down
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/Cyclotomic/CyclRat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ import FltRegular.NumberTheory.Cyclotomic.GaloisActionOnCyclo
import Mathlib.NumberTheory.Cyclotomic.Rat
import FltRegular.NumberTheory.Cyclotomic.UnitLemmas
import Mathlib.RingTheory.DedekindDomain.Ideal
import FltRegular.NumberTheory.Cyclotomic.ZetaSubOnePrime
import FltRegular.ReadyForMathlib.ZetaSubOnePrime
import FltRegular.NumberTheory.Cyclotomic.CyclotomicUnits
import Mathlib.Algebra.CharP.Quotient

Expand Down
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/Cyclotomic/UnitLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@ import FltRegular.NumberTheory.Cyclotomic.GaloisActionOnCyclo
import FltRegular.NumberTheory.Cyclotomic.CyclotomicUnits
import Mathlib.RingTheory.RootsOfUnity.Basic
import Mathlib.NumberTheory.NumberField.Embeddings
import FltRegular.NumberTheory.Cyclotomic.ZetaSubOnePrime
import FltRegular.ReadyForMathlib.ZetaSubOnePrime

variable {p : ℕ+} {K : Type _} [Field K]

Expand Down
File renamed without changes.

0 comments on commit a68ed38

Please sign in to comment.