2024-04-18 10:50:21 -04:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
2024-07-12 16:39:44 -04:00
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
2024-04-18 10:50:21 -04:00
|
|
|
|
Authors: Joseph Tooby-Smith
|
|
|
|
|
-/
|
2024-06-25 07:06:32 -04:00
|
|
|
|
import HepLean.AnomalyCancellation.PureU1.Basic
|
2024-04-18 10:50:21 -04:00
|
|
|
|
/-!
|
|
|
|
|
# The Pure U(1) case with 1 fermion
|
|
|
|
|
|
|
|
|
|
We show that in this case the charge must be zero.
|
|
|
|
|
-/
|
|
|
|
|
|
|
|
|
|
universe v u
|
|
|
|
|
|
|
|
|
|
open Nat
|
2024-07-12 11:23:02 -04:00
|
|
|
|
open Finset
|
2024-04-18 10:50:21 -04:00
|
|
|
|
|
|
|
|
|
namespace PureU1
|
|
|
|
|
|
|
|
|
|
variable {n : ℕ}
|
|
|
|
|
|
|
|
|
|
namespace One
|
|
|
|
|
|
|
|
|
|
theorem solEqZero (S : (PureU1 1).LinSols) : S = 0 := by
|
|
|
|
|
apply ACCSystemLinear.LinSols.ext
|
|
|
|
|
have hLin := pureU1_linear S
|
2024-10-12 08:16:24 +00:00
|
|
|
|
simp only [succ_eq_add_one, reduceAdd, PureU1_numberCharges, univ_unique, Fin.default_eq_zero,
|
|
|
|
|
Fin.isValue, sum_singleton] at hLin
|
2024-04-18 10:50:21 -04:00
|
|
|
|
funext i
|
2024-10-12 08:16:24 +00:00
|
|
|
|
simp only [PureU1_numberCharges] at i
|
2024-06-13 16:49:01 -04:00
|
|
|
|
rw [show i = (0 : Fin 1) from Fin.fin_one_eq_zero i]
|
2024-04-18 10:50:21 -04:00
|
|
|
|
exact hLin
|
|
|
|
|
|
|
|
|
|
end One
|
|
|
|
|
|
|
|
|
|
end PureU1
|