Documentation

Mathlib.Tactic.Core

#

Generally useful tactics.

Return the modifiers of declaration nm with (optional) docstring newDoc. Currently, recursive or partial definitions are not supported, and no attributes are provided.

Instances For
    def Lean.toPreDefinition (nm : Lean.Name) (newNm : Lean.Name) (newType : Lean.Expr) (newValue : Lean.Expr) (newDoc : optParam (Option String) none) :

    Make a PreDefinition taking some metadata from declaration nm. You can provide a new type, value and (optional) docstring, but the remaining information is taken from nm. Currently only implemented for definitions and theorems. Also see docstring of toModifiers

    Instances For

      Make nm protected.

      Instances For

        Introduce variables, giving them names from a specified list.

        Instances For

          Extract the arguments from a simpArgs syntax as an array of syntaxes

          Instances For

            Extract the arguments from a dsimpArgs syntax as an array of syntaxes

            Instances For

              Extract the arguments from a withArgs syntax as an array of syntaxes

              Instances For

                Extract the argument from a usingArg syntax as a syntax term

                Instances For

                  repeat1 tac applies tac to main goal at least once. If the application succeeds, the tactic is applied recursively to the generated subgoals until it eventually fails.

                  Instances For

                    Given a local context and an array of FVarIds assumed to be in that local context, remove all implementation details.

                    Instances For

                      Elaborate syntax for an FVarId in the local context of the given goal.

                      Instances For

                        Get the array of FVarIds in the local context of the given goal.

                        If ids is specified, elaborate them in the local context of the given goal to obtain the array of FVarIds.

                        If includeImplementationDetails is false (the default), we filter out implementation details (implDecls and auxDecls) from the resulting list of FVarIds.

                        Instances For

                          Run a tactic on all goals, and always succeeds.

                          (This is parallel to Lean.Elab.Tactic.evalAllGoals in core, which takes a Syntax rather than TacticM Unit. This function could be moved to core and evalAllGoals refactored to use it.)

                          Instances For

                            Simulates the <;> tactic combinator. First runs tac1 and then runs tac2 on all newly-generated subgoals.

                            Instances For

                              Repeats a tactic at most n times, stopping sooner if the tactic fails. Always succeeds.

                              Equations
                              Instances For
                                def Lean.Elab.Tactic.iterateExactly' {m : TypeType u_1} [Monad m] :
                                Natm Unitm Unit

                                iterateExactly' n t executes t n times. If any iteration fails, the whole tactic fails.

                                Equations
                                Instances For

                                  iterateRange m n t: Repeat the given tactic at least m times and at most n times or until t fails. Fails if t does not run at least m times.

                                  Equations
                                  Instances For

                                    Repeats a tactic until it fails. Always succeeds.

                                    partial def Lean.Elab.Tactic.iterateUntilFailureWithResults {m : TypeType u_1} [Monad m] [MonadExcept Lean.Exception m] {α : Type} (tac : m α) :
                                    m (List α)

                                    iterateUntilFailureWithResults is a helper tactic which accumulates the list of results obtained from iterating tac until it fails. Always succeeds.

                                    iterateUntilFailureCount is similar to iterateUntilFailure except it counts the number of successful calls to tac. Always succeeds.

                                    Instances For

                                      Returns the root directory which contains the package root file, e.g. Mathlib.lean.

                                      Instances For

                                        Returns the mathlib root directory.

                                        Instances For