refactor: Spelling

This commit is contained in:
jstoobysmith 2025-02-07 15:43:59 +00:00
parent b82791d671
commit f8f1e1757f
25 changed files with 80 additions and 80 deletions

View file

@ -6,7 +6,7 @@ Authors: Joseph Tooby-Smith
import Mathlib.Algebra.BigOperators.Group.Finset
/-!
# Creation and annihlation parts of fields
# Creation and annihilation parts of fields
-/
@ -33,8 +33,8 @@ instance : Fintype CreateAnnihilate where
lemma eq_create_or_annihilate (φ : CreateAnnihilate) : φ = create φ = annihilate := by
cases φ <;> simp
/-- The normal ordering on creation and annihlation operators.
Under this relation, `normalOrder a b` is false only if `a` is annihlate and `b` is create. -/
/-- The normal ordering on creation and annihilation operators.
Under this relation, `normalOrder a b` is false only if `a` is annihilate and `b` is create. -/
def normalOrder : CreateAnnihilate → CreateAnnihilate → Prop
| create, _ => True
| annihilate, annihilate => True