refactor: Lint
This commit is contained in:
parent
e00f14b552
commit
0228cd4cf1
3 changed files with 1 additions and 4 deletions
|
@ -90,9 +90,6 @@ lemma figureEight_connected : Connected figureEight := by decide
|
|||
`#eval symmetryFactor figureEight`. -/
|
||||
lemma figureEight_symmetryFactor : symmetryFactor figureEight = 8 := by decide
|
||||
|
||||
lemma figureEight_halfEdgeToEdgeIntMatrix :
|
||||
figureEight.halfEdgeToEdgeIntMatrix = !![1, 0; 1, 0 ; 0, 1; 0, 1] := by decide
|
||||
|
||||
end Example
|
||||
|
||||
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue