Skip to content

Commit

Permalink
fix typo
Browse files Browse the repository at this point in the history
  • Loading branch information
CBirkbeck committed Dec 4, 2023
1 parent d6c81c5 commit 8230196
Showing 1 changed file with 8 additions and 2 deletions.
10 changes: 8 additions & 2 deletions FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -799,8 +799,14 @@ 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) E = ((σ ^ i) (algebraMap k K ζ^((p : ℕ)^(h-1)))) * E :=
by sorry
have h1 : ∀ (i : ℕ), (σ ^ (i+1)) E = ((σ ^ (i+1)) (algebraMap k K ζ^((p : ℕ)^(h-1)))) * E :=
by
intro i
induction i
simp
sorry
sorry




Expand Down

0 comments on commit 8230196

Please sign in to comment.