diff --git a/Batteries/Data/List/Basic.lean b/Batteries/Data/List/Basic.lean index a983f2a6fb..e714463a76 100644 --- a/Batteries/Data/List/Basic.lean +++ b/Batteries/Data/List/Basic.lean @@ -515,7 +515,7 @@ def sigmaTR {σ : α → Type _} (l₁ : List α) (l₂ : ∀ a, List (σ a)) : def ofFnNthVal {n} (f : Fin n → α) (i : Nat) : Option α := if h : i < n then some (f ⟨i, h⟩) else none -/-- `disjoint l₁ l₂` means that `l₁` and `l₂` have no elements in common. -/ +/-- `Disjoint l₁ l₂` means that `l₁` and `l₂` have no elements in common. -/ def Disjoint (l₁ l₂ : List α) : Prop := ∀ ⦃a⦄, a ∈ l₁ → a ∈ l₂ → False