def
Std.DTreeMap.Internal.Zipper.prependMapGE
{α : Type u}
{β : α → Type v}
[Ord α]
(t : Impl α β)
(lowerBound : α)
(it : Zipper α β)
:
Zipper α β
Equations
- One or more equations did not get rendered due to their size.
- Std.DTreeMap.Internal.Zipper.prependMapGE Std.DTreeMap.Internal.Impl.leaf lowerBound it = it
Instances For
def
Std.DTreeMap.Internal.Zipper.prependMapGT
{α : Type u}
{β : α → Type v}
[Ord α]
(t : Impl α β)
(lowerBound : α)
(it : Zipper α β)
:
Zipper α β
Equations
- One or more equations did not get rendered due to their size.
- Std.DTreeMap.Internal.Zipper.prependMapGT Std.DTreeMap.Internal.Impl.leaf lowerBound it = it
Instances For
def
Std.DTreeMap.Internal.Zipper.step
{α : Type u}
{β : α → Type v}
:
Zipper α β → Iterators.IterStep (IterM Id ((a : α) × β a)) ((a : α) × β a)
Equations
- Std.DTreeMap.Internal.Zipper.done.step = Std.Iterators.IterStep.done
- (Std.DTreeMap.Internal.Zipper.cons k v tree next).step = Std.Iterators.IterStep.yield { internalState := Std.DTreeMap.Internal.Zipper.prependMap tree next } ⟨k, v⟩
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.
instance
Std.DTreeMap.Internal.instIteratorCollectZipperIdSigma
{α : Type u}
{β : α → Type v}
:
Iterators.IteratorCollect (Zipper α β) Id Id
instance
Std.DTreeMap.Internal.Zipper.instFinite
{α : Type u}
{β : α → Type v}
:
Iterators.Finite (Zipper α β) Id
def
Std.DTreeMap.Internal.Zipper.iterOfTree
{α : Type u}
{β : α → Type v}
(t : Impl α β)
:
Iter ((a : α) × β a)
Equations
Instances For
instance
Std.DTreeMap.Internal.instToIteratorZipperIdSigma
{α : Type u}
{β : α → Type v}
{z : Zipper α β}
:
Iterators.ToIterator z Id ((a : α) × β a)
Equations
- Std.DTreeMap.Internal.instToIteratorZipperIdSigma = { State := Std.DTreeMap.Internal.Zipper α β, iterMInternal := z.iter.toIterM }
theorem
Std.DTreeMap.Internal.Zipper.toList_iterOfTree
{α : Type u}
{β : α → Type v}
(t : Impl α β)
:
def
Std.DTreeMap.Internal.RxcIterator.step
{α : Type u}
{β : α → Type v}
[Ord α]
:
RxcIterator α β → Iterators.IterStep (IterM Id ((a : α) × β a)) ((a : α) × β a)
Equations
- One or more equations did not get rendered due to their size.
- { iter := Std.DTreeMap.Internal.Zipper.done, upper := upper }.step = Std.Iterators.IterStep.done
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.instIteratorCollectRxcIteratorIdSigma
{α : Type u}
{β : α → Type v}
[Ord α]
:
instance
Std.DTreeMap.Internal.instFinite
{α : Type u}
{β : α → Type v}
[Ord α]
:
Iterators.Finite (RxcIterator α β) Id
def
Std.DTreeMap.Internal.RxoIterator.step
{α : Type u}
{β : α → Type v}
[Ord α]
:
RxoIterator α β → Iterators.IterStep (IterM Id ((a : α) × β a)) ((a : α) × β a)
Equations
- One or more equations did not get rendered due to their size.
- { iter := Std.DTreeMap.Internal.Zipper.done, upper := upper }.step = Std.Iterators.IterStep.done
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.
instance
Std.DTreeMap.Internal.instIteratorCollectRxoIteratorIdSigma
{α : Type u}
{β : α → Type v}
[Ord α]
:
instance
Std.DTreeMap.Internal.Rxo.instFinite
{α : Type u}
{β : α → Type v}
[Ord α]
:
Iterators.Finite (RxoIterator α β) Id
@[reducible, inline]
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
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRicSlice
{α : Type u}
[Ord α]
:
Ric.Sliceable (Impl α fun (x : α) => Unit) α (RicSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRicSliceId
{α : Type u_1}
[Ord α]
{s : RicSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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)
@[reducible, inline]
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
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRioSlice
{α : Type u}
[Ord α]
:
Rio.Sliceable (Impl α fun (x : α) => Unit) α (RioSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRioSliceId
{α : Type u_1}
[Ord α]
{s : RioSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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)
@[reducible, inline]
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.
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRccSlice
{α : Type u}
[Ord α]
:
Rcc.Sliceable (Impl α fun (x : α) => Unit) α (RccSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRccSliceId
{α : Type u_1}
[Ord α]
{s : RccSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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)
@[reducible, inline]
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.
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRcoSlice
{α : Type u}
[Ord α]
:
Rco.Sliceable (Impl α fun (x : α) => Unit) α (RcoSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRcoSliceId
{α : Type u_1}
[Ord α]
{s : RcoSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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)
@[reducible, inline]
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.
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRooSlice
{α : Type u}
[Ord α]
:
Roo.Sliceable (Impl α fun (x : α) => Unit) α (RooSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRooSliceId
{α : Type u_1}
[Ord α]
{s : RooSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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)
@[reducible, inline]
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.
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRocSlice
{α : Type u}
[Ord α]
:
Roc.Sliceable (Impl α fun (x : α) => Unit) α (RocSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRocSliceId
{α : Type u_1}
[Ord α]
{s : RocSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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
- Std.DTreeMap.Internal.rciIterator t lowerBound = { internalState := Std.DTreeMap.Internal.Zipper.prependMapGE t lowerBound Std.DTreeMap.Internal.Zipper.done }
Instances For
@[reducible, inline]
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
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRciSlice
{α : Type u}
[Ord α]
:
Rci.Sliceable (Impl α fun (x : α) => Unit) α (RciSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRciSliceId
{α : Type u_1}
[Ord α]
{s : RciSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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
- Std.DTreeMap.Internal.roiIterator t lowerBound = { internalState := Std.DTreeMap.Internal.Zipper.prependMapGT t lowerBound Std.DTreeMap.Internal.Zipper.done }
Instances For
@[reducible, inline]
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
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRoiSlice
{α : Type u}
[Ord α]
:
Roi.Sliceable (Impl α fun (x : α) => Unit) α (RoiSlice α)
Equations
- One or more equations did not get rendered due to their size.
instance
Std.DTreeMap.Internal.Unit.instToIteratorRoiSliceId
{α : Type u_1}
[Ord α]
{s : RoiSlice α}
:
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
@[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 α β}
:
Iterators.ToIterator s Id (α × β)
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
@[reducible, inline]
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.
instance
Std.DTreeMap.Internal.instToIteratorRiiSliceIdSigma
{α : Type u_1}
{β : α → Type u_2}
{s : RiiSlice α β}
:
Iterators.ToIterator s Id ((a : α) × β a)
@[reducible, inline]
Equations
Instances For
instance
Std.DTreeMap.Internal.Unit.instSliceableImplUnitRiiSlice
{α : Type u}
:
Rii.Sliceable (Impl α fun (x : α) => Unit) α (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.
@[reducible, inline]
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.
instance
Std.DTreeMap.Internal.Const.instToIteratorRiiSliceIdProd
{α : Type u_1}
{β : Type u_2}
{s : RiiSlice α β}
:
Iterators.ToIterator s Id (α × β)
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 : α) => β)
: