Skip to content

Commit

Permalink
.
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed May 30, 2024
1 parent 6ab75df commit ca68259
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean
Original file line number Diff line number Diff line change
Expand Up @@ -123,7 +123,7 @@ lemma triangle_counting'
refine (Nat.cast_le.2 $ card_union_le _ _).trans ?_
rw [Nat.cast_add]
exact add_le_add h₁ h₂
rintro a ha b hy t
rintro a _ b hy t
rw [disjoint_left]
simp only [Prod.forall, mem_image, not_exists, exists_prop, mem_filter, Prod.mk.inj_iff,
exists_imp, and_imp, not_and, mem_product, or_assoc]
Expand Down

0 comments on commit ca68259

Please sign in to comment.