Update Basic.lean

This commit is contained in:
Pietro Monticone 2024-06-08 03:53:42 +02:00
parent 2e82d598ab
commit 776bce19fe

View file

@ -75,7 +75,7 @@ lemma toHiggsVec_smooth (φ : higgsField) : Smooth 𝓘(, spaceTime) 𝓘(
exact h1
lemma toField_toHiggsVec_apply (φ : higgsField) (x : spaceTime) :
(φ.toHiggsVec x).toField x = φ x := rfl
(φ.toHiggsVec x).toField x = φ x := rfl
lemma higgsVecToFin2_toHiggsVec (φ : higgsField) :
higgsVecToFin2 ∘ φ.toHiggsVec = φ := rfl