Documentation

Std.Lean.PersistentHashSet

instance Lean.PersistentHashSet.instForInPersistentHashSet {α : Type u_1} [BEq α] [Hashable α] {m : Type u_2 → Type u_3} :
Equations
  • One or more equations did not get rendered due to their size.
@[specialize #[]]
def Lean.PersistentHashSet.anyM {α : Type u_1} [BEq α] [Hashable α] {m : TypeType u_2} [Monad m] (s : Lean.PersistentHashSet α) (f : αm Bool) :

Returns true if f returns true for any element of the set.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[inline]
    def Lean.PersistentHashSet.any {α : Type u_1} [BEq α] [Hashable α] (s : Lean.PersistentHashSet α) (f : αBool) :

    Returns true if f returns true for any element of the set.

    Equations
    Instances For
      @[specialize #[]]
      def Lean.PersistentHashSet.allM {α : Type u_1} [BEq α] [Hashable α] {m : TypeType u_2} [Monad m] (s : Lean.PersistentHashSet α) (f : αm Bool) :

      Returns true if f returns true for all elements of the set.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[inline]
        def Lean.PersistentHashSet.all {α : Type u_1} [BEq α] [Hashable α] (s : Lean.PersistentHashSet α) (f : αBool) :

        Returns true if f returns true for all elements of the set.

        Equations
        Instances For
          Equations
          • One or more equations did not get rendered due to their size.
          @[inline]

          Similar to insert, but also returns a Boolean flag indicating whether an existing entry has been replaced with a => b.

          Equations
          Instances For
            def Lean.PersistentHashSet.insertMany {α : Type u_1} [BEq α] [Hashable α] {ρ : Type u_2} [ForIn Id ρ α] (s : Lean.PersistentHashSet α) (as : ρ) :

            Insert all elements from a collection into a PersistentHashSet.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[inline]

              Obtain a PersistentHashSet from an array.

              Equations
              Instances For
                @[inline]

                Obtain a PersistentHashSet from a list.

                Equations
                Instances For
                  @[inline]

                  Merge two PersistentHashSets.

                  Equations
                  Instances For