Documentation

Mathlib.Analysis.VonNeumannAlgebra.Basic

Von Neumann algebras #

We give the "abstract" and "concrete" definitions of a von Neumann algebra. We still have a major project ahead of us to show the equivalence between these definitions!

An abstract von Neumann algebra WStarAlgebra M is a C^* algebra with a Banach space predual, per Sakai (1971).

A concrete von Neumann algebra VonNeumannAlgebra H (where H is a Hilbert space) is a *-closed subalgebra of bounded operators on H which is equal to its double commutant.

We'll also need to prove the von Neumann double commutant theorem, that the concrete definition is equivalent to a *-closed subalgebra which is weakly closed.

Sakai's definition of a von Neumann algebra as a C^* algebra with a Banach space predual.

So that we can unambiguously talk about these "abstract" von Neumann algebras in parallel with the "concrete" ones (weakly closed *-subalgebras of B(H)), we name this definition WStarAlgebra.

Note that for now we only assert the mere existence of predual, rather than picking one. This may later prove problematic, and need to be revisited. Picking one may cause problems with definitional unification of different instances. One the other hand, not picking one means that the weak-* topology (which depends on a choice of predual) must be defined using the choice, and we may be unhappy with the resulting opaqueness of the definition.

Instances

    The double commutant definition of a von Neumann algebra, as a *-closed subalgebra of bounded operators on a Hilbert space, which is equal to its double commutant.

    Note that this definition is parameterised by the Hilbert space on which the algebra faithfully acts, as is standard in the literature. See WStarAlgebra for the abstract notion (a C^*-algebra with Banach space predual).

    Note this is a bundled structure, parameterised by the Hilbert space H, rather than a typeclass on the type of elements. Thus we can't say that the bounded operators H →L[ℂ] H form a VonNeumannAlgebra (although we will later construct the instance WStarAlgebra (H →L[ℂ] H)), and instead will use ⊤ : VonNeumannAlgebra H.

    Instances For
      Equations
      • VonNeumannAlgebra.instSetLike = { coe := fun (S : VonNeumannAlgebra H) => S.carrier, coe_injective' := }
      @[simp]
      theorem VonNeumannAlgebra.mem_carrier {H : Type u} [NormedAddCommGroup H] [InnerProductSpace H] [CompleteSpace H] {S : VonNeumannAlgebra H} {x : H →L[] H} :
      x S.toStarSubalgebra x S
      @[simp]
      @[simp]
      theorem VonNeumannAlgebra.coe_mk {H : Type u} [NormedAddCommGroup H] [InnerProductSpace H] [CompleteSpace H] (S : StarSubalgebra (H →L[] H)) (h : Set.centralizer (Set.centralizer S.carrier) = S.carrier) :
      { toStarSubalgebra := S, centralizer_centralizer' := h } = S
      theorem VonNeumannAlgebra.ext {H : Type u} [NormedAddCommGroup H] [InnerProductSpace H] [CompleteSpace H] {S : VonNeumannAlgebra H} {T : VonNeumannAlgebra H} (h : ∀ (x : H →L[] H), x S x T) :
      S = T

      The centralizer of a VonNeumannAlgebra, as a VonNeumannAlgebra.

      Equations
      Instances For