Skip to content

Commit

Permalink
Merge pull request #31 from pitmonticone/master
Browse files Browse the repository at this point in the history
Fix typos in docstrings
  • Loading branch information
jstoobysmith authored May 20, 2024
2 parents 926653a + ee3c758 commit bdb960b
Show file tree
Hide file tree
Showing 12 changed files with 24 additions and 24 deletions.
6 changes: 3 additions & 3 deletions HepLean/AnomalyCancellation/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -77,7 +77,7 @@ namespace ACCSystemLinear
structure LinSols (χ : ACCSystemLinear) where
/-- The underlying charge. -/
val : χ.1.charges
/-- The condition that the charge satifies the linear ACCs. -/
/-- The condition that the charge satisfies the linear ACCs. -/
linearSol : ∀ i : Fin χ.numberLinear, χ.linearACCs i val = 0

/-- Two solutions are equal if the underlying charges are equal. -/
Expand Down Expand Up @@ -172,7 +172,7 @@ namespace ACCSystemQuad

/-- The type of solutions to the linear and quadratic ACCs. -/
structure QuadSols (χ : ACCSystemQuad) extends χ.LinSols where
/-- The condition that the charge satifies the quadratic ACCs. -/
/-- The condition that the charge satisfies the quadratic ACCs. -/
quadSol : ∀ i : Fin χ.numberQuadratic, (χ.quadraticACCs i) val = 0

/-- Two `QuadSols` are equal if the underlying charges are equal. -/
Expand Down Expand Up @@ -225,7 +225,7 @@ namespace ACCSystem

/-- The type of solutions to the anomaly cancellation conditions. -/
structure Sols (χ : ACCSystem) extends χ.QuadSols where
/-- The condition that the charge satifies the cubic ACC. -/
/-- The condition that the charge satisfies the cubic ACC. -/
cubicSol : χ.cubicACC val = 0

/-- Two solutions are equal if the underlying charges are equal. -/
Expand Down
2 changes: 1 addition & 1 deletion HepLean/AnomalyCancellation/MSSMNu/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -206,7 +206,7 @@ lemma accSU2_ext {S T : MSSMCharges.charges}
rw [hd, hu]
rfl

/-- The anomaly cancelation condition for SU(3) anomaly. -/
/-- The anomaly cancellation condition for SU(3) anomaly. -/
@[simp]
def accSU3 : MSSMCharges.charges →ₗ[ℚ] ℚ where
toFun S := ∑ i, (2 * (Q S i) + (U S i) + (D S i))
Expand Down
2 changes: 1 addition & 1 deletion HepLean/AnomalyCancellation/MSSMNu/HyperCharge.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Mathlib.Tactic.Polyrith
/-!
# Hypercharge in MSSM.
Relavent definitions for the MSSM hypercharge.
Relevant definitions for the MSSM hypercharge.
-/

