Documentation

Init.Data.Vector.Basic

Vectors #

Vector α n is a thin wrapper around Array α for arrays of fixed size n.

structure Vector (α : Type u) (n : Nat) extends Array α :

Vector α n is an Array α with size n.

Instances For
    instance instReprVector {α✝ : Type u_1} {n✝ : Nat} [Repr α✝] :
    Repr (Vector α✝ n✝)
    Equations
    instance instDecidableEqVector {α✝ : Type u_1} {n✝ : Nat} [DecidableEq α✝] :
    DecidableEq (Vector α✝ n✝)
    Equations
    @[reducible, inline]
    abbrev Array.toVector {α : Type u_1} (xs : Array α) :
    Vector α xs.size

    Convert xs : Array α to Vector α xs.size.

    Equations
    • xs.toVector = { toArray := xs, size_toArray := }
    Instances For

      Syntax for Vector α n

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def Vector.elimAsArray {α : Type u_1} {n : Nat} {motive : Vector α nSort u} (mk : (a : Array α) → (ha : a.size = n) → motive { toArray := a, size_toArray := ha }) (v : Vector α n) :
        motive v

        Custom eliminator for Vector α n through Array α

        Equations
        Instances For
          def Vector.elimAsList {α : Type u_1} {n : Nat} {motive : Vector α nSort u} (mk : (a : List α) → (ha : a.length = n) → motive { toList := a, size_toArray := ha }) (v : Vector α n) :
          motive v

          Custom eliminator for Vector α n through List α

          Equations
          Instances For
            @[inline]
            def Vector.mkEmpty {α : Type u_1} (capacity : Nat) :
            Vector α 0

            Make an empty vector with pre-allocated capacity.

            Equations
            Instances For
              @[inline]
              def Vector.mkVector {α : Type u_1} (n : Nat) (v : α) :
              Vector α n

              Makes a vector of size n with all cells containing v.

              Equations
              Instances For
                instance Vector.instNonempty {α : Type u_1} {n : Nat} [Nonempty α] :
                @[inline]
                def Vector.singleton {α : Type u_1} (v : α) :
                Vector α 1

                Returns a vector of size 1 with element v.

                Equations
                Instances For
                  instance Vector.instInhabited {α : Type u_1} {n : Nat} [Inhabited α] :
                  Equations
                  @[inline]
                  def Vector.get {α : Type u_1} {n : Nat} (v : Vector α n) (i : Fin n) :
                  α

                  Get an element of a vector using a Fin index.

                  Equations
                  Instances For
                    @[inline]
                    def Vector.uget {α : Type u_1} {n : Nat} (v : Vector α n) (i : USize) (h : i.toNat < n) :
                    α

                    Get an element of a vector using a USize index and a proof that the index is within bounds.

                    Equations
                    Instances For
                      instance Vector.instGetElemNatLt {α : Type u_1} {n : Nat} :
                      GetElem (Vector α n) Nat α fun (x : Vector α n) (i : Nat) => i < n
                      Equations
                      def Vector.contains {α : Type u_1} {n : Nat} [BEq α] (v : Vector α n) (a : α) :

                      Check if there is an element which satisfies a == ·.

                      Equations
                      Instances For
                        structure Vector.Mem {α : Type u_1} {n : Nat} (as : Vector α n) (a : α) :

                        a ∈ v is a predicate which asserts that a is in the vector v.

                        Instances For
                          instance Vector.instMembership {α : Type u_1} {n : Nat} :
                          Membership α (Vector α n)
                          Equations
                          @[inline]
                          def Vector.getD {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (default : α) :
                          α

                          Get an element of a vector using a Nat index. Returns the given default value if the index is out of bounds.

                          Equations
                          Instances For
                            @[inline]
                            def Vector.back! {α : Type u_1} {n : Nat} [Inhabited α] (v : Vector α n) :
                            α

                            The last element of a vector. Panics if the vector is empty.

                            Equations
                            Instances For
                              @[inline]
                              def Vector.back? {α : Type u_1} {n : Nat} (v : Vector α n) :

                              The last element of a vector, or none if the vector is empty.

                              Equations
                              Instances For
                                @[inline]
                                def Vector.back {n : Nat} {α : Type u_1} [NeZero n] (v : Vector α n) :
                                α

                                The last element of a non-empty vector.

                                Equations
                                Instances For
                                  @[inline]
                                  def Vector.head {n : Nat} {α : Type u_1} [NeZero n] (v : Vector α n) :
                                  α

                                  The first element of a non-empty vector.

                                  Equations
                                  Instances For
                                    @[inline]
                                    def Vector.push {α : Type u_1} {n : Nat} (v : Vector α n) (x : α) :
                                    Vector α (n + 1)

                                    Push an element x to the end of a vector.

                                    Equations
                                    • v.push x = { toArray := v.push x, size_toArray := }
                                    Instances For
                                      @[inline]
                                      def Vector.pop {α : Type u_1} {n : Nat} (v : Vector α n) :
                                      Vector α (n - 1)

                                      Remove the last element of a vector.

                                      Equations
                                      • v.pop = { toArray := v.pop, size_toArray := }
                                      Instances For
                                        @[inline]
                                        def Vector.set {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (x : α) (h : i < n := by get_elem_tactic) :
                                        Vector α n

                                        Set an element in a vector using a Nat index, with a tactic provided proof that the index is in bounds.

                                        This will perform the update destructively provided that the vector has a reference count of 1.

                                        Equations
                                        • v.set i x h = { toArray := v.set i x , size_toArray := }
                                        Instances For
                                          @[inline]
                                          def Vector.setIfInBounds {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (x : α) :
                                          Vector α n

                                          Set an element in a vector using a Nat index. Returns the vector unchanged if the index is out of bounds.

                                          This will perform the update destructively provided that the vector has a reference count of 1.

                                          Equations
                                          Instances For
                                            @[inline]
                                            def Vector.set! {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (x : α) :
                                            Vector α n

                                            Set an element in a vector using a Nat index. Panics if the index is out of bounds.

                                            This will perform the update destructively provided that the vector has a reference count of 1.

                                            Equations
                                            • v.set! i x = { toArray := v.set! i x, size_toArray := }
                                            Instances For
                                              @[inline]
                                              def Vector.foldlM {m : Type u_1 → Type u_2} {β : Type u_1} {α : Type u_3} {n : Nat} [Monad m] (f : βαm β) (b : β) (v : Vector α n) :
                                              m β
                                              Equations
                                              Instances For
                                                @[inline]
                                                def Vector.foldrM {m : Type u_1 → Type u_2} {α : Type u_3} {β : Type u_1} {n : Nat} [Monad m] (f : αβm β) (b : β) (v : Vector α n) :
                                                m β
                                                Equations
                                                Instances For
                                                  @[inline]
                                                  def Vector.foldl {β : Type u_1} {α : Type u_2} {n : Nat} (f : βαβ) (b : β) (v : Vector α n) :
                                                  β
                                                  Equations
                                                  Instances For
                                                    @[inline]
                                                    def Vector.foldr {α : Type u_1} {β : Type u_2} {n : Nat} (f : αββ) (b : β) (v : Vector α n) :
                                                    β
                                                    Equations
                                                    Instances For
                                                      @[inline]
                                                      def Vector.append {α : Type u_1} {n m : Nat} (v : Vector α n) (w : Vector α m) :
                                                      Vector α (n + m)

                                                      Append two vectors.

                                                      Equations
                                                      Instances For
                                                        instance Vector.instHAppendHAddNat {α : Type u_1} {n m : Nat} :
                                                        HAppend (Vector α n) (Vector α m) (Vector α (n + m))
                                                        Equations
                                                        @[inline]
                                                        def Vector.cast {n m : Nat} {α : Type u_1} (h : n = m) (v : Vector α n) :
                                                        Vector α m

                                                        Creates a vector from another with a provably equal length.

                                                        Equations
                                                        Instances For
                                                          @[inline]
                                                          def Vector.extract {α : Type u_1} {n : Nat} (v : Vector α n) (start : Nat := 0) (stop : Nat := n) :
                                                          Vector α (min stop n - start)

                                                          Extracts the slice of a vector from indices start to stop (exclusive). If start ≥ stop, the result is empty. If stop is greater than the size of the vector, the size is used instead.

                                                          Equations
                                                          • v.extract start stop = { toArray := v.extract start stop, size_toArray := }
                                                          Instances For
                                                            @[inline]
                                                            def Vector.take {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                            Vector α (min m n)

                                                            Extract the first m elements of a vector. If m is greater than or equal to the size of the vector then the vector is returned unchanged.

                                                            Equations
                                                            • v.take m = { toArray := v.take m, size_toArray := }
                                                            Instances For
                                                              @[simp]
                                                              theorem Vector.take_eq_extract {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                              v.take m = v.extract 0 m
                                                              @[inline]
                                                              def Vector.drop {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                              Vector α (n - m)

                                                              Deletes the first m elements of a vector. If m is greater than or equal to the size of the vector then the empty vector is returned.

                                                              Equations
                                                              • v.drop m = { toArray := v.drop m, size_toArray := }
                                                              Instances For
                                                                @[simp]
                                                                theorem Vector.drop_eq_cast_extract {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                                v.drop m = Vector.cast (v.extract m)
                                                                @[inline]
                                                                def Vector.shrink {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                                Vector α (min m n)

                                                                Shrinks a vector to the first m elements, by repeatedly popping the last element.

                                                                Equations
                                                                Instances For
                                                                  @[simp]
                                                                  theorem Vector.shrink_eq_take {α : Type u_1} {n : Nat} (v : Vector α n) (m : Nat) :
                                                                  v.shrink m = v.take m
                                                                  @[inline]
                                                                  def Vector.map {α : Type u_1} {β : Type u_2} {n : Nat} (f : αβ) (v : Vector α n) :
                                                                  Vector β n

                                                                  Maps elements of a vector using the function f.

                                                                  Equations
                                                                  Instances For
                                                                    @[inline]
                                                                    def Vector.mapIdx {α : Type u_1} {β : Type u_2} {n : Nat} (f : Natαβ) (v : Vector α n) :
                                                                    Vector β n

                                                                    Maps elements of a vector using the function f, which also receives the index of the element.

                                                                    Equations
                                                                    Instances For
                                                                      @[inline]
                                                                      def Vector.mapFinIdx {α : Type u_1} {n : Nat} {β : Type u_2} (v : Vector α n) (f : (i : Nat) → αi < nβ) :
                                                                      Vector β n

                                                                      Maps elements of a vector using the function f, which also receives the index of the element, and the fact that the index is less than the size of the vector.

                                                                      Equations
                                                                      Instances For
                                                                        @[inline]
                                                                        def Vector.mapM {m : Type u_1 → Type u_2} {α : Type u_3} {β : Type u_1} {n : Nat} [Monad m] (f : αm β) (v : Vector α n) :
                                                                        m (Vector β n)

                                                                        Map a monadic function over a vector.

                                                                        Equations
                                                                        Instances For
                                                                          @[irreducible]
                                                                          def Vector.mapM.go {m : Type u_1 → Type u_2} {α : Type u_3} {β : Type u_1} {n : Nat} [Monad m] (f : αm β) (v : Vector α n) (i : Nat) (h : i n) (r : Vector β i) :
                                                                          m (Vector β n)
                                                                          Equations
                                                                          Instances For
                                                                            @[inline]
                                                                            def Vector.forM {m : Type u_1 → Type u_2} {α : Type u_3} {n : Nat} [Monad m] (v : Vector α n) (f : αm PUnit) :
                                                                            Equations
                                                                            Instances For
                                                                              @[inline]
                                                                              def Vector.flatMapM {m : Type u_1 → Type u_2} {α : Type u_3} {n : Nat} {β : Type u_1} {k : Nat} [Monad m] (v : Vector α n) (f : αm (Vector β k)) :
                                                                              m (Vector β (n * k))
                                                                              Equations
                                                                              Instances For
                                                                                @[irreducible]
                                                                                def Vector.flatMapM.go {m : Type u_1 → Type u_2} {α : Type u_3} {n : Nat} {β : Type u_1} {k : Nat} [Monad m] (v : Vector α n) (f : αm (Vector β k)) (i : Nat) (h : i n) (r : Vector β (i * k)) :
                                                                                m (Vector β (n * k))
                                                                                Equations
                                                                                Instances For
                                                                                  @[inline]
                                                                                  def Vector.mapFinIdxM {n : Nat} {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : Vector α n) (f : (i : Nat) → αi < nm β) :
                                                                                  m (Vector β n)

                                                                                  Variant of mapIdxM which receives the index i along with the bound `i < n.

                                                                                  Equations
                                                                                  Instances For
                                                                                    @[specialize #[]]
                                                                                    def Vector.mapFinIdxM.map {n : Nat} {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : Vector α n) (f : (i : Nat) → αi < nm β) (i j : Nat) (inv : i + j = n) (bs : Vector β (n - i)) :
                                                                                    m (Vector β n)
                                                                                    Equations
                                                                                    Instances For
                                                                                      @[inline]
                                                                                      def Vector.mapIdxM {n : Nat} {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : Natαm β) (as : Vector α n) :
                                                                                      m (Vector β n)
                                                                                      Equations
                                                                                      Instances For
                                                                                        @[inline]
                                                                                        def Vector.firstM {β : Type v} {n : Nat} {α : Type u} {m : Type v → Type w} [Alternative m] (f : αm β) (as : Vector α n) :
                                                                                        m β
                                                                                        Equations
                                                                                        Instances For
                                                                                          @[inline]
                                                                                          def Vector.flatten {α : Type u_1} {n m : Nat} (v : Vector (Vector α n) m) :
                                                                                          Vector α (m * n)
                                                                                          Equations
                                                                                          Instances For
                                                                                            @[inline]
                                                                                            def Vector.flatMap {α : Type u_1} {n : Nat} {β : Type u_2} {m : Nat} (v : Vector α n) (f : αVector β m) :
                                                                                            Vector β (n * m)
                                                                                            Equations
                                                                                            Instances For
                                                                                              @[inline]
                                                                                              def Vector.zipIdx {α : Type u_1} {n : Nat} (v : Vector α n) (k : Nat := 0) :
                                                                                              Vector (α × Nat) n
                                                                                              Equations
                                                                                              Instances For
                                                                                                @[reducible, inline, deprecated Vector.zipIdx (since := "2025-01-21")]
                                                                                                abbrev Vector.zipWithIndex {α : Type u_1} {n : Nat} (v : Vector α n) (k : Nat := 0) :
                                                                                                Vector (α × Nat) n
                                                                                                Equations
                                                                                                Instances For
                                                                                                  @[inline]
                                                                                                  def Vector.zip {α : Type u_1} {n : Nat} {β : Type u_2} (v : Vector α n) (w : Vector β n) :
                                                                                                  Vector (α × β) n
                                                                                                  Equations
                                                                                                  Instances For
                                                                                                    @[inline]
                                                                                                    def Vector.zipWith {α : Type u_1} {β : Type u_2} {φ : Type u_3} {n : Nat} (f : αβφ) (a : Vector α n) (b : Vector β n) :
                                                                                                    Vector φ n

                                                                                                    Maps corresponding elements of two vectors of equal size using the function f.

                                                                                                    Equations
                                                                                                    Instances For
                                                                                                      @[inline]
                                                                                                      def Vector.unzip {α : Type u_1} {β : Type u_2} {n : Nat} (v : Vector (α × β) n) :
                                                                                                      Vector α n × Vector β n
                                                                                                      Equations
                                                                                                      Instances For
                                                                                                        @[inline]
                                                                                                        def Vector.ofFn {n : Nat} {α : Type u_1} (f : Fin nα) :
                                                                                                        Vector α n

                                                                                                        The vector of length n whose i-th element is f i.

                                                                                                        Equations
                                                                                                        Instances For
                                                                                                          @[inline]
                                                                                                          def Vector.swap {α : Type u_1} {n : Nat} (v : Vector α n) (i j : Nat) (hi : i < n := by get_elem_tactic) (hj : j < n := by get_elem_tactic) :
                                                                                                          Vector α n

                                                                                                          Swap two elements of a vector using Fin indices.

                                                                                                          This will perform the update destructively provided that the vector has a reference count of 1.

                                                                                                          Equations
                                                                                                          • v.swap i j hi hj = { toArray := v.swap i j , size_toArray := }
                                                                                                          Instances For
                                                                                                            @[inline]
                                                                                                            def Vector.swapIfInBounds {α : Type u_1} {n : Nat} (v : Vector α n) (i j : Nat) :
                                                                                                            Vector α n

                                                                                                            Swap two elements of a vector using Nat indices. Panics if either index is out of bounds.

                                                                                                            This will perform the update destructively provided that the vector has a reference count of 1.

                                                                                                            Equations
                                                                                                            Instances For
                                                                                                              @[inline]
                                                                                                              def Vector.swapAt {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (x : α) (hi : i < n := by get_elem_tactic) :
                                                                                                              α × Vector α n

                                                                                                              Swaps an element of a vector with a given value using a Fin index. The original value is returned along with the updated vector.

                                                                                                              This will perform the update destructively provided that the vector has a reference count of 1.

                                                                                                              Equations
                                                                                                              Instances For
                                                                                                                @[inline]
                                                                                                                def Vector.swapAt! {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (x : α) :
                                                                                                                α × Vector α n

                                                                                                                Swaps an element of a vector with a given value using a Nat index. Panics if the index is out of bounds. The original value is returned along with the updated vector.

                                                                                                                This will perform the update destructively provided that the vector has a reference count of 1.

                                                                                                                Equations
                                                                                                                Instances For
                                                                                                                  @[inline]
                                                                                                                  def Vector.range (n : Nat) :

                                                                                                                  The vector #v[0, 1, 2, ..., n-1].

                                                                                                                  Equations
                                                                                                                  Instances For
                                                                                                                    @[inline]
                                                                                                                    def Vector.range' (start size : Nat) (step : Nat := 1) :
                                                                                                                    Vector Nat size

                                                                                                                    The vector #v[start, start + step, start + 2 * step, ..., start + (size - 1) * step].

                                                                                                                    Equations
                                                                                                                    Instances For
                                                                                                                      @[inline]
                                                                                                                      def Vector.isEqv {α : Type u_1} {n : Nat} (v w : Vector α n) (r : ααBool) :

                                                                                                                      Compares two vectors of the same size using a given boolean relation r. isEqv v w r returns true if and only if r v[i] w[i] is true for all indices i.

                                                                                                                      Equations
                                                                                                                      Instances For
                                                                                                                        instance Vector.instBEq {α : Type u_1} {n : Nat} [BEq α] :
                                                                                                                        BEq (Vector α n)
                                                                                                                        Equations
                                                                                                                        @[inline]
                                                                                                                        def Vector.reverse {α : Type u_1} {n : Nat} (v : Vector α n) :
                                                                                                                        Vector α n

                                                                                                                        Reverse the elements of a vector.

                                                                                                                        Equations
                                                                                                                        Instances For
                                                                                                                          @[inline]
                                                                                                                          def Vector.eraseIdx {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) (h : i < n := by get_elem_tactic) :
                                                                                                                          Vector α (n - 1)

                                                                                                                          Delete an element of a vector using a Nat index and a tactic provided proof.

                                                                                                                          Equations
                                                                                                                          Instances For
                                                                                                                            @[inline]
                                                                                                                            def Vector.eraseIdx! {α : Type u_1} {n : Nat} (v : Vector α n) (i : Nat) :
                                                                                                                            Vector α (n - 1)

                                                                                                                            Delete an element of a vector using a Nat index. Panics if the index is out of bounds.

                                                                                                                            Equations
                                                                                                                            Instances For
                                                                                                                              @[inline]
                                                                                                                              def Vector.tail {α : Type u_1} {n : Nat} (v : Vector α n) :
                                                                                                                              Vector α (n - 1)

                                                                                                                              Delete the first element of a vector. Returns the empty vector if the input vector is empty.

                                                                                                                              Equations
                                                                                                                              Instances For
                                                                                                                                @[inline]
                                                                                                                                def Vector.finIdxOf? {α : Type u_1} {n : Nat} [BEq α] (v : Vector α n) (x : α) :

                                                                                                                                Finds the first index of a given value in a vector using == for comparison. Returns none if the no element of the index matches the given value.

                                                                                                                                Equations
                                                                                                                                Instances For
                                                                                                                                  @[reducible, inline, deprecated Vector.finIdxOf? (since := "2025-01-29")]
                                                                                                                                  abbrev Vector.indexOf? {α : Type u_1} {n : Nat} [BEq α] (v : Vector α n) (x : α) :
                                                                                                                                  Equations
                                                                                                                                  Instances For
                                                                                                                                    @[inline]
                                                                                                                                    def Vector.findFinIdx? {α : Type u_1} {n : Nat} (p : αBool) (v : Vector α n) :

                                                                                                                                    Finds the first index of a given value in a vector using a predicate. Returns none if the no element of the index matches the given value.

                                                                                                                                    Equations
                                                                                                                                    Instances For
                                                                                                                                      @[inline]
                                                                                                                                      def Vector.findM? {n : Nat} {α : Type} {m : TypeType} [Monad m] (f : αm Bool) (as : Vector α n) :
                                                                                                                                      m (Option α)

                                                                                                                                      Note that the universe level is contrained to Type here, to avoid having to have the predicate live in p : α → m (ULift Bool).

                                                                                                                                      Equations
                                                                                                                                      Instances For
                                                                                                                                        @[inline]
                                                                                                                                        def Vector.findSomeM? {m : Type u_1 → Type u_2} {α : Type u_3} {β : Type u_1} {n : Nat} [Monad m] (f : αm (Option β)) (as : Vector α n) :
                                                                                                                                        m (Option β)
                                                                                                                                        Equations
                                                                                                                                        Instances For
                                                                                                                                          @[inline]
                                                                                                                                          def Vector.findRevM? {n : Nat} {α : Type} {m : TypeType} [Monad m] (f : αm Bool) (as : Vector α n) :
                                                                                                                                          m (Option α)

                                                                                                                                          Note that the universe level is contrained to Type here, to avoid having to have the predicate live in p : α → m (ULift Bool).

                                                                                                                                          Equations
                                                                                                                                          Instances For
                                                                                                                                            @[inline]
                                                                                                                                            def Vector.findSomeRevM? {m : Type u_1 → Type u_2} {α : Type u_3} {β : Type u_1} {n : Nat} [Monad m] (f : αm (Option β)) (as : Vector α n) :
                                                                                                                                            m (Option β)
                                                                                                                                            Equations
                                                                                                                                            Instances For
                                                                                                                                              @[inline]
                                                                                                                                              def Vector.find? {n : Nat} {α : Type} (f : αBool) (as : Vector α n) :
                                                                                                                                              Equations
                                                                                                                                              Instances For
                                                                                                                                                @[inline]
                                                                                                                                                def Vector.findRev? {n : Nat} {α : Type} (f : αBool) (as : Vector α n) :
                                                                                                                                                Equations
                                                                                                                                                Instances For
                                                                                                                                                  @[inline]
                                                                                                                                                  def Vector.findSome? {α : Type u_1} {β : Type u_2} {n : Nat} (f : αOption β) (as : Vector α n) :
                                                                                                                                                  Equations
                                                                                                                                                  Instances For
                                                                                                                                                    @[inline]
                                                                                                                                                    def Vector.findSomeRev? {α : Type u_1} {β : Type u_2} {n : Nat} (f : αOption β) (as : Vector α n) :
                                                                                                                                                    Equations
                                                                                                                                                    Instances For
                                                                                                                                                      @[inline]
                                                                                                                                                      def Vector.isPrefixOf {α : Type u_1} {m n : Nat} [BEq α] (v : Vector α m) (w : Vector α n) :

                                                                                                                                                      Returns true when v is a prefix of the vector w.

                                                                                                                                                      Equations
                                                                                                                                                      Instances For
                                                                                                                                                        @[inline]
                                                                                                                                                        def Vector.anyM {m : TypeType u_1} {α : Type u_2} {n : Nat} [Monad m] (p : αm Bool) (v : Vector α n) :

                                                                                                                                                        Returns true with the monad if p returns true for any element of the vector.

                                                                                                                                                        Equations
                                                                                                                                                        Instances For
                                                                                                                                                          @[inline]
                                                                                                                                                          def Vector.allM {m : TypeType u_1} {α : Type u_2} {n : Nat} [Monad m] (p : αm Bool) (v : Vector α n) :

                                                                                                                                                          Returns true with the monad if p returns true for all elements of the vector.

                                                                                                                                                          Equations
                                                                                                                                                          Instances For
                                                                                                                                                            @[inline]
                                                                                                                                                            def Vector.any {α : Type u_1} {n : Nat} (v : Vector α n) (p : αBool) :

                                                                                                                                                            Returns true if p returns true for any element of the vector.

                                                                                                                                                            Equations
                                                                                                                                                            Instances For
                                                                                                                                                              @[inline]
                                                                                                                                                              def Vector.all {α : Type u_1} {n : Nat} (v : Vector α n) (p : αBool) :

                                                                                                                                                              Returns true if p returns true for all elements of the vector.

                                                                                                                                                              Equations
                                                                                                                                                              Instances For
                                                                                                                                                                @[inline]
                                                                                                                                                                def Vector.countP {α : Type u_1} {n : Nat} (p : αBool) (v : Vector α n) :

                                                                                                                                                                Count the number of elements of a vector that satisfy the predicate p.

                                                                                                                                                                Equations
                                                                                                                                                                Instances For
                                                                                                                                                                  @[inline]
                                                                                                                                                                  def Vector.count {α : Type u_1} {n : Nat} [BEq α] (a : α) (v : Vector α n) :

                                                                                                                                                                  Count the number of elements of a vector that are equal to a.

                                                                                                                                                                  Equations
                                                                                                                                                                  Instances For

                                                                                                                                                                    ForIn instance #

                                                                                                                                                                    @[simp]
                                                                                                                                                                    theorem Vector.mem_toArray_iff {α : Type u_1} {n : Nat} (a : α) (v : Vector α n) :
                                                                                                                                                                    a v.toArray a v
                                                                                                                                                                    instance Vector.instForIn'InferInstanceMembership {m : Type u_1 → Type u_2} {α : Type u_3} {n : Nat} :
                                                                                                                                                                    Equations
                                                                                                                                                                    • One or more equations did not get rendered due to their size.

                                                                                                                                                                    ForM instance #

                                                                                                                                                                    instance Vector.instForM {m : Type u_1 → Type u_2} {α : Type u_3} {n : Nat} :
                                                                                                                                                                    ForM m (Vector α n) α
                                                                                                                                                                    Equations
                                                                                                                                                                    @[simp]
                                                                                                                                                                    theorem Vector.forM_eq_forM {m : Type u_1 → Type u_2} {α : Type u_3} {n✝ : Nat} {v : Vector α n✝} [Monad m] (f : αm PUnit) :
                                                                                                                                                                    v.forM f = forM v f

                                                                                                                                                                    ToStream instance #

                                                                                                                                                                    instance Vector.instToStreamSubarray {α : Type u_1} {n : Nat} :
                                                                                                                                                                    Equations

                                                                                                                                                                    Lexicographic ordering #

                                                                                                                                                                    instance Vector.instLT {α : Type u_1} {n : Nat} [LT α] :
                                                                                                                                                                    LT (Vector α n)
                                                                                                                                                                    Equations
                                                                                                                                                                    instance Vector.instLE {α : Type u_1} {n : Nat} [LT α] :
                                                                                                                                                                    LE (Vector α n)
                                                                                                                                                                    Equations
                                                                                                                                                                    def Vector.lex {α : Type u_1} {n : Nat} [BEq α] (v w : Vector α n) (lt : ααBool := by exact (· < ·)) :

                                                                                                                                                                    Lexicographic comparator for vectors.

                                                                                                                                                                    lex v w lt is true if

                                                                                                                                                                    • v is pairwise equivalent via == to w, or
                                                                                                                                                                    • there is an index i such that lt v[i] w[i], and for all j < i, v[j] == w[j].
                                                                                                                                                                    Equations
                                                                                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                                                                                    Instances For