Documentation

Lake.Build.Targets

Build Target Fetching #

Utilities for fetching package, library, module, and executable targets and facets.

@[inline]
def Lake.KConfigDecl.get {m : TypeType u_1} {kind : Lean.Name} [Monad m] [MonadError m] [MonadLake m] (self : KConfigDecl kind) :
m (ConfigTarget kind)

Get the target in the workspace corresponding to this configuration.

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

    Package Facets & Targets #

    Fetch the build job of the specified package target.

    Equations
    Instances For
      def Lake.TargetDecl.fetch {α : Type} (self : TargetDecl) [FamilyOut (CustomData self.pkg) self.name α] :
      FetchM (Job α)

      Fetch the build result of a target.

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

        Fetch the build job of the target.

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

          Fetch the build result of a package facet.

          Equations
          Instances For

            Fetch the build job of a library facet.

            Equations
            Instances For

              Module Facets #

              @[inline]

              Fetch the build result of a module facet.

              Equations
              Instances For

                Fetch the build job of a module facet.

                Equations
                Instances For

                  Lean Library Facets #

                  @[inline]
                  def Lake.LeanLibDecl.get {m : TypeType u_1} (self : LeanLibDecl) [Monad m] [MonadError m] [MonadLake m] :

                  Get the Lean library in the workspace corresponding to this configuration.

                  Equations
                  Instances For
                    @[inline]

                    Fetch the build result of a library facet.

                    Equations
                    Instances For

                      Fetch the build job of a library facet.

                      Equations
                      Instances For

                        Lean Executable Target #

                        @[inline]
                        def Lake.LeanExeDecl.get {m : TypeType u_1} (self : LeanExeDecl) [Monad m] [MonadError m] [MonadLake m] :

                        Get the Lean executable in the workspace corresponding to this configuration.

                        Equations
                        Instances For
                          @[inline]

                          Fetch the build of the Lean executable.

                          Equations
                          Instances For
                            @[inline]

                            Fetch the build of the Lean executable.

                            Equations
                            Instances For

                              Input File / Directory Targets #

                              @[inline]

                              Fetch the input file.

                              Equations
                              Instances For
                                @[inline]

                                Get the input file in the workspace corresponding to this configuration.

                                Equations
                                Instances For
                                  @[inline]

                                  Fetch the input file.

                                  Equations
                                  Instances For
                                    @[inline]

                                    Fetch the files in the input directory.

                                    Equations
                                    Instances For
                                      @[inline]
                                      def Lake.InputDirDecl.get {m : TypeType u_1} (self : InputDirDecl) [Monad m] [MonadError m] [MonadLake m] :

                                      Get the input directory in the workspace corresponding to this configuration.

                                      Equations
                                      Instances For
                                        @[inline]

                                        Fetch the files in the input directory.

                                        Equations
                                        Instances For