PhysLean/HepLean/StandardModel/Basic.lean

33 lines
866 B
Text
Raw Normal View History

2024-05-03 06:12:59 -04:00
/-
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license.
Authors: Joseph Tooby-Smith
-/
import Mathlib.Data.Complex.Exponential
import Mathlib.Geometry.Manifold.VectorBundle.Basic
import Mathlib.Geometry.Manifold.VectorBundle.SmoothSection
import Mathlib.Geometry.Manifold.Instances.Real
import Mathlib.RepresentationTheory.Basic
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-05-03 06:12:59 -04:00
universe v u
namespace StandardModel
open Manifold
open Matrix
open Complex
open ComplexConjugate
/-- The space-time (TODO: Change to Minkowski.) -/
abbrev spaceTime := EuclideanSpace (Fin 4)
2024-05-06 11:09:37 -04:00
/-- The global gauge group of the standard model. -/
abbrev guageGroup : Type := specialUnitaryGroup (Fin 3) ×
specialUnitaryGroup (Fin 2) × unitary
2024-05-03 06:12:59 -04:00
end StandardModel