PhysLean/HepLean/BeyondTheStandardModel/PatiSalam/Basic.lean
2024-09-19 06:07:27 -04:00

65 lines
2.5 KiB
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

/-
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.StandardModel.Basic
import HepLean.Meta.Informal
/-!
# The Pati-Salam Model
The Pati-Salam model is a grand unified theory that unifies the Standard Model gauge group into
`SU(4) x SU(2) x SU(2)`.
This file current contains informal-results about the Pati-Salam group.
-/
namespace PatiSalam
/-!
## The Pati-Salam gauge group.
-/
informal_definition GaugeGroupI where
math :≈ "The group `SU(4) x SU(2) x SU(2)`."
physics :≈ "The gauge group of the Pati-Salam model (unquotiented by ℤ₂)."
informal_definition embedSM where
physics :≈ "The embedding of the Standard Model gauge group into the Pati-Salam gauge group."
math :≈ "The group homomorphism `SU(3) x SU(2) x U(1) -> SU(4) x SU(2) x SU(2)`
taking (h, g, α) to (blockdiag (α h, α ^ (-3)), g, diag(α ^ (3), α ^(-3)))."
ref :≈ "Page 54 of https://math.ucr.edu/home/baez/guts.pdf"
deps :≈ [``GaugeGroupI, ``StandardModel.GaugeGroupI]
informal_definition gaugeGroupISpinEquiv where
math :≈ "The equivalence between `GaugeGroupI` and `Spin(6) × Spin(4)`."
deps :≈ [``GaugeGroupI]
informal_definition gaugeGroup₂SubGroup where
physics :≈ "The ℤ₂-subgroup of the un-quotiented gauge group which acts trivially on
all particles in the standard model."
math :≈ "The ℤ₂-subgroup of ``GaugeGroupI with the non-trivial element (-1, -1, -1)."
ref :≈ "https://math.ucr.edu/home/baez/guts.pdf"
deps :≈ [``GaugeGroupI]
informal_definition GaugeGroup₂ where
physics :≈ "The gauge group of the Pati-Salam model with a ℤ₂ quotient."
math :≈ "The quotient of ``GaugeGroupI by the ℤ₂-subgroup `gaugeGroup₂SubGroup`."
ref :≈ "https://math.ucr.edu/home/baez/guts.pdf"
deps :≈ [``GaugeGroupI, ``gaugeGroup₂SubGroup]
informal_lemma sm_₆_factor_through_gaugeGroup₂SubGroup where
math :≈ "The group ``StandardModel.gaugeGroup₆SubGroup under the homomorphism ``embedSM factors
through the subgroup ``gaugeGroup₂SubGroup."
deps :≈ [``embedSM, ``StandardModel.gaugeGroup₆SubGroup, ``gaugeGroup₂SubGroup]
informal_definition embedSM₆To₂ where
math :≈ "The group homomorphism from ``StandardModel.GaugeGroup₆ to ``GaugeGroup
induced by ``embedSM."
deps :≈ [``embedSM, ``StandardModel.GaugeGroup₆, ``GaugeGroup₂,
``sm_₆_factor_through_gaugeGroup₂SubGroup]
end PatiSalam