Merge pull request #217 from HEPLean/gitpod

Add .gitpod.yml
This commit is contained in:
Joseph Tooby-Smith 2024-10-31 05:52:23 +00:00 committed by GitHub
commit 76c64ea45b
No known key found for this signature in database
GPG key ID: B5690EEEBB952194
2 changed files with 14 additions and 0 deletions

12
.gitpod.yml Normal file
View file

@ -0,0 +1,12 @@
# This is run when starting a Gitpod workspace on this repository
image: leanprovercommunity/gitpod4
vscode:
extensions:
- leanprover.lean4 # install the Lean 4 VS Code extension
tasks:
- init: |
elan self update
lake exe cache get

View file

@ -52,6 +52,8 @@ lemma coMetric_basis_expand : {η' | μ ν}ᵀ.tensor =
simp only [Fin.isValue, Lorentz.complexCoBasisFin4, Basis.coe_reindex, Function.comp_apply]
rfl
/-- Provides the explicit expansion of the co-metric tensor in terms of the basis elements, as
a tensor tree.-/
lemma coMetric_basis_expand_tree : {η' | μ ν}ᵀ.tensor =
(TensorTree.add (tensorNode (basisVector ![Color.down, Color.down] (fun _ => 0))) <|
TensorTree.add (smul (-1) (tensorNode (basisVector ![Color.down, Color.down] (fun _ => 1)))) <|