refactor: Some properties of field specifications (#285)

* refactor: Fix field struct defn.

* rename: FieldStruct to FieldSpecification

* feat: Add examples of field specifications

* docs: Slight improvement of module docs
This commit is contained in:
Joseph Tooby-Smith 2025-01-21 06:11:47 +00:00 committed by GitHub
parent bb1db930b5
commit b5c987180a
No known key found for this signature in database
GPG key ID: B5690EEEBB952194
29 changed files with 153 additions and 126 deletions

View file

@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import HepLean.PerturbationTheory.Algebras.StateAlgebra.Basic
import HepLean.PerturbationTheory.FieldStruct.CrAnSection
import HepLean.PerturbationTheory.FieldSpecification.CrAnSection
/-!
# Creation and annihlation free-algebra
@ -31,15 +31,15 @@ super commutation relations between creation and annihilation operators.
-/
namespace FieldStruct
variable {𝓕 : FieldStruct}
namespace FieldSpecification
variable {𝓕 : FieldSpecification}
/-- The creation and annihlation free-algebra.
The free algebra generated by `CrAnStates`,
that is a position based states or assymptotic states with a specification of
whether the state is a creation or annihlation state.
As a module `CrAnAlgebra` is spanned by lists of `CrAnStates`. -/
abbrev CrAnAlgebra (𝓕 : FieldStruct) : Type := FreeAlgebra 𝓕.CrAnStates
abbrev CrAnAlgebra (𝓕 : FieldSpecification) : Type := FreeAlgebra 𝓕.CrAnStates
namespace CrAnAlgebra
@ -263,4 +263,4 @@ noncomputable def smulLinearMap (c : ) : CrAnAlgebra 𝓕 →ₗ[] CrAnAlg
end CrAnAlgebra
end FieldStruct
end FieldSpecification