Idris2Doc : Data.Fin.Split

Data.Fin.Split(source)

Splitting operations and their properties

Reexports

importpublic Data.Fin

Definitions

indexSum : Either (Finm) (Finn) ->Fin (m+n)
  Converts `Fin`s that are used as indexes of parts to an index of a sum.

For example, if you have a `Vect` that is a concatenation of two `Vect`s and
you have an index either in the first or the second of the original `Vect`s,
using this function you can get an index in the concatenated one.

Totality: total
Visibility: public export
splitSum : Fin (m+n) ->Either (Finm) (Finn)
  Extracts an index of the first or the second part from the index of a sum.

For example, if you have a `Vect` that is a concatenation of the `Vect`s and
you have an index of this `Vect`, you have get an index of either left or right
original `Vect` using this function.

Totality: total
Visibility: public export
indexProd : Finm->Finn->Fin (m*n)
  Calculates the index of a square matrix of size `a * b` by indices of each side.

Totality: total
Visibility: public export
splitProd : Fin (m*n) -> (Finm, Finn)
  Splits the index of a square matrix of size `a * b` to indices of each side.

Totality: total
Visibility: public export
indexSumPreservesLast : (m : Nat) -> (n : Nat) ->indexSum (Rightlast) ~~~last
Totality: total
Visibility: export
indexProdPreservesLast : (m : Nat) -> (n : Nat) ->indexProdlastlast=last
Totality: total
Visibility: export
splitSumOfWeakenN : (k : Finm) ->splitSum (weakenNnk) =Leftk
Totality: total
Visibility: export
splitSumOfShift : (k : Finn) ->splitSum (shiftmk) =Rightk
Totality: total
Visibility: export
splitOfIndexSumInverse : (e : Either (Finm) (Finn)) ->splitSum (indexSume) =e
Totality: total
Visibility: export
indexOfSplitSumInverse : (f : Fin (m+n)) ->indexSum (splitSumf) =f
Totality: total
Visibility: export
splitOfIndexProdInverse : (k : Finm) -> (l : Finn) ->splitProd (indexProdkl) = (k, l)
Totality: total
Visibility: export
indexOfSplitProdInverse : (f : Fin (m*n)) ->uncurryindexProd (splitProdf) =f
Totality: total
Visibility: export