refactor: Lint

This commit is contained in:
jstoobysmith 2025-02-03 06:13:13 +00:00
parent fca3f02eca
commit c8e9c285a3
8 changed files with 229 additions and 194 deletions

View file

@ -44,7 +44,6 @@ instance : DecidableEq (WickContraction n) := Subtype.instDecidableEq
/-- The contraction consisting of no contracted pairs. -/
def empty : WickContraction n := ⟨∅, by simp, by simp⟩
@[simp]
lemma card_zero_iff_empty (c : WickContraction n) : c.1.card = 0 ↔ c = empty := by
rw [Subtype.eq_iff]
simp [empty]