Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
alexjbest committed Nov 29, 2023
1 parent ab6801d commit c11304e
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -82,4 +82,4 @@ end thm91
lemma Hilbert92
[Algebra k K] [IsGalois k K] [FiniteDimensional k K]
(hKL : finrank k K = p) (σ : K ≃ₐ[k] K) (hσ : ∀ x, x ∈ Subgroup.zpowers σ) :
∃ η : (𝓞 K)ˣ, Algebra.norm K (η : K) = 1 ∧ ∀ ε : (𝓞 K)ˣ, (η : K) ≠ ε / (σ ε : K) := sorry
∃ η : (𝓞 K)ˣ, Algebra.norm k (η : K) = 1 ∧ ∀ ε : (𝓞 K)ˣ, (η : K) ≠ ε / (σ ε : K) := sorry

0 comments on commit c11304e

Please sign in to comment.