Documentation

Lean.Data.NameMap

Instances For
    Instances For
      def Lean.NameMap.find? {α : Type} (m : Lean.NameMap α) (n : Lean.Name) :
      Equations
      Instances For
        instance Lean.NameMap.instForInProdName {α : Type} {m : Type u_1 → Type u_2} :
        def Lean.NameMap.filter {α : Type} (f : Lean.NameαBool) (m : Lean.NameMap α) :

        filter f m returns the NameMap consisting of all "key/val"-pairs in m where f key val returns true.

        Instances For
          def Lean.NameMap.filterMap {α β : Type} (f : Lean.NameαOption β) (m : Lean.NameMap α) :

          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
            Instances For
              Equations
              Instances For

                The union of two NameSets.

                Instances For

                  filter f s returns the NameSet consisting of all x in s where f x returns true.

                  Equations
                  Instances For
                    Instances For
                      @[reducible, inline]
                      Equations
                      Instances For
                        @[reducible, inline]
                        Instances For
                          @[reducible, inline]
                          Equations
                          Instances For
                            Instances For
                              @[inline]
                              Equations
                              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)
                                    Instances For