Skip to content

Commit cce0137

Browse files
authored
doc: Fix typo (#1155)
1 parent b8e1430 commit cce0137

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Batteries/Data/List/Basic.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -515,7 +515,7 @@ def sigmaTR {σ : α → Type _} (l₁ : List α) (l₂ : ∀ a, List (σ a)) :
515515
def ofFnNthVal {n} (f : Fin n → α) (i : Nat) : Option α :=
516516
if h : i < n then some (f ⟨i, h⟩) else none
517517

518-
/-- `disjoint l₁ l₂` means that `l₁` and `l₂` have no elements in common. -/
518+
/-- `Disjoint l₁ l₂` means that `l₁` and `l₂` have no elements in common. -/
519519
def Disjoint (l₁ l₂ : List α) : Prop :=
520520
∀ ⦃a⦄, a ∈ l₁ → a ∈ l₂ → False
521521

0 commit comments

Comments
 (0)