Expand Down
2 changes: 1 addition & 1 deletion HepLean/AnomalyCancellation/PureU1/Even/LineInCubic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -67,7 +67,7 @@ lemma line_in_cubic_P_P_P! {S : (PureU1 (2 * n.succ)).LinSols} (h : lineInCubic
linear_combination 2 / 3 * (lineInCubic_expand h g f hS 1 1) -
(lineInCubic_expand h g f hS 1 2) / 6

/-- We say a `LinSol` satifies `lineInCubicPerm` if all its permutations satsify `lineInCubic`. -/
/-- We say a `LinSol` satisfies `lineInCubicPerm` if all its permutations satisfy `lineInCubic`. -/
def lineInCubicPerm (S : (PureU1 (2 * n.succ)).LinSols) : Prop :=
∀ (M : (FamilyPermutations (2 * n.succ)).group ),
lineInCubic ((FamilyPermutations (2 * n.succ)).linSolRep M S)
Expand Down
4 changes: 2 additions & 2 deletions HepLean/AnomalyCancellation/PureU1/LineInPlaneCond.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ import Mathlib.RepresentationTheory.Basic
/-!
# Line in plane condition
We say a `LinSol` satifies the `line in plane` condition if for all distinct `i1`, `i2`, `i3` in
We say a `LinSol` satisfies the `line in plane` condition if for all distinct `i1`, `i2`, `i3` in
`Fin n`, we have
`S i1 = S i2` or `S i1 = - S i2` or `2 S i3 + S i1 + S i2 = 0`.
Expand All @@ -21,7 +21,7 @@ The main reference for this material is
- https://arxiv.org/pdf/1912.04804.pdf
We will show that `n ≥ 4` the `line in plane` condition on solutions inplies the
We will show that `n ≥ 4` the `line in plane` condition on solutions implies the
`constAbs` condition.
-/
Expand Down
2 changes: 1 addition & 1 deletion HepLean/AnomalyCancellation/PureU1/Odd/BasisLinear.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ import Mathlib.Logic.Equiv.Fin
/-!
# Basis of `LinSols` in the odd case
We give a basis of `LinSols` in the odd case. This basis has the special propoerty
We give a basis of `LinSols` in the odd case. This basis has the special property
that splits into two planes on which every point is a solution to the ACCs.
-/
universe v u
Expand Down
8 changes: 4 additions & 4 deletions HepLean/AnomalyCancellation/PureU1/Odd/LineInCubic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -16,10 +16,10 @@ import Mathlib.RepresentationTheory.Basic
# Line In Cubic Odd case
We say that a linear solution satisfies the `lineInCubic` property
if the line through that point and through the two different planes formed by the baisis of
if the line through that point and through the two different planes formed by the basis of
`LinSols` lies in the cubic.
We show that for a solution all its permutations satsfiy this property,
We show that for a solution all its permutations satisfy this property,
then the charge must be zero.
The main reference for this file is:
Expand All @@ -34,7 +34,7 @@ open BigOperators
variable {n : ℕ}
open VectorLikeOddPlane

/-- A property on `LinSols`, statified if every point on the line between the two planes
/-- A property on `LinSols`, satisfied if every point on the line between the two planes
in the basis through that point is in the cubic. -/
def lineInCubic (S : (PureU1 (2 * n + 1)).LinSols) : Prop :=
∀ (g f : Fin n → ℚ) (_ : S.val = Pa g f) (a b : ℚ) ,
Expand Down Expand Up @@ -64,7 +64,7 @@ lemma line_in_cubic_P_P_P! {S : (PureU1 (2 * n + 1)).LinSols} (h : lineInCubic S



/-- We say a `LinSol` satifies `lineInCubicPerm` if all its permutations satsify `lineInCubic`. -/
/-- We say a `LinSol` satisfies `lineInCubicPerm` if all its permutations satisfy `lineInCubic`. -/
def lineInCubicPerm (S : (PureU1 (2 * n + 1)).LinSols) : Prop :=
∀ (M : (FamilyPermutations (2 * n + 1)).group ),
lineInCubic ((FamilyPermutations (2 * n + 1)).linSolRep M S)
Expand Down
4 changes: 2 additions & 2 deletions HepLean/AnomalyCancellation/SM/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,15 +13,15 @@ import Mathlib.Logic.Equiv.Fin
/-!
# Anomaly cancellation conditions for n family SM.
We define the ACC system for the Standard Model with`n`-famlies and no RHN.
We define the ACC system for the Standard Model with`n`-families and no RHN.
-/

universe v u
open Nat
open BigOperators

/-- Aassociate to each (including RHN) SM fermion a set of charges-/
/-- Associate to each (including RHN) SM fermion a set of charges-/
@[simps!]
def SMCharges (n : ℕ) : ACCSystemCharges := ACCSystemChargesMk (5 * n)

Expand Down
6 changes: 3 additions & 3 deletions HepLean/AnomalyCancellation/SM/FamilyMaps.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ import HepLean.AnomalyCancellation.SM.Basic
/-!
# Family maps for the Standard Model ACCs
We define the a series of maps between the charges for different numbers of famlies.
We define the a series of maps between the charges for different numbers of families.
-/

Expand Down Expand Up @@ -84,7 +84,7 @@ other charges zero. -/
def familyEmbedding (m n : ℕ) : (SMCharges m).charges →ₗ[ℚ] (SMCharges n).charges :=
chargesMapOfSpeciesMap (speciesEmbed m n)

/-- For species, the embeddding of the `1`-family charges into the `n`-family charges in
/-- For species, the embedding of the `1`-family charges into the `n`-family charges in
a universal manor. -/
@[simps!]
def speciesFamilyUniversial (n : ℕ) :
Expand All @@ -98,7 +98,7 @@ def speciesFamilyUniversial (n : ℕ) :
simp [HSMul.hSMul]
--rw [show Rat.cast a = a from rfl]

/-- The embeddding of the `1`-family charges into the `n`-family charges in
/-- The embedding of the `1`-family charges into the `n`-family charges in
a universal manor. -/
def familyUniversal ( n : ℕ) : (SMCharges 1).charges →ₗ[ℚ] (SMCharges n).charges :=
chargesMapOfSpeciesMap (speciesFamilyUniversial n)
Expand Down
4 changes: 2 additions & 2 deletions HepLean/AnomalyCancellation/SM/NoGrav/One/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ import HepLean.AnomalyCancellation.SM.NoGrav.One.LinearParameterization
The main result of this file is the conclusion of this paper:
https://arxiv.org/abs/1907.00514
That eveery solution to the ACCs without gravity satifies for free the gravitational anomaly.
That eveery solution to the ACCs without gravity satisfies for free the gravitational anomaly.
-/

universe v u
Expand Down Expand Up @@ -67,7 +67,7 @@ lemma accGrav_Q_neq_zero {S : (SMNoGrav 1).Sols} (hQ : Q S.val (0 : Fin 1) ≠ 0
rw [← hS']
exact S'.grav_of_cubic hC FLTThree

/-- Any solution to the ACCs without gravity satifies the gravitational ACC. -/
/-- Any solution to the ACCs without gravity satisfies the gravitational ACC. -/
theorem accGravSatisfied {S : (SMNoGrav 1).Sols} (FLTThree : FermatLastTheoremWith ℚ 3) :
accGrav S.val = 0 := by
by_cases hQ : Q S.val (0 : Fin 1)= 0
Expand Down
6 changes: 3 additions & 3 deletions HepLean/AnomalyCancellation/SMNu/FamilyMaps.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ import HepLean.AnomalyCancellation.SMNu.Basic
/-!
# Family maps for the Standard Model for RHN ACCs
We define the a series of maps between the charges for different numbers of famlies.
We define the a series of maps between the charges for different numbers of families.
-/

Expand Down Expand Up @@ -89,7 +89,7 @@ other charges zero. -/
def familyEmbedding (m n : ℕ) : (SMνCharges m).charges →ₗ[ℚ] (SMνCharges n).charges :=
chargesMapOfSpeciesMap (speciesEmbed m n)

/-- For species, the embeddding of the `1`-family charges into the `n`-family charges in
/-- For species, the embedding of the `1`-family charges into the `n`-family charges in
a universal manor. -/
@[simps!]
def speciesFamilyUniversial (n : ℕ) :
Expand All @@ -103,7 +103,7 @@ def speciesFamilyUniversial (n : ℕ) :
simp [HSMul.hSMul]
-- rw [show Rat.cast a = a from rfl]

/-- The embeddding of the `1`-family charges into the `n`-family charges in
/-- The embedding of the `1`-family charges into the `n`-family charges in
a universal manor. -/
def familyUniversal (n : ℕ) : (SMνCharges 1).charges →ₗ[ℚ] (SMνCharges n).charges :=
chargesMapOfSpeciesMap (speciesFamilyUniversial n)
Expand Down
2 changes: 1 addition & 1 deletion HepLean/FlavorPhysics/CKMMatrix/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ import Mathlib.Tactic.Polyrith
/-!
# The CKM Matrix
The definition of the type of CKM matries as unitary $3×3$-matries.
The definition of the type of CKM matrices as unitary $3×3$-matrices.
An equivalence relation on CKM matrices is defined, where two matrices are equivalent if they are
related by phase shifts.
Expand Down

0 comments on commit bdb960b

Please sign in to comment.