Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
oop
Browse files Browse the repository at this point in the history
  • Loading branch information
b-mehta committed Oct 1, 2023
1 parent 3452f9a commit 7f64056
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/combinatorics/simple_graph/exponential_ramsey/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -201,8 +201,8 @@ begin
simp only [function.embedding.coe_fn_mk, mem_neighbor_finset, iff_self, implies_true_iff],
end

lemma col_density_eq_sum {K : Type*} [fintype V] [decidable_eq K] {χ : top_edge_labelling V K} {k : K}
{A B : finset V} :
lemma col_density_eq_sum {K : Type*} [fintype V] [decidable_eq K] {χ : top_edge_labelling V K}
{k : K} {A B : finset V} :
col_density χ k A B = (∑ x in A, (col_neighbors χ k x ∩ B).card) / (A.card * B.card) :=
begin
rw [col_density, edge_density_def, interedges_card_eq_sum],
Expand Down

0 comments on commit 7f64056

Please sign in to comment.