Documentation

Lake.Config.FacetConfig

structure Lake.FacetConfig (DataFam : Lean.NameType) (ι : Type) (name : Lean.Name) :

A facet's declarative configuration.

  • fetchFn : ιFetchM (Job (DataFam name))

    The facet's fetch function.

  • buildable : Bool

    Is this facet compatible with the lake build CLI?

  • format : OutFormatDataFam nameString

    Format this facet's output (e.g., for lake query).

Instances For
    instance Lake.instInhabitedFacetConfig {a✝ : Lean.NameType} {a✝¹ : Type} {a✝² : Lean.Name} :
    Inhabited (FacetConfig a✝ a✝¹ a✝²)
    Equations
    @[reducible, inline]
    abbrev Lake.FacetConfig.name {DataFam : Lean.NameType} {ι : Type} {name : Lean.Name} :
    FacetConfig DataFam ι nameLean.Name
    Equations
    Instances For
      @[inline]
      def Lake.mkFacetJobConfig {α : Type} {Fam : Lean.NameType} {facet : Lean.Name} {ι : Type} [FormatQuery α] [h : FamilyOut Fam facet α] (build : ιFetchM (Job α)) (buildable : Bool := true) :
      FacetConfig Fam ι facet

      A smart constructor for facet configurations that generate jobs for the CLI.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        structure Lake.NamedConfigDecl (β : Lean.NameType u) :

        A dependently typed configuration based on its registered name.

        Instances For
          @[reducible, inline]

          A module facet's declarative configuration.

          Equations
          Instances For
            @[reducible, inline]

            A module facet declaration from a configuration file.

            Equations
            Instances For
              @[reducible, inline]

              A package facet's declarative configuration.

              Equations
              Instances For
                @[reducible, inline]

                A package facet declaration from a configuration file.

                Equations
                Instances For
                  @[reducible, inline]

                  A library facet's declarative configuration.

                  Equations
                  Instances For
                    @[reducible, inline]

                    A library facet declaration from a configuration file.

                    Equations
                    Instances For