refactor: lint

This commit is contained in:
jstoobysmith 2025-03-21 11:12:58 -04:00
parent 1d7eeb7c4e
commit 08f0a01e9d
5 changed files with 5 additions and 9 deletions

View file

@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import PhysLean.Electromagnetism.Basic
import PhysLean.Relativity.SpaceTime.Basic
/-!
# Maxwell's equations

View file

@ -4,10 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import PhysLean.Relativity.SpaceTime.Basic
import Mathlib.Tactic.Polyrith
import Mathlib.Geometry.Manifold.VectorBundle.SmoothSection
import Mathlib.Geometry.Manifold.Instances.Real
import PhysLean.Meta.Informal.Basic
/-!
# The Higgs field

View file

@ -4,10 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import PhysLean.Particles.StandardModel.HiggsBoson.Basic
import Mathlib.RepresentationTheory.Basic
import PhysLean.Particles.StandardModel.Basic
import PhysLean.Particles.StandardModel.Representations
import Mathlib.Analysis.InnerProductSpace.Adjoint
/-!
# The action of the gauge group on the Higgs field

View file

@ -82,9 +82,11 @@ lemma toCoord_tprod {d : } (p : (i : Fin 1) →
((Lorentz.contrBasisFin d).repr (p 0))
(indexEquiv.symm i 0) := by
rw [toCoord_apply]
simp
simp only [Nat.succ_eq_add_one, Nat.reduceAdd, C_eq_color, OverColor.mk_left, Functor.id_obj,
OverColor.mk_hom, Equiv.piCongrLeft'_apply, Finsupp.equivFunOnFinite_apply, Fin.isValue]
erw [TensorSpecies.TensorBasis.tensorBasis_repr_tprod]
simp
simp only [Finset.univ_unique, Fin.default_eq_zero, Fin.isValue, C_eq_color,
Finset.prod_singleton, cons_val_zero]
rfl
lemma tensorNode_repr_apply {d : } (p : Vector d)
@ -294,7 +296,6 @@ lemma action_apply_eq_sum (i : Fin 1 ⊕ Fin d) (Λ : LorentzGroup d) (p : Vecto
rw [← mul_assoc, mul_comm _ r, mul_assoc]
rw [← Finset.mul_sum]
congr
have hl : (𝟭 Type).obj (OverColor.mk ![Color.up]).left = Fin 1 := by rfl
simp_all only [Nat.succ_eq_add_one, OverColor.mk_left, _root_.zero_add, Functor.id_obj,
C_eq_color, OverColor.mk_hom]
erw [toCoord_tprod]

View file

@ -54,7 +54,7 @@ lemma contrBasisFin_toFin1d {d : } (i : Fin (1 + d)) :
simp only [contrBasisFin, Basis.reindex_apply, contrBasis_toFin1d, Basis.coe_ofEquivFun]
lemma contrBasisFin_repr_apply {d : } (p : Contr d) (i : Fin (1 + d)) :
(contrBasisFin d).repr p i = p.val (finSumFinEquiv.symm i) := by rfl
(contrBasisFin d).repr p i = p.val (finSumFinEquiv.symm i) := by rfl
/-- The representation of contravariant Lorentz vectors forms a topological space, induced
by its equivalence to `Fin 1 ⊕ Fin d → `. -/