Skip to content

Commit

Permalink
chore(SimpleGraph): fix 3 DecidableEq assumptions (#11762)
Browse files Browse the repository at this point in the history
Found by a WIP linter in #10235
  • Loading branch information
urkud authored and atarnoam committed Apr 16, 2024
1 parent c80df95 commit 8eae373
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Combinatorics/SimpleGraph/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -157,6 +157,7 @@ instance : Fintype (edge s t).edgeSet := by rw [edge]; infer_instance

theorem edgeFinset_sup_edge [Fintype (edgeSet (G ⊔ edge s t))] (hn : ¬G.Adj s t) (h : s ≠ t) :
(G ⊔ edge s t).edgeFinset = G.edgeFinset.cons s(s, t) (by simp_all) := by
letI := Classical.decEq V
rw [edgeFinset_sup, cons_eq_insert, insert_eq, union_comm]
simp_rw [edgeFinset, edge_edgeSet_of_ne h]; rfl

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean
Original file line number Diff line number Diff line change
Expand Up @@ -183,6 +183,7 @@ set_option linter.uppercaseLean3 false in
`k * (k - ℓ - 1) = (n - k - 1) * μ`. -/
theorem IsSRGWith.param_eq (h : G.IsSRGWith n k ℓ μ) (hn : 0 < n) :
k * (k - ℓ - 1) = (n - k - 1) * μ := by
letI := Classical.decEq V
rw [← h.card, Fintype.card_pos_iff] at hn
obtain ⟨v⟩ := hn
convert card_mul_eq_card_mul G.Adj (s := G.neighborFinset v) (t := Gᶜ.neighborFinset v) _ _
Expand Down

0 comments on commit 8eae373

Please sign in to comment.