2024-09-15 19:01:34 -04: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
|
|
|
|
|
-/
|
|
|
|
|
import HepLean.Meta.Informal
|
|
|
|
|
/-!
|
|
|
|
|
|
|
|
|
|
# Weyl fermions
|
|
|
|
|
|
|
|
|
|
-/
|
|
|
|
|
|
|
|
|
|
/-!
|
|
|
|
|
|
|
|
|
|
## The definition of Weyl fermion vector spaces.
|
|
|
|
|
|
|
|
|
|
-/
|
|
|
|
|
|
|
|
|
|
informal_definition leftHandedWeylFermion where
|
|
|
|
|
math :≈ "The vector space ℂ^2 carrying the fundamental representation of SL(2,C)."
|
2024-09-16 13:41:52 -04:00
|
|
|
|
physics :≈ "A Weyl fermion with indices ψ_a."
|
2024-09-15 19:01:34 -04:00
|
|
|
|
ref :≈ "https://particle.physics.ucdavis.edu/modernsusy/slides/slideimages/spinorfeynrules.pdf"
|
|
|
|
|
|
|
|
|
|
informal_definition rightHandedWeylFermion where
|
|
|
|
|
math :≈ "The vector space ℂ^2 carrying the conjguate representation of SL(2,C)."
|
2024-09-16 13:41:52 -04:00
|
|
|
|
physics :≈ "A Weyl fermion with indices ψ_{dot a}."
|
2024-09-15 19:01:34 -04:00
|
|
|
|
ref :≈ "https://particle.physics.ucdavis.edu/modernsusy/slides/slideimages/spinorfeynrules.pdf"
|
|
|
|
|
|
|
|
|
|
informal_definition altLeftHandedWeylFermion where
|
|
|
|
|
math :≈ "The vector space ℂ^2 carrying the representation of SL(2,C) given by
|
|
|
|
|
M → (M⁻¹)ᵀ."
|
2024-09-16 13:41:52 -04:00
|
|
|
|
physics :≈ "A Weyl fermion with indices ψ^a."
|
2024-09-15 19:01:34 -04:00
|
|
|
|
ref :≈ "https://particle.physics.ucdavis.edu/modernsusy/slides/slideimages/spinorfeynrules.pdf"
|
|
|
|
|
|
|
|
|
|
informal_definition altRightHandedWeylFermion where
|
|
|
|
|
math :≈ "The vector space ℂ^2 carrying the representation of SL(2,C) given by
|
|
|
|
|
M → (M⁻¹)^†."
|
2024-09-16 13:41:52 -04:00
|
|
|
|
physics :≈ "A Weyl fermion with indices ψ^{dot a}."
|
2024-09-15 19:01:34 -04:00
|
|
|
|
ref :≈ "https://particle.physics.ucdavis.edu/modernsusy/slides/slideimages/spinorfeynrules.pdf"
|
|
|
|
|
|
|
|
|
|
/-!
|
|
|
|
|
|
|
|
|
|
## Equivalences between Weyl fermion vector spaces.
|
|
|
|
|
|
|
|
|
|
-/
|
2024-09-16 07:40:15 -04:00
|
|
|
|
|
2024-09-15 19:01:34 -04:00
|
|
|
|
informal_definition leftHandedWeylFermionAltEquiv where
|
|
|
|
|
math :≈ "The linear equiv between leftHandedWeylFermion and altLeftHandedWeylFermion given
|
2024-09-16 10:07:40 -04:00
|
|
|
|
by multiplying an element of rightHandedWeylFermion by the matrix `εᵃ⁰ᵃ¹ = !![0, 1; -1, 0]]`."
|
2024-09-16 05:32:40 -04:00
|
|
|
|
deps :≈ [`leftHandedWeylFermion, `altLeftHandedWeylFermion]
|
2024-09-15 19:01:34 -04:00
|
|
|
|
|
|
|
|
|
informal_lemma leftHandedWeylFermionAltEquiv_equivariant where
|
|
|
|
|
math :≈ "The linear equiv leftHandedWeylFermionAltEquiv is equivariant with respect to the
|
|
|
|
|
action of SL(2,C) on leftHandedWeylFermion and altLeftHandedWeylFermion."
|
2024-09-16 05:32:40 -04:00
|
|
|
|
deps :≈ [`leftHandedWeylFermionAltEquiv]
|
2024-09-15 19:01:34 -04:00
|
|
|
|
|
|
|
|
|
informal_definition rightHandedWeylFermionAltEquiv where
|
|
|
|
|
math :≈ "The linear equiv between rightHandedWeylFermion and altRightHandedWeylFermion given
|
2024-09-16 10:07:40 -04:00
|
|
|
|
by multiplying an element of rightHandedWeylFermion by the matrix `εᵃ⁰ᵃ¹ = !![0, 1; -1, 0]]`"
|
2024-09-16 07:40:15 -04:00
|
|
|
|
deps :≈ [`rightHandedWeylFermion, `altRightHandedWeylFermion]
|
2024-09-15 19:01:34 -04:00
|
|
|
|
|
|
|
|
|
informal_lemma rightHandedWeylFermionAltEquiv_equivariant where
|
|
|
|
|
math :≈ "The linear equiv rightHandedWeylFermionAltEquiv is equivariant with respect to the
|
|
|
|
|
action of SL(2,C) on rightHandedWeylFermion and altRightHandedWeylFermion."
|
2024-09-16 07:40:15 -04:00
|
|
|
|
deps :≈ [`rightHandedWeylFermionAltEquiv]
|
2024-09-16 13:41:52 -04:00
|
|
|
|
|
|
|
|
|
/-!
|
|
|
|
|
|
|
|
|
|
## Contraction of Weyl fermions.
|
|
|
|
|
|
|
|
|
|
-/
|
|
|
|
|
|
|
|
|
|
informal_definition leftAltWeylFermionContraction where
|
|
|
|
|
math :≈ "The linear map from leftHandedWeylFermion ⊗ altLeftHandedWeylFermion to ℂ given by
|
|
|
|
|
summing over components of leftHandedWeylFermion and altLeftHandedWeylFermion in the
|
|
|
|
|
standard basis (i.e. the dot product)."
|
|
|
|
|
physics :≈ "The contraction of a left-handed Weyl fermion with a right-handed Weyl fermion.
|
|
|
|
|
In index notation this is ψ_a φ^a."
|
|
|
|
|
ref :≈ "https://particle.physics.ucdavis.edu/modernsusy/slides/slideimages/spinorfeynrules.pdf"
|
|
|
|
|
deps :≈ [``leftHandedWeylFermion, ``altLeftHandedWeylFermion]
|
|
|
|
|
|
|
|
|
|
informal_lemma leftAltWeylFermionContraction_invariant where
|
|
|
|
|
math :≈ "The contraction leftAltWeylFermionContraction is invariant with respect to
|
|
|
|
|
the action of SL(2,C) on leftHandedWeylFermion and altLeftHandedWeylFermion."
|
|
|
|
|
deps :≈ [`leftAltWeylFermionContraction]
|