refactor: Some lint
This commit is contained in:
parent
af1db2b6cb
commit
2681709f93
2 changed files with 2 additions and 2 deletions
|
@ -5,7 +5,6 @@ Authors: Joseph Tooby-Smith
|
|||
-/
|
||||
import HepLean.SpaceTime.LorentzVector.Basic
|
||||
import Mathlib.CategoryTheory.Limits.FintypeCat
|
||||
import LeanCopilot
|
||||
/-!
|
||||
|
||||
# Lorentz Tensors
|
||||
|
@ -158,6 +157,7 @@ lemma congrSet_refl : @congrSet d _ _ (Equiv.refl X) = Equiv.refl _ := by
|
|||
## Rising and lowering indices
|
||||
|
||||
Rising or lowering an index corresponds to changing the color of that index.
|
||||
|
||||
-/
|
||||
|
||||
/-! TODO: Define the rising and lowering of indices using contraction with the metric. -/
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue