Skip to content

Commit

Permalink
this never ends
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Sep 12, 2024
1 parent d689fc5 commit a557f17
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 @@ -780,7 +780,7 @@ lemma almostHilbert92 (hpodd : (p : ℕ) ≠ 2) :
classical
obtain ⟨h, ν, hν, hν'⟩ := h_exists' p (k := k) hp
by_cases H : ∀ ε : (𝓞 K)ˣ, algebraMap k K ν ^ ((p : ℕ)^(h - 1)) ≠ ε / (σ ε : K)
/- ν is ν' in Hilbert, so their ν is our ν ^ ((p : ℕ)^(h - 1)) -/
/- ν is ζ' in Hilbert, so their ζ is our ν ^ ((p : ℕ)^(h - 1)) -/
· exact Hilbert92_aux0 p hKL σ h ν hν H
simp only [ne_eq, not_forall, not_not] at H
obtain ⟨E, hE⟩ := H
Expand Down

0 comments on commit a557f17

Please sign in to comment.