2024-11-25 05:41:46 +00:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
Authors: Joseph Tooby-Smith
|
|
|
|
|
-/
|
2024-11-29 15:02:07 +00:00
|
|
|
|
import HepLean.FeynmanDiagrams.Wick.Species
|
2024-11-25 05:41:46 +00:00
|
|
|
|
/-!
|
2024-11-25 10:13:24 +00:00
|
|
|
|
|
|
|
|
|
# Operator algebra
|
2024-11-25 05:41:46 +00:00
|
|
|
|
|
|
|
|
|
Currently this file is only for an example of Wick strings, correpsonding to a
|
|
|
|
|
theory with two complex scalar fields. The concepts will however generalize.
|
|
|
|
|
|
|
|
|
|
This file is currently a stub.
|
|
|
|
|
|
|
|
|
|
We will formally define the operator ring, in terms of the fields present in the theory.
|
|
|
|
|
|
2024-11-26 09:05:55 +00:00
|
|
|
|
## Futher reading
|
|
|
|
|
|
|
|
|
|
- https://physics.stackexchange.com/questions/258718/ and links therein
|
|
|
|
|
- Ryan Thorngren (https://physics.stackexchange.com/users/10336/ryan-thorngren), Fermions,
|
2024-11-29 06:38:52 +00:00
|
|
|
|
different species and (anti-)commutation rules, URL (version: 2019-02-20) :
|
2024-11-26 09:05:55 +00:00
|
|
|
|
https://physics.stackexchange.com/q/461929
|
2024-11-25 05:41:46 +00:00
|
|
|
|
-/
|
|
|
|
|
|
2024-11-29 15:02:07 +00:00
|
|
|
|
namespace Wick
|
2024-11-25 05:41:46 +00:00
|
|
|
|
open CategoryTheory
|
|
|
|
|
open FeynmanDiagram
|
|
|
|
|
open PreFeynmanRule
|
|
|
|
|
|
2024-11-29 10:02:37 +00:00
|
|
|
|
informal_definition WickAlgebra where
|
|
|
|
|
math :≈ "
|
|
|
|
|
Modifications of this may be needed.
|
|
|
|
|
A structure with the following data:
|
|
|
|
|
- A ℤ₂-graded algebra A.
|
|
|
|
|
- A map from `ψ : 𝓔 × SpaceTime → A` where 𝓔 are field colors.
|
2024-11-29 10:33:29 +00:00
|
|
|
|
- A map `ψ₊ : 𝓔 × SpaceTime → A`.
|
|
|
|
|
- A map `ψ₋ : 𝓔 × SpaceTime → A`.
|
2024-11-29 10:02:37 +00:00
|
|
|
|
Subject to the conditions:
|
|
|
|
|
- The sum of `ψ0` and `ψ1` is `ψ`.
|
|
|
|
|
- Two fields super-commute if there colors are not dual to each other.
|
|
|
|
|
- The super-commutator of two fields is always in the
|
|
|
|
|
center of the algebra. "
|
2024-11-29 10:33:29 +00:00
|
|
|
|
physics :≈ "This is defined to be an
|
|
|
|
|
abstraction of the notion of an operator algebra."
|
2024-11-29 10:02:37 +00:00
|
|
|
|
ref :≈ "https://physics.stackexchange.com/questions/24157/"
|
|
|
|
|
|
|
|
|
|
informal_definition WickMonomial where
|
|
|
|
|
math :≈ "The type of elements of the Wick algebra which is a product of fields."
|
|
|
|
|
deps :≈ [``WickAlgebra]
|
|
|
|
|
|
|
|
|
|
namespace WickMonomial
|
|
|
|
|
|
|
|
|
|
informal_definition toWickAlgebra where
|
|
|
|
|
math :≈ "A function from WickMonomial to WickAlgebra which takes a monomial and
|
|
|
|
|
returns the product of the fields in the monomial."
|
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial]
|
|
|
|
|
|
2024-11-29 10:33:29 +00:00
|
|
|
|
informal_definition timeOrder where
|
2024-11-29 10:02:37 +00:00
|
|
|
|
math :≈ "A function from WickMonomial to WickAlgebra which takes a monomial and
|
|
|
|
|
returns the monomial with the fields time ordered, with the correct sign
|
|
|
|
|
determined by the Koszul sign factor."
|
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial]
|
|
|
|
|
|
2024-11-29 10:33:29 +00:00
|
|
|
|
informal_definition normalOrder where
|
2024-11-29 10:02:37 +00:00
|
|
|
|
math :≈ "A function from WickMonomial to WickAlgebra which takes a monomial and
|
|
|
|
|
returns the element in `WickAlgebra` defined as follows
|
|
|
|
|
- The ψ₊ fields are move to the right.
|
|
|
|
|
- The ψ₋ fields are moved to the left.
|
|
|
|
|
- Othewise the order of the fields is preserved."
|
|
|
|
|
ref :≈ "https://www.imperial.ac.uk/media/imperial-college/research-centres-and-groups/theoretical-physics/msc/current/qft/handouts/qftwickstheorem.pdf"
|
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial]
|
|
|
|
|
|
|
|
|
|
end WickMonomial
|
|
|
|
|
|
|
|
|
|
informal_definition contraction where
|
|
|
|
|
math :≈ "Given two `i j : 𝓔 × SpaceTime`, the element of WickAlgebra
|
|
|
|
|
defined by subtracting the normal ordering of `ψ i ψ j` from the time-ordering of
|
|
|
|
|
`ψ i ψ j`."
|
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial]
|
|
|
|
|
|
2024-11-29 10:33:29 +00:00
|
|
|
|
informal_lemma contraction_in_center where
|
|
|
|
|
math :≈ "The contraction of two fields is in the center of the algebra."
|
|
|
|
|
deps :≈ [``WickAlgebra, ``contraction]
|
|
|
|
|
|
|
|
|
|
informal_lemma contraction_non_dual_is_zero where
|
|
|
|
|
math :≈ "The contraction of two fields is zero if the fields are not dual to each other."
|
|
|
|
|
deps :≈ [``WickAlgebra, ``contraction]
|
|
|
|
|
|
|
|
|
|
informal_lemma timeOrder_single where
|
|
|
|
|
math :≈ "The time ordering of a single field is the normal ordering of that field."
|
2024-11-29 10:53:20 +00:00
|
|
|
|
proof :≈ "Follows from the definitions."
|
2024-11-29 10:33:29 +00:00
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial.timeOrder, ``WickMonomial.normalOrder]
|
|
|
|
|
|
|
|
|
|
informal_lemma timeOrder_pair where
|
|
|
|
|
math :≈ "The time ordering of two fields is the normal ordering of the fields plus the
|
|
|
|
|
contraction of the fields."
|
2024-11-29 10:53:20 +00:00
|
|
|
|
proof :≈ "Follows from the definition of contraction."
|
2024-11-29 10:33:29 +00:00
|
|
|
|
deps :≈ [``WickAlgebra, ``WickMonomial.timeOrder, ``WickMonomial.normalOrder,
|
|
|
|
|
``contraction]
|
|
|
|
|
|
2024-11-29 11:20:37 +00:00
|
|
|
|
/-! TODO: Need to set up data and structure for vaccum expectation values. -/
|
2024-11-29 11:49:55 +00:00
|
|
|
|
|
2024-11-29 15:02:07 +00:00
|
|
|
|
end Wick
|