Equations
Instances For
@[inline]
Equations
Instances For
Equations
Equations
- Lean.NameMap.instEmptyCollection α = { emptyCollection := Lean.mkNameMap α }
Equations
- Lean.NameMap.instInhabited α = { default := ∅ }
Equations
- m.insert n a = Std.TreeMap.insert m n a
Instances For
Equations
- m.contains n = Std.TreeMap.contains m n
Instances For
Equations
- m.find? n = Std.TreeMap.get? m n
Instances For
Equations
filter f m
returns the NameMap
consisting of all
"key
/val
"-pairs in m
where f key val
returns true
.
Equations
- Lean.NameMap.filter f m = Std.TreeMap.filter f m
Instances For
Equations
Instances For
Equations
- Lean.NameSet.instEmptyCollection = { emptyCollection := Lean.NameSet.empty }
Equations
- Lean.NameSet.instInhabited = { default := Lean.NameSet.empty }
Equations
- s.insert n = Std.TreeSet.insert s n
Instances For
Equations
- s.contains n = Std.TreeSet.contains s n
Instances For
Equations
- Lean.NameSet.instAppend = { append := Lean.NameSet.append }
Equations
- Lean.NameSet.instUnion = { union := Lean.NameSet.append }
Equations
- Lean.NameSet.instInter = { inter := fun (s t : Lean.NameSet) => Std.TreeSet.foldl (fun (r : Lean.NameSet) (n : Lean.Name) => if t.contains n = true then r.insert n else r) ∅ s }
Equations
- Lean.NameSet.instSDiff = { sdiff := fun (s t : Lean.NameSet) => Std.TreeSet.foldl (fun (s : Lean.NameSet) (n : Lean.Name) => Std.TreeSet.erase s n) s t }
filter f s
returns the NameSet
consisting of all x
in s
where f x
returns true
.
Equations
- Lean.NameSet.filter f s = Std.TreeSet.filter f s
Instances For
Equations
Instances For
Equations
Instances For
@[reducible, inline]
Equations
Instances For
Equations
- Lean.NameSSet.instEmptyCollection = { emptyCollection := Lean.NameSSet.empty }
Equations
- Lean.NameSSet.instInhabited = { default := Lean.NameSSet.empty }
@[inline]
Equations
Instances For
Equations
- Lean.NameHashSet.instEmptyCollection = { emptyCollection := Lean.NameHashSet.empty }
Equations
- Lean.NameHashSet.instInhabited = { default := ∅ }
Equations
- s.insert n = Std.HashSet.insert s n
Instances For
Equations
- s.contains n = Std.HashSet.contains s n
Instances For
filter f s
returns the NameHashSet
consisting of all x
in s
where f x
returns true
.
Equations
Instances For
Equations
- v₁.isPrefixOf v₂ = (v₁.name.isPrefixOf v₂.name && v₁.scopes == v₂.scopes && v₁.mainModule == v₂.mainModule && v₁.imported == v₂.imported)
Instances For
Equations
- v₁.isSuffixOf v₂ = (v₁.name.isSuffixOf v₂.name && v₁.scopes == v₂.scopes && v₁.mainModule == v₂.mainModule && v₁.imported == v₂.imported)