Skip to content

Commit

Permalink
nicer
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Sep 9, 2024
1 parent eb68f8f commit 190acb7
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/Hilbert94.lean
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ open Polynomial
variable {L} [Field L] [Algebra K L] [FiniteDimensional K L]
(σ : L ≃ₐ[K] L) (hσ : ∀ x, x ∈ Subgroup.zpowers σ) (hKL : FiniteDimensional.finrank K L = p)

variable {A B} [CommRing A] [CommRing B] [Algebra A B] [Algebra A L] [Algebra A K]
variable {A B : Type*} [CommRing A] [CommRing B] [Algebra A B] [Algebra A L] [Algebra A K]
[Algebra B L] [IsScalarTower A B L] [IsScalarTower A K L] [IsFractionRing A K]
[IsIntegralClosure B A L]

Expand Down

0 comments on commit 190acb7

Please sign in to comment.