Skip to content

Commit

Permalink
properly fix the typo now
Browse files Browse the repository at this point in the history
  • Loading branch information
CBirkbeck committed Dec 4, 2023
1 parent 8230196 commit 9fe72a8
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -799,11 +799,13 @@ lemma Hilbert92ish (hp : Nat.Prime p)
obtain ⟨S, hS⟩ := Hilbert91ish p (K := K) (k := k) hp hKL σ hσ
have NE_p_pow : (Units.map (algebraMap (𝓞 k) (𝓞 K)).toMonoidHom NE) = E ^ (p : ℕ) := by

have h1 : ∀ (i : ℕ), (σ ^ (i+1)) E = ((σ ^ (i+1)) (algebraMap k K ζ^((p : ℕ)^(h-1)))) * E :=
have h1 : ∀ (i : ℕ), (σ ^ (i+1)) E = ((σ ^ (i+1)) (algebraMap k K ζ^((p : ℕ)^(h-1)))⁻¹) * E :=
by
intro i
induction i
simp
rw [hE]

sorry
sorry

Expand Down

0 comments on commit 9fe72a8

Please sign in to comment.