Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
alexjbest committed Nov 29, 2023
2 parents c42707b + 1636c21 commit 94459a0
Showing 1 changed file with 1 addition and 5 deletions.
6 changes: 1 addition & 5 deletions FltRegular/NumberTheory/Hilbert90.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ import FltRegular.NumberTheory.Cyclotomic.UnitLemmas
import FltRegular.NumberTheory.AuxLemmas
import FltRegular.NumberTheory.GaloisPrime
import Mathlib.Tactic.Widget.Conv
import Mathlib.RepresentationTheory.GroupCohomology.Hilbert90

open scoped NumberField nonZeroDivisors
open FiniteDimensional Finset BigOperators Submodule
Expand All @@ -12,11 +13,6 @@ variable [IsGalois K L] [FiniteDimensional K L]
variable (σ : L ≃ₐ[K] L) (hσ : ∀ x, x ∈ Subgroup.zpowers σ)
variable {η : L} (hη : Algebra.norm K η = 1)

--This is proved in #8599
theorem hilbert90 (f : (L ≃ₐ[K] L) → Lˣ)
(hf : ∀ (g h : (L ≃ₐ[K] L)), f (g * h) = g (f h) * f g) :
∃ β : Lˣ, ∀ g : (L ≃ₐ[K] L), f g * Units.map g β = β := by sorry

noncomputable
def ηu : Lˣ := (Ne.isUnit (fun h ↦ by simp [h] at hη) : IsUnit η).unit

Expand Down

0 comments on commit 94459a0

Please sign in to comment.