Documentation

Mathlib.RepresentationTheory.GroupCohomology.Hilbert90

Hilbert's Theorem 90 #

Let L/K be a finite extension of fields. Then this file proves Noether's generalization of Hilbert's Theorem 90: that the 1st group cohomology $H^1(Aut_K(L), Lˣ)$ is trivial. We state it both in terms of $H^1$ and in terms of cocycles being coboundaries.

Hilbert's original statement was that if $L/K$ is Galois, and $Gal(L/K)$ is cyclic, generated by an element σ, then for every x : L such that $N_{L/K}(x) = 1,$ there exists y : L such that $x = y/σ(y).$ This can be deduced from the fact that the function $Gal(L/K) → L^\times$ sending $σ^i \mapsto xσ(x)σ^2(x)...σ^{i-1}(x)$ is a 1-cocycle. Alternatively, we can derive it by analyzing the cohomology of finite cyclic groups in general.

Noether's generalization also holds for infinite Galois extensions.

Main statements #

Implementation notes #

Given a commutative ring k and a group G, group cohomology is developed in terms of k-linear G-representations on k-modules. Therefore stating Noether's generalization of Hilbert 90 in terms of requires us to turn the natural action of Aut_K(L) on into a morphism Aut_K(L) →* (Additive Lˣ →ₗ[ℤ] Additive Lˣ). Thus we provide the non- version too, as its statement is clearer.

TODO #

noncomputable def groupCohomology.Hilbert90.aux {K : Type u_1} {L : Type u_2} [Field K] [Field L] [Algebra K L] [FiniteDimensional K L] (f : (L ≃ₐ[K] L)Lˣ) :
LL

Given f : Aut_K(L) → Lˣ, the sum ∑ f(φ) • φ for φ ∈ Aut_K(L), as a function L → L.

Equations
Instances For

    Noether's generalization of Hilbert's Theorem 90: given a finite extension of fields and a function f : Aut_K(L) → Lˣ satisfying f(gh) = g(f(h)) * f(g) for all g, h : Aut_K(L), there exists β : Lˣ such that g(β)/β = f(g) for all g : Aut_K(L).

    Noether's generalization of Hilbert's Theorem 90: given a finite extension of fields L/K, the first group cohomology H¹(Aut_K(L), Lˣ) is trivial.

    Equations