diff --git a/Mathlib/Combinatorics/SimpleGraph/Clique.lean b/Mathlib/Combinatorics/SimpleGraph/Clique.lean index 27b0dec7200f2..5e38fb4547ee0 100644 --- a/Mathlib/Combinatorics/SimpleGraph/Clique.lean +++ b/Mathlib/Combinatorics/SimpleGraph/Clique.lean @@ -165,8 +165,6 @@ lemma isClique_compl_map_iff_isClique_map_compl {f : α ↪ β} {s : Set α} : end Clique --- examle {f : α ↪ β} {s : Set α} (a : α) (h : a ∈ f '' s) ↔ : - /-! ### `n`-cliques -/