2024-05-09 15:09:14 -04:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license.
|
|
|
|
|
Authors: Joseph Tooby-Smith
|
|
|
|
|
-/
|
2024-06-25 07:06:32 -04:00
|
|
|
|
import HepLean.SpaceTime.Basic
|
2024-05-09 15:09:14 -04:00
|
|
|
|
import HepLean.StandardModel.Basic
|
|
|
|
|
import HepLean.StandardModel.HiggsBoson.TargetSpace
|
|
|
|
|
import Mathlib.Data.Complex.Exponential
|
|
|
|
|
import Mathlib.Tactic.Polyrith
|
|
|
|
|
import Mathlib.Geometry.Manifold.VectorBundle.Basic
|
|
|
|
|
import Mathlib.Geometry.Manifold.VectorBundle.SmoothSection
|
|
|
|
|
import Mathlib.Geometry.Manifold.Instances.Real
|
|
|
|
|
import Mathlib.RepresentationTheory.Basic
|
|
|
|
|
import Mathlib.Analysis.InnerProductSpace.Basic
|
|
|
|
|
import Mathlib.Analysis.InnerProductSpace.Adjoint
|
|
|
|
|
import Mathlib.Geometry.Manifold.ContMDiff.Product
|
|
|
|
|
import Mathlib.Algebra.QuadraticDiscriminant
|
|
|
|
|
/-!
|
|
|
|
|
# The Higgs field
|
|
|
|
|
|
|
|
|
|
This file defines the basic properties for the higgs field in the standard model.
|
|
|
|
|
|
|
|
|
|
## References
|
|
|
|
|
|
|
|
|
|
- We use conventions given in: https://pdg.lbl.gov/2019/reviews/rpp2019-rev-higgs-boson.pdf
|
|
|
|
|
|
|
|
|
|
-/
|
|
|
|
|
universe v u
|
|
|
|
|
namespace StandardModel
|
|
|
|
|
noncomputable section
|
|
|
|
|
|
|
|
|
|
open Manifold
|
|
|
|
|
open Matrix
|
|
|
|
|
open Complex
|
|
|
|
|
open ComplexConjugate
|
2024-06-26 11:54:02 -04:00
|
|
|
|
open SpaceTime
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
|
|
|
|
/-- The trivial vector bundle 𝓡² × ℂ². (TODO: Make associated bundle.) -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
abbrev HiggsBundle := Bundle.Trivial SpaceTime HiggsVec
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
instance : SmoothVectorBundle HiggsVec HiggsBundle SpaceTime.asSmoothManifold :=
|
|
|
|
|
Bundle.Trivial.smoothVectorBundle HiggsVec 𝓘(ℝ, SpaceTime)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
|
|
|
|
/-- A higgs field is a smooth section of the higgs bundle. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
abbrev HiggsField : Type := SmoothSection SpaceTime.asSmoothManifold HiggsVec HiggsBundle
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
|
|
|
|
instance : NormedAddCommGroup (Fin 2 → ℂ) := by
|
|
|
|
|
exact Pi.normedAddCommGroup
|
|
|
|
|
|
|
|
|
|
/-- Given a vector `ℂ²` the constant higgs field with value equal to that
|
|
|
|
|
section. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
noncomputable def HiggsVec.toField (φ : HiggsVec) : HiggsField where
|
2024-06-08 03:47:16 +02:00
|
|
|
|
toFun := fun _ ↦ φ
|
2024-05-09 15:09:14 -04:00
|
|
|
|
contMDiff_toFun := by
|
|
|
|
|
intro x
|
|
|
|
|
rw [Bundle.contMDiffAt_section]
|
|
|
|
|
exact smoothAt_const
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
namespace HiggsField
|
2024-05-09 15:09:14 -04:00
|
|
|
|
open Complex Real
|
|
|
|
|
|
|
|
|
|
/-- Given a `higgsField`, the corresponding map from `spaceTime` to `higgsVec`. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
def toHiggsVec (φ : HiggsField) : SpaceTime → HiggsVec := φ
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma toHiggsVec_smooth (φ : HiggsField) : Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, HiggsVec) φ.toHiggsVec := by
|
2024-05-09 15:09:14 -04:00
|
|
|
|
intro x0
|
|
|
|
|
have h1 := φ.contMDiff x0
|
|
|
|
|
rw [Bundle.contMDiffAt_section] at h1
|
|
|
|
|
have h2 :
|
2024-06-26 11:54:02 -04:00
|
|
|
|
(fun x => ((trivializationAt HiggsVec (Bundle.Trivial SpaceTime HiggsVec) x0)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
{ proj := x, snd := φ x }).2) = φ := by
|
|
|
|
|
rfl
|
|
|
|
|
simp only [h2] at h1
|
|
|
|
|
exact h1
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma toField_toHiggsVec_apply (φ : HiggsField) (x : SpaceTime) :
|
2024-06-08 03:56:15 +02:00
|
|
|
|
(φ.toHiggsVec x).toField x = φ x := rfl
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma higgsVecToFin2ℂ_toHiggsVec (φ : HiggsField) :
|
2024-06-08 03:56:15 +02:00
|
|
|
|
higgsVecToFin2ℂ ∘ φ.toHiggsVec = φ := rfl
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma toVec_smooth (φ : HiggsField) : Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, Fin 2 → ℂ) φ :=
|
2024-06-08 03:49:34 +02:00
|
|
|
|
smooth_higgsVecToFin2ℂ.comp φ.toHiggsVec_smooth
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma apply_smooth (φ : HiggsField) :
|
|
|
|
|
∀ i, Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, ℂ) (fun (x : SpaceTime) => (φ x i)) :=
|
2024-06-08 03:47:16 +02:00
|
|
|
|
(smooth_pi_space).mp (φ.toVec_smooth)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma apply_re_smooth (φ : HiggsField) (i : Fin 2):
|
|
|
|
|
Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, ℝ) (reCLM ∘ (fun (x : SpaceTime) => (φ x i))) :=
|
2024-06-08 03:47:16 +02:00
|
|
|
|
(ContinuousLinearMap.smooth reCLM).comp (φ.apply_smooth i)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma apply_im_smooth (φ : HiggsField) (i : Fin 2):
|
|
|
|
|
Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, ℝ) (imCLM ∘ (fun (x : SpaceTime) => (φ x i))) :=
|
2024-06-08 03:47:16 +02:00
|
|
|
|
(ContinuousLinearMap.smooth imCLM).comp (φ.apply_smooth i)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-07 14:37:09 -04:00
|
|
|
|
/-- Given two `higgsField`, the map `spaceTime → ℂ` obtained by taking their inner product. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
def innerProd (φ1 φ2 : HiggsField) : SpaceTime → ℂ := fun x => ⟪φ1 x, φ2 x⟫_ℂ
|
2024-06-07 14:37:09 -04:00
|
|
|
|
|
|
|
|
|
|
2024-05-09 15:09:14 -04:00
|
|
|
|
/-- Given a `higgsField`, the map `spaceTime → ℝ` obtained by taking the square norm of the
|
|
|
|
|
higgs vector. -/
|
|
|
|
|
@[simp]
|
2024-06-26 11:54:02 -04:00
|
|
|
|
def normSq (φ : HiggsField) : SpaceTime → ℝ := fun x => ( ‖φ x‖ ^ 2)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma toHiggsVec_norm (φ : HiggsField) (x : SpaceTime) :
|
2024-05-09 15:09:14 -04:00
|
|
|
|
‖φ x‖ = ‖φ.toHiggsVec x‖ := rfl
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma normSq_expand (φ : HiggsField) :
|
2024-05-09 15:09:14 -04:00
|
|
|
|
φ.normSq = fun x => (conj (φ x 0) * (φ x 0) + conj (φ x 1) * (φ x 1) ).re := by
|
|
|
|
|
funext x
|
2024-06-08 03:47:16 +02:00
|
|
|
|
simp [normSq, add_re, mul_re, conj_re, conj_im, neg_mul, sub_neg_eq_add, @norm_sq_eq_inner ℂ]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma normSq_smooth (φ : HiggsField) : Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, ℝ) φ.normSq := by
|
2024-05-09 15:09:14 -04:00
|
|
|
|
rw [normSq_expand]
|
|
|
|
|
refine Smooth.add ?_ ?_
|
|
|
|
|
simp only [mul_re, conj_re, conj_im, neg_mul, sub_neg_eq_add]
|
|
|
|
|
refine Smooth.add ?_ ?_
|
|
|
|
|
refine Smooth.smul ?_ ?_
|
|
|
|
|
exact φ.apply_re_smooth 0
|
|
|
|
|
exact φ.apply_re_smooth 0
|
|
|
|
|
refine Smooth.smul ?_ ?_
|
|
|
|
|
exact φ.apply_im_smooth 0
|
|
|
|
|
exact φ.apply_im_smooth 0
|
|
|
|
|
simp only [mul_re, conj_re, conj_im, neg_mul, sub_neg_eq_add]
|
|
|
|
|
refine Smooth.add ?_ ?_
|
|
|
|
|
refine Smooth.smul ?_ ?_
|
|
|
|
|
exact φ.apply_re_smooth 1
|
|
|
|
|
exact φ.apply_re_smooth 1
|
|
|
|
|
refine Smooth.smul ?_ ?_
|
|
|
|
|
exact φ.apply_im_smooth 1
|
|
|
|
|
exact φ.apply_im_smooth 1
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma normSq_nonneg (φ : HiggsField) (x : SpaceTime) : 0 ≤ φ.normSq x := by
|
2024-06-08 03:47:16 +02:00
|
|
|
|
simp [normSq, ge_iff_le, norm_nonneg, pow_nonneg]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma normSq_zero (φ : HiggsField) (x : SpaceTime) : φ.normSq x = 0 ↔ φ x = 0 := by
|
2024-06-08 03:47:16 +02:00
|
|
|
|
simp [normSq, ne_eq, OfNat.ofNat_ne_zero, not_false_eq_true, pow_eq_zero_iff, norm_eq_zero]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
|
|
|
|
/-- The Higgs potential of the form `- μ² * |φ|² + λ * |φ|⁴`. -/
|
|
|
|
|
@[simp]
|
2024-06-26 11:54:02 -04:00
|
|
|
|
def potential (φ : HiggsField) (μSq lambda : ℝ ) (x : SpaceTime) : ℝ :=
|
2024-05-09 15:09:14 -04:00
|
|
|
|
- μSq * φ.normSq x + lambda * φ.normSq x * φ.normSq x
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma potential_smooth (φ : HiggsField) (μSq lambda : ℝ) :
|
|
|
|
|
Smooth 𝓘(ℝ, SpaceTime) 𝓘(ℝ, ℝ) (fun x => φ.potential μSq lambda x) := by
|
2024-05-09 15:09:14 -04:00
|
|
|
|
simp only [potential, normSq, neg_mul]
|
2024-06-08 03:47:16 +02:00
|
|
|
|
exact (smooth_const.smul φ.normSq_smooth).neg.add
|
|
|
|
|
((smooth_const.smul φ.normSq_smooth).smul φ.normSq_smooth)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma potential_apply (φ : HiggsField) (μSq lambda : ℝ) (x : SpaceTime) :
|
|
|
|
|
(φ.potential μSq lambda) x = HiggsVec.potential μSq lambda (φ.toHiggsVec x) := by
|
|
|
|
|
simp [HiggsVec.potential, toHiggsVec_norm]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
ring
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
/-- A higgs field is constant if it is equal for all `x` `y` in `spaceTime`. -/
|
2024-06-26 11:54:02 -04:00
|
|
|
|
def IsConst (Φ : HiggsField) : Prop := ∀ x y, Φ x = Φ y
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma isConst_of_higgsVec (φ : HiggsVec) : φ.toField.IsConst := by
|
2024-05-09 15:09:14 -04:00
|
|
|
|
intro x _
|
2024-06-26 11:54:02 -04:00
|
|
|
|
simp [HiggsVec.toField]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma isConst_iff_of_higgsVec (Φ : HiggsField) : Φ.IsConst ↔ ∃ (φ : HiggsVec), Φ = φ.toField :=
|
2024-06-08 03:47:16 +02:00
|
|
|
|
Iff.intro (fun h ↦ ⟨Φ 0, by ext x y; rw [← h x 0]; rfl⟩) (fun ⟨φ, hφ⟩ x y ↦ by subst hφ; rfl)
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma normSq_of_higgsVec (φ : HiggsVec) : φ.toField.normSq = fun x => (norm φ) ^ 2 := by
|
2024-05-09 15:09:14 -04:00
|
|
|
|
funext x
|
2024-06-26 11:54:02 -04:00
|
|
|
|
simp [normSq, HiggsVec.toField]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
lemma potential_of_higgsVec (φ : HiggsVec) (μSq lambda : ℝ) :
|
|
|
|
|
φ.toField.potential μSq lambda = fun _ => HiggsVec.potential μSq lambda φ := by
|
|
|
|
|
simp [HiggsVec.potential]
|
2024-05-09 15:09:14 -04:00
|
|
|
|
unfold potential
|
|
|
|
|
rw [normSq_of_higgsVec]
|
|
|
|
|
ring_nf
|
|
|
|
|
|
2024-06-26 11:54:02 -04:00
|
|
|
|
end HiggsField
|
2024-05-09 15:09:14 -04:00
|
|
|
|
end
|
|
|
|
|
end StandardModel
|