Documentation

Mathlib.Tactic.Linter.EmptyLine

The "emptyLine" linter #

The "emptyLine" linter emits a warning on empty lines inside a command, but outside of a doc-string/module-doc.

Retrieve the String.Range of a Substring.

Equations
Instances For

    Syntax filters #

    partial def Lean.Syntax.filterMapM {m : TypeType} [Monad m] {α : Type} (stx : Syntax) (f : Syntaxm (Option α)) :
    m (Array α)

    filterMapM stx f takes as input a Syntax stx and a monadic function f : Syntax → m α. It produces the array of the some values that f takes while traversing stx.

    See filterMap for a non-monadic version.

    def Lean.Syntax.filterMap {α : Type} (stx : Syntax) (f : SyntaxOption α) :

    filterMap stx f takes as input a Syntax stx and a function f : Syntax → α. It produces the array of the some values that f takes while traversing stx.

    See filterMapM for a non-monadic version.

    Equations
    Instances For

      filter stx f takes as input a Syntax stx and a function f : Syntax → Bool. It produces the array of the syntax nodes in stx where f is true.

      See also the similar filterMap and filterMapM.

      Equations
      Instances For

        The "emptyLine" linter emits a warning on empty lines inside a command, but outside of a doc-string/module-doc.

        The linter is only active when there are no other warnings, so as to not add noise when developing incomplete proofs.

        @[reducible, inline]

        The SyntaxNodeKinds where the EmptyLine linter is not active

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[reducible, inline]

          If a file contains one of these names as segments, we disable the emptyLine linter.

          Equations
          Instances For

            The "emptyLine" linter emits a warning on empty lines inside a command, but outside of a doc-string/module-doc.

            The linter is only active when there are no other warnings, so as to not add noise when developing incomplete proofs.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For