Skip to content

Commit

Permalink
docs(data/list/sections): add module docstring (#8033)
Browse files Browse the repository at this point in the history


Co-authored-by: Floris van Doorn <fpvdoorn@gmail.com>
  • Loading branch information
YaelDillies and fpvandoorn committed Jun 29, 2021
1 parent 2c749b1 commit 2600baf
Showing 1 changed file with 8 additions and 4 deletions.
12 changes: 8 additions & 4 deletions src/data/list/sections.lean
Expand Up @@ -5,14 +5,18 @@ Authors: Mario Carneiro
-/
import data.list.forall2

universes u v
/-!
# List sections
This file proves some stuff about `list.sections` (definition in `data.list.defs`). A section of a
list of lists `[l₁, ..., lₙ]` is a list whose `i`-th element comes from the `i`-th list.
-/


open nat function
variables {α : Type u} {β : Type v}

namespace list

/- sections -/
variables {α β : Type*}

theorem mem_sections {L : list (list α)} {f} : f ∈ sections L ↔ forall₂ (∈) f L :=
begin
Expand Down

0 comments on commit 2600baf

Please sign in to comment.