Documentation

Std.Data.DTreeMap.Internal.Zipper

inductive Std.DTreeMap.Internal.Zipper (α : Type u) (β : αType v) :
Type (max u v)
Instances For
    def Std.DTreeMap.Internal.Zipper.toList {α : Type u} {β : αType v} :
    Zipper α βList ((a : α) × β a)
    Equations
    Instances For
      def Std.DTreeMap.Internal.Zipper.Ordered {α : Type u} {β : αType v} [Ord α] (t : Zipper α β) :
      Equations
      Instances For
        def Std.DTreeMap.Internal.Zipper.prependMapGE {α : Type u} {β : αType v} [Ord α] (t : Impl α β) (lowerBound : α) (it : Zipper α β) :
        Zipper α β
        Equations
        Instances For
          def Std.DTreeMap.Internal.Zipper.prependMapGT {α : Type u} {β : αType v} [Ord α] (t : Impl α β) (lowerBound : α) (it : Zipper α β) :
          Zipper α β
          Equations
          Instances For
            instance Std.DTreeMap.Internal.instIteratorZipperIdSigma {α : Type u} {β : αType v} :
            Iterators.Iterator (Zipper α β) Id ((a : α) × β a)
            Equations
            • One or more equations did not get rendered due to their size.
            def Std.DTreeMap.Internal.Zipper.iter {α : Type u} {β : αType v} (t : Zipper α β) :
            Iter ((a : α) × β a)
            Equations
            Instances For
              instance Std.DTreeMap.Internal.instToIteratorZipperIdSigma {α : Type u} {β : αType v} {z : Zipper α β} :
              Iterators.ToIterator z Id ((a : α) × β a)
              Equations
              theorem Std.DTreeMap.Internal.Zipper.toList_iterOfTree {α : Type u} {β : αType v} (t : Impl α β) :
              structure Std.DTreeMap.Internal.RxcIterator (α : Type u) (β : αType v) [Ord α] :
              Type (max u v)
              Instances For
                def Std.DTreeMap.Internal.RxcIterator.step {α : Type u} {β : αType v} [Ord α] :
                RxcIterator α βIterators.IterStep (IterM Id ((a : α) × β a)) ((a : α) × β a)
                Equations
                Instances For
                  instance Std.DTreeMap.Internal.instIteratorRxcIteratorIdSigma {α : Type u} {β : αType v} [Ord α] :
                  Iterators.Iterator (RxcIterator α β) Id ((a : α) × β a)
                  Equations
                  • One or more equations did not get rendered due to their size.
                  instance Std.DTreeMap.Internal.instFinite {α : Type u} {β : αType v} [Ord α] :
                  theorem Std.DTreeMap.Internal.RxcIterator.takeWhile_toList {α : Type u_1} {β : αType u_2} [Ord α] [TransOrd α] {z : Zipper α β} {bound : α} {z_ord : z.Ordered} :
                  List.takeWhile (fun (e : (a : α) × β a) => (compare e.fst bound).isLE) z.toList = List.filter (fun (e : (a : α) × β a) => (compare e.fst bound).isLE) z.toList
                  structure Std.DTreeMap.Internal.RxoIterator (α : Type u) (β : αType v) [Ord α] :
                  Type (max u v)
                  Instances For
                    def Std.DTreeMap.Internal.RxoIterator.step {α : Type u} {β : αType v} [Ord α] :
                    RxoIterator α βIterators.IterStep (IterM Id ((a : α) × β a)) ((a : α) × β a)
                    Equations
                    Instances For
                      instance Std.DTreeMap.Internal.instIteratorRxoIteratorIdSigma {α : Type u} {β : αType v} [Ord α] :
                      Iterators.Iterator (RxoIterator α β) Id ((a : α) × β a)
                      Equations
                      • One or more equations did not get rendered due to their size.
                      theorem Std.DTreeMap.Internal.RxoIterator.takeWhile_toList {α : Type u_1} {β : αType u_2} [Ord α] [TransOrd α] {z : Zipper α β} {bound : α} {z_ord : z.Ordered} :
                      List.takeWhile (fun (e : (a : α) × β a) => (compare e.fst bound).isLT) z.toList = List.filter (fun (e : (a : α) × β a) => (compare e.fst bound).isLT) z.toList
                      structure Std.DTreeMap.Internal.RicSliceData (α : Type u) (β : αType v) [Ord α] :
                      Type (max u v)
                      Instances For
                        @[reducible, inline]
                        abbrev Std.DTreeMap.Internal.RicSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                        Type (max u_2 u_1)
                        Equations
                        Instances For
                          instance Std.DTreeMap.Internal.instSliceableImplRicSlice {α : Type u} {β : αType v} [Ord α] :
                          Ric.Sliceable (Impl α β) α (RicSlice α β)
                          Equations
                          • One or more equations did not get rendered due to their size.
                          instance Std.DTreeMap.Internal.instToIteratorRicSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RicSlice α β} :
                          Iterators.ToIterator s Id ((a : α) × β a)
                          Equations
                          • One or more equations did not get rendered due to their size.
                          theorem Std.DTreeMap.Internal.toList_ric {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (bound : α) :
                          Slice.toList (Ric.Sliceable.mkSlice t *...=bound) = List.filter (fun (e : (a : α) × β a) => (compare e.fst bound).isLE) t.toList
                          Instances For
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Equations
                            • One or more equations did not get rendered due to their size.
                            theorem Std.DTreeMap.Internal.Unit.toList_ric {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (bound : α) :
                            Slice.toList (Ric.Sliceable.mkSlice t *...=bound) = List.filter (fun (e : α) => (compare e bound).isLE) t.keys
                            structure Std.DTreeMap.Internal.Const.RicSliceData (α : Type u) (β : Type v) [Ord α] :
                            Type (max u v)
                            • treeMap : Impl α fun (x : α) => β
                            • range : Ric α
                            Instances For
                              @[reducible, inline]
                              abbrev Std.DTreeMap.Internal.Const.RicSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                              Type (max u_2 u_1)
                              Equations
                              Instances For
                                instance Std.DTreeMap.Internal.Const.instSliceableImplRicSlice {α : Type u} {β : Type v} [Ord α] :
                                Ric.Sliceable (Impl α fun (x : α) => β) α (RicSlice α β)
                                Equations
                                • One or more equations did not get rendered due to their size.
                                instance Std.DTreeMap.Internal.Const.instToIteratorRicSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RicSlice α β} :
                                Equations
                                • One or more equations did not get rendered due to their size.
                                theorem Std.DTreeMap.Internal.Const.toList_ric {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (bound : α) :
                                Slice.toList (Ric.Sliceable.mkSlice t *...=bound) = List.filter (fun (e : α × β) => (compare e.fst bound).isLE) (Impl.Const.toList t)
                                structure Std.DTreeMap.Internal.RioSliceData (α : Type u) (β : αType v) [Ord α] :
                                Type (max u v)
                                Instances For
                                  @[reducible, inline]
                                  abbrev Std.DTreeMap.Internal.RioSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                  Type (max u_2 u_1)
                                  Equations
                                  Instances For
                                    instance Std.DTreeMap.Internal.instSliceableImplRioSlice {α : Type u} {β : αType v} [Ord α] :
                                    Rio.Sliceable (Impl α β) α (RioSlice α β)
                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    instance Std.DTreeMap.Internal.instToIteratorRioSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RioSlice α β} :
                                    Iterators.ToIterator s Id ((a : α) × β a)
                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    theorem Std.DTreeMap.Internal.toList_rio {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (bound : α) :
                                    Slice.toList (Rio.Sliceable.mkSlice t *...bound) = List.filter (fun (e : (a : α) × β a) => (compare e.fst bound).isLT) t.toList
                                    Instances For
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      theorem Std.DTreeMap.Internal.Unit.toList_rio {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (bound : α) :
                                      Slice.toList (Rio.Sliceable.mkSlice t *...bound) = List.filter (fun (e : α) => (compare e bound).isLT) t.keys
                                      structure Std.DTreeMap.Internal.Const.RioSliceData (α : Type u) (β : Type v) [Ord α] :
                                      Type (max u v)
                                      • treeMap : Impl α fun (x : α) => β
                                      • range : Rio α
                                      Instances For
                                        @[reducible, inline]
                                        abbrev Std.DTreeMap.Internal.Const.RioSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                        Type (max u_2 u_1)
                                        Equations
                                        Instances For
                                          instance Std.DTreeMap.Internal.Const.instSliceableImplRioSlice {α : Type u} {β : Type v} [Ord α] :
                                          Rio.Sliceable (Impl α fun (x : α) => β) α (RioSlice α β)
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          instance Std.DTreeMap.Internal.Const.instToIteratorRioSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RioSlice α β} :
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          theorem Std.DTreeMap.Internal.Const.toList_rio {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (bound : α) :
                                          Slice.toList (Rio.Sliceable.mkSlice t *...bound) = List.filter (fun (e : α × β) => (compare e.fst bound).isLT) (Impl.Const.toList t)
                                          @[always_inline]
                                          def Std.DTreeMap.Internal.rccIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound upperBound : α) :
                                          Iter ((a : α) × β a)
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For
                                            structure Std.DTreeMap.Internal.RccSliceData (α : Type u) (β : αType v) [Ord α] :
                                            Type (max u v)
                                            Instances For
                                              @[reducible, inline]
                                              abbrev Std.DTreeMap.Internal.RccSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                              Type (max u_2 u_1)
                                              Equations
                                              Instances For
                                                instance Std.DTreeMap.Internal.instSliceableImplRccSlice {α : Type u} {β : αType v} [Ord α] :
                                                Rcc.Sliceable (Impl α β) α (RccSlice α β)
                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                instance Std.DTreeMap.Internal.instToIteratorRccSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RccSlice α β} :
                                                Iterators.ToIterator s Id ((a : α) × β a)
                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                theorem Std.DTreeMap.Internal.toList_rcc {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                Slice.toList (Rcc.Sliceable.mkSlice t lowerBound...=upperBound) = List.filter (fun (e : (a : α) × β a) => decide ((compare e.fst lowerBound).isGE = true (compare e.fst upperBound).isLE = true)) t.toList
                                                Instances For
                                                  Equations
                                                  • One or more equations did not get rendered due to their size.
                                                  Equations
                                                  • One or more equations did not get rendered due to their size.
                                                  theorem Std.DTreeMap.Internal.Unit.toList_rcc {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                  Slice.toList (Rcc.Sliceable.mkSlice t lowerBound...=upperBound) = List.filter (fun (e : α) => decide ((compare e lowerBound).isGE = true (compare e upperBound).isLE = true)) t.keys
                                                  structure Std.DTreeMap.Internal.Const.RccSliceData (α : Type u) (β : Type v) [Ord α] :
                                                  Type (max u v)
                                                  • treeMap : Impl α fun (x : α) => β
                                                  • range : Rcc α
                                                  Instances For
                                                    @[reducible, inline]
                                                    abbrev Std.DTreeMap.Internal.Const.RccSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                    Type (max u_2 u_1)
                                                    Equations
                                                    Instances For
                                                      instance Std.DTreeMap.Internal.Const.instSliceableImplRccSlice {α : Type u} {β : Type v} [Ord α] :
                                                      Rcc.Sliceable (Impl α fun (x : α) => β) α (RccSlice α β)
                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      instance Std.DTreeMap.Internal.Const.instToIteratorRccSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RccSlice α β} :
                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      theorem Std.DTreeMap.Internal.Const.toList_rcc {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                      Slice.toList (Rcc.Sliceable.mkSlice t lowerBound...=upperBound) = List.filter (fun (e : α × β) => decide ((compare e.fst lowerBound).isGE = true (compare e.fst upperBound).isLE = true)) (Impl.Const.toList t)
                                                      @[always_inline]
                                                      def Std.DTreeMap.Internal.rcoIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound upperBound : α) :
                                                      Iter ((a : α) × β a)
                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      Instances For
                                                        structure Std.DTreeMap.Internal.RcoSliceData (α : Type u) (β : αType v) [Ord α] :
                                                        Type (max u v)
                                                        Instances For
                                                          @[reducible, inline]
                                                          abbrev Std.DTreeMap.Internal.RcoSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                                          Type (max u_2 u_1)
                                                          Equations
                                                          Instances For
                                                            instance Std.DTreeMap.Internal.instSliceableImplRcoSlice {α : Type u} {β : αType v} [Ord α] :
                                                            Rco.Sliceable (Impl α β) α (RcoSlice α β)
                                                            Equations
                                                            • One or more equations did not get rendered due to their size.
                                                            instance Std.DTreeMap.Internal.instToIteratorRcoSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RcoSlice α β} :
                                                            Iterators.ToIterator s Id ((a : α) × β a)
                                                            Equations
                                                            • One or more equations did not get rendered due to their size.
                                                            theorem Std.DTreeMap.Internal.toList_rco {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                            Slice.toList (Rco.Sliceable.mkSlice t lowerBound...upperBound) = List.filter (fun (e : (a : α) × β a) => decide ((compare e.fst lowerBound).isGE = true (compare e.fst upperBound).isLT = true)) t.toList
                                                            Instances For
                                                              Equations
                                                              • One or more equations did not get rendered due to their size.
                                                              Equations
                                                              • One or more equations did not get rendered due to their size.
                                                              theorem Std.DTreeMap.Internal.Unit.toList_rco {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                              Slice.toList (Rco.Sliceable.mkSlice t lowerBound...upperBound) = List.filter (fun (e : α) => decide ((compare e lowerBound).isGE = true (compare e upperBound).isLT = true)) t.keys
                                                              structure Std.DTreeMap.Internal.Const.RcoSliceData (α : Type u) (β : Type v) [Ord α] :
                                                              Type (max u v)
                                                              • treeMap : Impl α fun (x : α) => β
                                                              • range : Rco α
                                                              Instances For
                                                                @[reducible, inline]
                                                                abbrev Std.DTreeMap.Internal.Const.RcoSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                                Type (max u_2 u_1)
                                                                Equations
                                                                Instances For
                                                                  instance Std.DTreeMap.Internal.Const.instSliceableImplRcoSlice {α : Type u} {β : Type v} [Ord α] :
                                                                  Rco.Sliceable (Impl α fun (x : α) => β) α (RcoSlice α β)
                                                                  Equations
                                                                  • One or more equations did not get rendered due to their size.
                                                                  instance Std.DTreeMap.Internal.Const.instToIteratorRcoSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RcoSlice α β} :
                                                                  Equations
                                                                  • One or more equations did not get rendered due to their size.
                                                                  theorem Std.DTreeMap.Internal.Const.toList_rco {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                  Slice.toList (Rco.Sliceable.mkSlice t lowerBound...upperBound) = List.filter (fun (e : α × β) => decide ((compare e.fst lowerBound).isGE = true (compare e.fst upperBound).isLT = true)) (Impl.Const.toList t)
                                                                  @[always_inline]
                                                                  def Std.DTreeMap.Internal.rooIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound upperBound : α) :
                                                                  Iter ((a : α) × β a)
                                                                  Equations
                                                                  • One or more equations did not get rendered due to their size.
                                                                  Instances For
                                                                    structure Std.DTreeMap.Internal.RooSliceData (α : Type u) (β : αType v) [Ord α] :
                                                                    Type (max u v)
                                                                    Instances For
                                                                      @[reducible, inline]
                                                                      abbrev Std.DTreeMap.Internal.RooSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                                                      Type (max u_2 u_1)
                                                                      Equations
                                                                      Instances For
                                                                        instance Std.DTreeMap.Internal.instSliceableImplRooSlice {α : Type u} {β : αType v} [Ord α] :
                                                                        Roo.Sliceable (Impl α β) α (RooSlice α β)
                                                                        Equations
                                                                        • One or more equations did not get rendered due to their size.
                                                                        instance Std.DTreeMap.Internal.instToIteratorRooSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RooSlice α β} :
                                                                        Iterators.ToIterator s Id ((a : α) × β a)
                                                                        Equations
                                                                        • One or more equations did not get rendered due to their size.
                                                                        theorem Std.DTreeMap.Internal.toList_roo {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                        Slice.toList (Roo.Sliceable.mkSlice t lowerBound<...upperBound) = List.filter (fun (e : (a : α) × β a) => decide ((compare e.fst lowerBound).isGT = true (compare e.fst upperBound).isLT = true)) t.toList
                                                                        Instances For
                                                                          Equations
                                                                          • One or more equations did not get rendered due to their size.
                                                                          Equations
                                                                          • One or more equations did not get rendered due to their size.
                                                                          theorem Std.DTreeMap.Internal.Unit.toList_roo {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                          Slice.toList (Roo.Sliceable.mkSlice t lowerBound<...upperBound) = List.filter (fun (e : α) => decide ((compare e lowerBound).isGT = true (compare e upperBound).isLT = true)) t.keys
                                                                          structure Std.DTreeMap.Internal.Const.RooSliceData (α : Type u) (β : Type v) [Ord α] :
                                                                          Type (max u v)
                                                                          • treeMap : Impl α fun (x : α) => β
                                                                          • range : Roo α
                                                                          Instances For
                                                                            @[reducible, inline]
                                                                            abbrev Std.DTreeMap.Internal.Const.RooSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                                            Type (max u_2 u_1)
                                                                            Equations
                                                                            Instances For
                                                                              instance Std.DTreeMap.Internal.Const.instSliceableImplRooSlice {α : Type u} {β : Type v} [Ord α] :
                                                                              Roo.Sliceable (Impl α fun (x : α) => β) α (RooSlice α β)
                                                                              Equations
                                                                              • One or more equations did not get rendered due to their size.
                                                                              instance Std.DTreeMap.Internal.Const.instToIteratorRooSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RooSlice α β} :
                                                                              Equations
                                                                              • One or more equations did not get rendered due to their size.
                                                                              theorem Std.DTreeMap.Internal.Const.toList_roo {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                              Slice.toList (Roo.Sliceable.mkSlice t lowerBound<...upperBound) = List.filter (fun (e : α × β) => decide ((compare e.fst lowerBound).isGT = true (compare e.fst upperBound).isLT = true)) (Impl.Const.toList t)
                                                                              @[always_inline]
                                                                              def Std.DTreeMap.Internal.rocIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound upperBound : α) :
                                                                              Iter ((a : α) × β a)
                                                                              Equations
                                                                              • One or more equations did not get rendered due to their size.
                                                                              Instances For
                                                                                structure Std.DTreeMap.Internal.RocSliceData (α : Type u) (β : αType v) [Ord α] :
                                                                                Type (max u v)
                                                                                Instances For
                                                                                  @[reducible, inline]
                                                                                  abbrev Std.DTreeMap.Internal.RocSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                                                                  Type (max u_2 u_1)
                                                                                  Equations
                                                                                  Instances For
                                                                                    instance Std.DTreeMap.Internal.instSliceableImplRocSlice {α : Type u} {β : αType v} [Ord α] :
                                                                                    Roc.Sliceable (Impl α β) α (RocSlice α β)
                                                                                    Equations
                                                                                    • One or more equations did not get rendered due to their size.
                                                                                    instance Std.DTreeMap.Internal.instToIteratorRocSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RocSlice α β} :
                                                                                    Iterators.ToIterator s Id ((a : α) × β a)
                                                                                    Equations
                                                                                    • One or more equations did not get rendered due to their size.
                                                                                    theorem Std.DTreeMap.Internal.toList_roc {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                                    Slice.toList (Roc.Sliceable.mkSlice t lowerBound<...=upperBound) = List.filter (fun (e : (a : α) × β a) => decide ((compare e.fst lowerBound).isGT = true (compare e.fst upperBound).isLE = true)) t.toList
                                                                                    Instances For
                                                                                      Equations
                                                                                      • One or more equations did not get rendered due to their size.
                                                                                      Equations
                                                                                      • One or more equations did not get rendered due to their size.
                                                                                      theorem Std.DTreeMap.Internal.Unit.toList_roc {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                                      Slice.toList (Roc.Sliceable.mkSlice t lowerBound<...=upperBound) = List.filter (fun (e : α) => decide ((compare e lowerBound).isGT = true (compare e upperBound).isLE = true)) t.keys
                                                                                      structure Std.DTreeMap.Internal.Const.RocSliceData (α : Type u) (β : Type v) [Ord α] :
                                                                                      Type (max u v)
                                                                                      • treeMap : Impl α fun (x : α) => β
                                                                                      • range : Roc α
                                                                                      Instances For
                                                                                        @[reducible, inline]
                                                                                        abbrev Std.DTreeMap.Internal.Const.RocSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                                                        Type (max u_2 u_1)
                                                                                        Equations
                                                                                        Instances For
                                                                                          instance Std.DTreeMap.Internal.Const.instSliceableImplRocSlice {α : Type u} {β : Type v} [Ord α] :
                                                                                          Roc.Sliceable (Impl α fun (x : α) => β) α (RocSlice α β)
                                                                                          Equations
                                                                                          • One or more equations did not get rendered due to their size.
                                                                                          instance Std.DTreeMap.Internal.Const.instToIteratorRocSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RocSlice α β} :
                                                                                          Equations
                                                                                          • One or more equations did not get rendered due to their size.
                                                                                          theorem Std.DTreeMap.Internal.Const.toList_roc {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound upperBound : α) :
                                                                                          Slice.toList (Roc.Sliceable.mkSlice t lowerBound<...=upperBound) = List.filter (fun (e : α × β) => decide ((compare e.fst lowerBound).isGT = true (compare e.fst upperBound).isLE = true)) (Impl.Const.toList t)
                                                                                          @[always_inline]
                                                                                          def Std.DTreeMap.Internal.rciIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound : α) :
                                                                                          Iter ((a : α) × β a)
                                                                                          Equations
                                                                                          Instances For
                                                                                            structure Std.DTreeMap.Internal.RciSliceData (α : Type u) (β : αType v) [Ord α] :
                                                                                            Type (max u v)
                                                                                            Instances For
                                                                                              @[reducible, inline]
                                                                                              abbrev Std.DTreeMap.Internal.RciSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                                                                              Type (max u_2 u_1)
                                                                                              Equations
                                                                                              Instances For
                                                                                                instance Std.DTreeMap.Internal.instSliceableImplRciSlice {α : Type u} {β : αType v} [Ord α] :
                                                                                                Rci.Sliceable (Impl α β) α (RciSlice α β)
                                                                                                Equations
                                                                                                • One or more equations did not get rendered due to their size.
                                                                                                instance Std.DTreeMap.Internal.instToIteratorRciSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RciSlice α β} :
                                                                                                Iterators.ToIterator s Id ((a : α) × β a)
                                                                                                Equations
                                                                                                • One or more equations did not get rendered due to their size.
                                                                                                theorem Std.DTreeMap.Internal.toList_rci {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                Slice.toList (Rci.Sliceable.mkSlice t lowerBound...*) = List.filter (fun (e : (a : α) × β a) => (compare e.fst lowerBound).isGE) t.toList
                                                                                                Instances For
                                                                                                  Equations
                                                                                                  • One or more equations did not get rendered due to their size.
                                                                                                  Equations
                                                                                                  • One or more equations did not get rendered due to their size.
                                                                                                  theorem Std.DTreeMap.Internal.Unit.toList_rci {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                  Slice.toList (Rci.Sliceable.mkSlice t lowerBound...*) = List.filter (fun (e : α) => (compare e lowerBound).isGE) t.keys
                                                                                                  structure Std.DTreeMap.Internal.Const.RciSliceData (α : Type u) (β : Type v) [Ord α] :
                                                                                                  Type (max u v)
                                                                                                  • treeMap : Impl α fun (x : α) => β
                                                                                                  • range : Rci α
                                                                                                  Instances For
                                                                                                    @[reducible, inline]
                                                                                                    abbrev Std.DTreeMap.Internal.Const.RciSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                                                                    Type (max u_2 u_1)
                                                                                                    Equations
                                                                                                    Instances For
                                                                                                      instance Std.DTreeMap.Internal.Const.instSliceableImplRciSlice {α : Type u} {β : Type v} [Ord α] :
                                                                                                      Rci.Sliceable (Impl α fun (x : α) => β) α (RciSlice α β)
                                                                                                      Equations
                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                      instance Std.DTreeMap.Internal.Const.instToIteratorRciSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RciSlice α β} :
                                                                                                      Equations
                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                      theorem Std.DTreeMap.Internal.Const.toList_rci {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                      Slice.toList (Rci.Sliceable.mkSlice t lowerBound...*) = List.filter (fun (e : α × β) => (compare e.fst lowerBound).isGE) (Impl.Const.toList t)
                                                                                                      @[always_inline]
                                                                                                      def Std.DTreeMap.Internal.roiIterator {α : Type u_1} {β : αType u_2} [Ord α] (t : Impl α β) (lowerBound : α) :
                                                                                                      Iter ((a : α) × β a)
                                                                                                      Equations
                                                                                                      Instances For
                                                                                                        structure Std.DTreeMap.Internal.RoiSliceData (α : Type u) (β : αType v) [Ord α] :
                                                                                                        Type (max u v)
                                                                                                        Instances For
                                                                                                          @[reducible, inline]
                                                                                                          abbrev Std.DTreeMap.Internal.RoiSlice (α : Type u_1) (β : αType u_2) [Ord α] :
                                                                                                          Type (max u_2 u_1)
                                                                                                          Equations
                                                                                                          Instances For
                                                                                                            instance Std.DTreeMap.Internal.instSliceableImplRoiSlice {α : Type u} {β : αType v} [Ord α] :
                                                                                                            Roi.Sliceable (Impl α β) α (RoiSlice α β)
                                                                                                            Equations
                                                                                                            • One or more equations did not get rendered due to their size.
                                                                                                            instance Std.DTreeMap.Internal.instToIteratorRoiSliceIdSigma {α : Type u_1} {β : αType u_2} [Ord α] {s : RoiSlice α β} :
                                                                                                            Iterators.ToIterator s Id ((a : α) × β a)
                                                                                                            Equations
                                                                                                            • One or more equations did not get rendered due to their size.
                                                                                                            theorem Std.DTreeMap.Internal.toList_roi {α : Type u} {β : αType v} [Ord α] [TransOrd α] (t : Impl α β) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                            Slice.toList (Roi.Sliceable.mkSlice t lowerBound<...*) = List.filter (fun (e : (a : α) × β a) => (compare e.fst lowerBound).isGT) t.toList
                                                                                                            Instances For
                                                                                                              Equations
                                                                                                              • One or more equations did not get rendered due to their size.
                                                                                                              Equations
                                                                                                              • One or more equations did not get rendered due to their size.
                                                                                                              theorem Std.DTreeMap.Internal.Unit.toList_roi {α : Type u} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => Unit) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                              Slice.toList (Roi.Sliceable.mkSlice t lowerBound<...*) = List.filter (fun (e : α) => (compare e lowerBound).isGT) t.keys
                                                                                                              structure Std.DTreeMap.Internal.Const.RoiSliceData (α : Type u) (β : Type v) [Ord α] :
                                                                                                              Type (max u v)
                                                                                                              • treeMap : Impl α fun (x : α) => β
                                                                                                              • range : Roi α
                                                                                                              Instances For
                                                                                                                @[reducible, inline]
                                                                                                                abbrev Std.DTreeMap.Internal.Const.RoiSlice (α : Type u_1) (β : Type u_2) [Ord α] :
                                                                                                                Type (max u_2 u_1)
                                                                                                                Equations
                                                                                                                Instances For
                                                                                                                  instance Std.DTreeMap.Internal.Const.instSliceableImplRoiSlice {α : Type u} {β : Type v} [Ord α] :
                                                                                                                  Roi.Sliceable (Impl α fun (x : α) => β) α (RoiSlice α β)
                                                                                                                  Equations
                                                                                                                  • One or more equations did not get rendered due to their size.
                                                                                                                  instance Std.DTreeMap.Internal.Const.instToIteratorRoiSliceIdProd {α : Type u_1} {β : Type u_2} [Ord α] {s : RoiSlice α β} :
                                                                                                                  Equations
                                                                                                                  • One or more equations did not get rendered due to their size.
                                                                                                                  theorem Std.DTreeMap.Internal.Const.toList_roi {α : Type u} {β : Type v} [Ord α] [TransOrd α] (t : Impl α fun (x : α) => β) (ordered : t.Ordered) (lowerBound : α) :
                                                                                                                  Slice.toList (Roi.Sliceable.mkSlice t lowerBound<...*) = List.filter (fun (e : α × β) => (compare e.fst lowerBound).isGT) (Impl.Const.toList t)
                                                                                                                  def Std.DTreeMap.Internal.riiIterator {α : Type u_1} {β : αType u_2} (t : Impl α β) :
                                                                                                                  Iter ((a : α) × β a)
                                                                                                                  Equations
                                                                                                                  Instances For
                                                                                                                    structure Std.DTreeMap.Internal.RiiSliceData (α : Type u) (β : αType v) :
                                                                                                                    Type (max u v)
                                                                                                                    Instances For
                                                                                                                      @[reducible, inline]
                                                                                                                      abbrev Std.DTreeMap.Internal.RiiSlice (α : Type u_1) (β : αType u_2) :
                                                                                                                      Type (max u_2 u_1)
                                                                                                                      Equations
                                                                                                                      Instances For
                                                                                                                        instance Std.DTreeMap.Internal.instSliceableImplRiiSlice {α : Type u} {β : αType v} :
                                                                                                                        Rii.Sliceable (Impl α β) α (RiiSlice α β)
                                                                                                                        Equations
                                                                                                                        • One or more equations did not get rendered due to their size.
                                                                                                                        theorem Std.DTreeMap.Internal.toList_rii {α : Type u} {β : αType v} (t : Impl α β) :
                                                                                                                        Instances For
                                                                                                                          Equations
                                                                                                                          • One or more equations did not get rendered due to their size.
                                                                                                                          Equations
                                                                                                                          • One or more equations did not get rendered due to their size.
                                                                                                                          theorem Std.DTreeMap.Internal.Unit.toList_rii {α : Type u} (t : Impl α fun (x : α) => Unit) :
                                                                                                                          structure Std.DTreeMap.Internal.Const.RiiSliceData (α : Type u) (β : Type v) :
                                                                                                                          Type (max u v)
                                                                                                                          • treeMap : Impl α fun (x : α) => β
                                                                                                                          • range : Rii α
                                                                                                                          Instances For
                                                                                                                            @[reducible, inline]
                                                                                                                            abbrev Std.DTreeMap.Internal.Const.RiiSlice (α : Type u_1) (β : Type u_2) :
                                                                                                                            Type (max u_2 u_1)
                                                                                                                            Equations
                                                                                                                            Instances For
                                                                                                                              instance Std.DTreeMap.Internal.Const.instSliceableImplRiiSlice {α : Type u} {β : Type v} :
                                                                                                                              Rii.Sliceable (Impl α fun (x : α) => β) α (RiiSlice α β)
                                                                                                                              Equations
                                                                                                                              • One or more equations did not get rendered due to their size.
                                                                                                                              Equations
                                                                                                                              • One or more equations did not get rendered due to their size.
                                                                                                                              theorem Std.DTreeMap.Internal.Const.toList_rii {α : Type u} {β : Type v} (t : Impl α fun (x : α) => β) :