Equations
Instances For
@[inline]
Equations
Instances For
Equations
- Lean.NameMap.instInhabited α = { default := ∅ }
Instances For
Equations
- m.find? n = Lean.RBMap.find? m n
Instances For
instance
Lean.NameMap.instForInProdName
{α : Type}
{m : Type u_1 → Type u_2}
:
ForIn m (Lean.NameMap α) (Lean.Name × α)
filterMap f m
filters an NameMap
and simultaneously modifies the filtered values.
It takes a function f : Name → α → Option β
and applies f name
to the value with key name
.
The resulting entries with non-none
value are collected to form the output NameMap
.
Instances For
Equations
- Lean.NameSet.instEmptyCollection = { emptyCollection := Lean.NameSet.empty }
Equations
- s.insert n = Lean.RBTree.insert s n
Instances For
Equations
- Lean.NameSet.instForInName = inferInstanceAs (ForIn m (Lean.RBTree Lean.Name Lean.Name.quickCmp) Lean.Name)
The union of two NameSet
s.
Instances For
filter f s
returns the NameSet
consisting of all x
in s
where f x
returns true
.
Equations
- Lean.NameSet.filter f s = Lean.RBTree.filter f s
Instances For
Equations
- Lean.NameSSet.instEmptyCollection = { emptyCollection := Lean.NameSSet.empty }
@[reducible, inline]
Instances For
Equations
- s.insert n = Std.HashSet.insert s n
Instances For
filter f s
returns the NameHashSet
consisting of all x
in s
where f x
returns true
.