Documentation

Lake.DSL.Targets

DSL for Targets & Facets #

Macros for declaring Lake targets and facets.

Facet Declarations #

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

        Custom Target Declaration #

        @[reducible, inline]
        abbrev Lake.DSL.mkTargetDecl (α : Type) (pkgName target : Lean.Name) [OptDataKind α] [FormatQuery α] [FamilyDef (CustomData pkgName) target α] (f : NPackage pkgNameFetchM (Job α)) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          Lean Library & Executable Target Declarations #

          @[reducible, inline]
          abbrev Lake.DSL.mkConfigDecl (pkg name kind : Lean.Name) (config : ConfigType kind pkg name) [FamilyDef (CustomData pkg) name (ConfigTarget kind)] [FamilyDef DataType kind (ConfigTarget kind)] :
          Equations
          • Lake.DSL.mkConfigDecl pkg name kind config = { pkg := pkg, name := name, kind := kind, config := config, wf_data := , kind_eq := }
          Instances For

            External Library Target Declaration #

            @[reducible, inline]
            Equations
            Instances For