A facet's declarative configuration.
The facet's fetch function.
- buildable : Bool
Is this facet compatible with the
lake build
CLI? Format this facet's output (e.g., for
lake query
).
Instances For
instance
Lake.instInhabitedFacetConfig
{a✝ : Lean.Name → Type}
{a✝¹ : Type}
{a✝² : Lean.Name}
:
Inhabited (FacetConfig a✝ a✝¹ a✝²)
Equations
- Lake.instInhabitedFacetConfig = { default := { fetchFn := default, buildable := default, format := default } }
@[reducible, inline]
abbrev
Lake.FacetConfig.name
{DataFam : Lean.Name → Type}
{ι : Type}
{name : Lean.Name}
:
FacetConfig DataFam ι name → Lean.Name
Instances For
@[inline]
def
Lake.mkFacetJobConfig
{α : Type}
{Fam : Lean.Name → Type}
{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
@[reducible, inline]
A module facet's declarative configuration.
Instances For
@[reducible, inline]
A module facet declaration from a configuration file.
Instances For
@[reducible, inline]
A package facet's declarative configuration.
Instances For
@[reducible, inline]
A package facet declaration from a configuration file.
Instances For
@[reducible, inline]
A library facet's declarative configuration.
Instances For
@[reducible, inline]
A library facet declaration from a configuration file.