2024-08-20 09:27:51 -04:00
|
|
|
/-
|
|
|
|
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
Authors: Joseph Tooby-Smith
|
|
|
|
-/
|
|
|
|
import Mathlib.LinearAlgebra.StdBasis
|
2024-09-04 10:01:14 -04:00
|
|
|
import HepLean.Tensors.Basic
|
2024-08-20 09:27:51 -04:00
|
|
|
import Mathlib.LinearAlgebra.DirectSum.Finsupp
|
|
|
|
import Mathlib.LinearAlgebra.Finsupp
|
|
|
|
/-!
|
|
|
|
|
|
|
|
# Dualizing indices of Einstein tensors
|
|
|
|
|
|
|
|
Dualizing indices (the more general notion of rising and lowering indices) does
|
|
|
|
nothing for Einstein tensors, since they only have one color of index.
|
|
|
|
|
|
|
|
The aim of this file is show this result.
|
|
|
|
|
|
|
|
This file is currently a stub.
|
|
|
|
-/
|
|
|
|
/-! TODO: Prove dualizing indices for Einstein tensors does nothing. -/
|