2024-05-03 06:12:59 -04:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
2024-07-12 16:39:44 -04:00
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
2024-05-03 06:12:59 -04:00
|
|
|
|
Authors: Joseph Tooby-Smith
|
|
|
|
|
-/
|
|
|
|
|
import Mathlib.Data.Complex.Exponential
|
|
|
|
|
import Mathlib.Geometry.Manifold.Instances.Real
|
2024-05-09 08:16:23 -04:00
|
|
|
|
import Mathlib.LinearAlgebra.Matrix.ToLin
|
2024-05-06 11:09:37 -04:00
|
|
|
|
/-!
|
|
|
|
|
# The Standard Model
|
2024-05-03 06:12:59 -04:00
|
|
|
|
|
2024-05-06 11:09:37 -04:00
|
|
|
|
This file defines the basic properties of the standard model in particle physics.
|
|
|
|
|
|
|
|
|
|
-/
|
2024-07-09 16:31:26 -04:00
|
|
|
|
/-! TODO: Redefine the gauge group as a quotient of SU(3) x SU(2) x U(1) by a subgroup of ℤ₆. -/
|
2024-05-03 06:12:59 -04:00
|
|
|
|
universe v u
|
|
|
|
|
namespace StandardModel
|
|
|
|
|
|
|
|
|
|
open Manifold
|
|
|
|
|
open Matrix
|
|
|
|
|
open Complex
|
|
|
|
|
open ComplexConjugate
|
|
|
|
|
|
2024-07-09 19:22:16 -04:00
|
|
|
|
/-- The global gauge group of the standard model. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
abbrev GaugeGroup : Type :=
|
2024-05-09 15:09:14 -04:00
|
|
|
|
specialUnitaryGroup (Fin 3) ℂ × specialUnitaryGroup (Fin 2) ℂ × unitary ℂ
|
2024-05-09 08:16:23 -04:00
|
|
|
|
|
2024-05-03 06:12:59 -04:00
|
|
|
|
end StandardModel
|