Documentation

Lean.Util.FindExpr

@[reducible, inline]
unsafe abbrev Lean.Expr.FindImpl.FindM (m : TypeType u_1) (α : Type) :
Type u_1
Equations
Instances For
    @[inline]
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        unsafe def Lean.Expr.FindImpl.findUnsafeM? {m : TypeType u_1} [Monad m] (p : Lean.Exprm Bool) (e : Lean.Expr) :
        Equations
        Instances For
          @[implemented_by Lean.Expr.FindImpl.findUnsafeM?]
          def Lean.Expr.findM? {m : TypeType u_1} [Monad m] (p : Lean.Exprm Bool) (e : Lean.Expr) :
          Instances For
            @[implemented_by Lean.Expr.FindImpl.findUnsafe?]
            Equations
            Instances For

              Return true if e occurs in t

              Equations
              Instances For

                Return type for findExt? function argument.

                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      @[implemented_by Lean.Expr.FindExtImpl.findUnsafe?]

                      Similar to find?, but p can return FindStep.done to interrupt the search on subterms. Remark: Differently from find?, we do not invoke p for partial applications of an application.