refactor: Lint

This commit is contained in:
jstoobysmith 2024-12-03 09:52:11 +00:00
parent da70d65c6d
commit bd2a915e03
4 changed files with 4 additions and 5 deletions

View file

@ -124,7 +124,7 @@ informal_lemma timeOrder_pair where
informal_definition WickMap where
math :≈ "A linear map `vev` from the Wick algebra `A` to the underlying field such that
`vev(...ψd(t)) = 0` and `vev(ψc(t)...) = 0`."
`vev(...ψd(t)) = 0` and `vev(ψc(t)...) = 0`."
physics :≈ "An abstraction of the notion of a vacuum expectation value, containing
the necessary properties for lots of theorems to hold."
deps :≈ [``WickAlgebra, ``WickMonomial]

View file

@ -256,8 +256,8 @@ lemma mem_snoc' {ni : } {i : Fin ni → 𝓔} {n : } {c : Fin n → 𝓔}
(hilej : i < j) → (hb1 : ∀ r, b1 r < i) → (hb2i : ∀ r, b2 r ≠ i) → (hb2j : ∀ r, b2 r ≠ j) →
(hb1' : Fin.snoc b1 i = b1' ∘ Fin.cast hk') →
(hb2' : Fin.snoc b2 j = b2' ∘ Fin.cast hk') →
∃ (w' : WickContract str b1 b2), w = castMaps hk' hb1' hb2' (
contr i j h hilej hb1 hb2i hb2j w') := fun
∃ (w' : WickContract str b1 b2), w = castMaps hk' hb1' hb2'
(contr i j h hilej hb1 hb2i hb2j w') := fun
| string => fun hk' => by
simp at hk'
| contr i' j' h' hilej' hb1' hb2i' hb2j' w' => by

View file

@ -21,5 +21,4 @@ The following reference provides a good resource for Wick contractions of extern
namespace Wick
end Wick

View file

@ -23,7 +23,7 @@ namespace Wick
calculate the corresponding Feynman diagrams.
WARNING: This definition is not yet complete.
-/
-/
structure Species where
/-- The color of Field operators which appear in a theory.
One may wish to call these `half-edges`, however we restrict this terminology