- keys : Array Lean.Meta.DiscrTree.Key
- val : Lean.Expr
- priority : Nat
Equations
- Lean.Meta.instInhabitedInstanceEntry = { default := { keys := default, val := default, priority := default, globalName? := default } }
Equations
- Lean.Meta.instBEqInstanceEntry = { beq := fun e₁ e₂ => e₁.val == e₂.val }
Equations
- Lean.Meta.instToFormatInstanceEntry = { format := fun e => match e.globalName? with | some n => Lean.format n | x => Std.Format.text "<local>" }
- discrTree : Lean.Meta.DiscrTree Lean.Meta.InstanceEntry
- instanceNames : Std.PHashSet Lean.Name
- erased : Std.PHashSet Lean.Name
Equations
- Lean.Meta.instInhabitedInstances = { default := { discrTree := default, instanceNames := default, erased := default } }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.Instances.erase
{m : Type → Type}
[inst : Monad m]
[inst : Lean.MonadError m]
(d : Lean.Meta.Instances)
(declName : Lean.Name)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.getGlobalInstancesIndex = do let a ← Lean.getEnv pure (Lean.ScopedEnvExtension.getState Lean.Meta.instanceExtension a).discrTree
Equations
- Lean.Meta.getErasedInstances = do let a ← Lean.getEnv pure (Lean.ScopedEnvExtension.getState Lean.Meta.instanceExtension a).erased
@[inline]
Equations
- Lean.Meta.PrioritySet = Std.RBTree Nat fun x y => compare y x
- defaultInstances : Lean.NameMap (List (Lean.Name × Nat))
- priorities : Lean.Meta.PrioritySet
Equations
- Lean.Meta.instInhabitedDefaultInstances = { default := { defaultInstances := default, priorities := default } }
def
Lean.Meta.addDefaultInstanceEntry
(d : Lean.Meta.DefaultInstances)
(e : Lean.Meta.DefaultInstanceEntry)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.getDefaultInstancesPriorities
{m : Type → Type}
[inst : Monad m]
[inst : Lean.MonadEnv m]
:
Equations
- Lean.Meta.getDefaultInstancesPriorities = do let a ← Lean.getEnv pure (Lean.SimplePersistentEnvExtension.getState Lean.Meta.defaultInstanceExtension a).priorities
def
Lean.Meta.getDefaultInstances
{m : Type → Type}
[inst : Monad m]
[inst : Lean.MonadEnv m]
(className : Lean.Name)
:
Equations
- One or more equations did not get rendered due to their size.