refactor: Lint
This commit is contained in:
parent
0a90f67a46
commit
4632b66854
4 changed files with 44 additions and 66 deletions
|
@ -19,6 +19,7 @@ open CategoryTheory
|
|||
open FeynmanDiagram
|
||||
open PreFeynmanRule
|
||||
|
||||
/-- The pre-Feynman rules for `Phi^4` theory. -/
|
||||
@[simps!]
|
||||
def phi4PreFeynmanRules : PreFeynmanRule where
|
||||
/- There is only 1 type of `half-edge`. -/
|
||||
|
@ -65,19 +66,5 @@ instance : IsFinitePreFeynmanRule phi4PreFeynmanRules where
|
|||
| 0 => instDecidableEqFin _
|
||||
|
||||
|
||||
def figureEight : FeynmanDiagram phi4PreFeynmanRules :=
|
||||
mk' ![0, 0] ![1] ![⟨0, 0, 0⟩, ⟨0, 0, 0⟩, ⟨0, 1, 0⟩, ⟨0, 1, 0⟩] (by decide)
|
||||
|
||||
instance : IsFiniteDiagram figureEight where
|
||||
𝓔Fintype := Fin.fintype _
|
||||
𝓔DecidableEq := instDecidableEqFin _
|
||||
𝓥Fintype := Fin.fintype _
|
||||
𝓥DecidableEq := instDecidableEqFin _
|
||||
𝓱𝓔Fintype := Fin.fintype _
|
||||
𝓱𝓔DecidableEq := instDecidableEqFin _
|
||||
|
||||
#eval symmetryFactor figureEight
|
||||
|
||||
#eval Connected figureEight
|
||||
|
||||
end PhiFour
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue