Documentation

Init.Data.Repr

class Repr (α : Type u) :
Type u
Instances
@[inline]
abbrev repr {α : Type u_1} [inst : Repr α] (a : α) :
Equations
@[inline]
abbrev reprStr {α : Type u_1} [inst : Repr α] (a : α) :
Equations
@[inline]
abbrev reprArg {α : Type u_1} [inst : Repr α] (a : α) :
Equations
instance instReprIdType {α : Type u_1} [inst : Repr α] :
Repr (id α)
Equations
instance instReprId {α : Type u_1} [inst : Repr α] :
Repr (Id α)
Equations
Equations
Equations
instance instReprDecidable {p : Prop} :
Equations
  • One or more equations did not get rendered due to their size.
Equations
instance instReprULift {α : Type u_1} [inst : Repr α] :
Repr (ULift α)
Equations
Equations
instance instReprOption {α : Type u_1} [inst : Repr α] :
Equations
  • One or more equations did not get rendered due to their size.
instance instReprSum {α : Type u_1} {β : Type u_2} [inst : Repr α] [inst : Repr β] :
Repr (α β)
Equations
  • One or more equations did not get rendered due to their size.
class ReprTuple (α : Type u) :
Type u
Instances
instance instReprTuple {α : Type u_1} [inst : Repr α] :
Equations
  • instReprTuple = { reprTuple := fun a xs => repr a :: xs }
instance instReprTupleProd {α : Type u_1} {β : Type u_2} [inst : Repr α] [inst : ReprTuple β] :
ReprTuple (α × β)
Equations
  • instReprTupleProd = { reprTuple := fun x x_1 => match x, x_1 with | (a, b), xs => reprTuple b (repr a :: xs) }
instance instReprProd {α : Type u_1} {β : Type u_2} [inst : Repr α] [inst : ReprTuple β] :
Repr (α × β)
Equations
  • One or more equations did not get rendered due to their size.
instance instReprSigma {α : Type u_1} {β : αType v} [inst : Repr α] [inst : (x : α) → Repr (β x)] :
Repr (Sigma β)
Equations
  • One or more equations did not get rendered due to their size.
instance instReprSubtype {α : Type u_1} {p : αProp} [inst : Repr α] :
Equations
  • instReprSubtype = { reprPrec := fun s prec => reprPrec s.val prec }
Equations
  • One or more equations did not get rendered due to their size.
def Nat.toDigitsCore (base : Nat) :
NatNatList CharList Char
Equations
  • One or more equations did not get rendered due to their size.
  • Nat.toDigitsCore base 0 _fun_discr _fun_discr = _fun_discr
def Nat.toDigits (base : Nat) (n : Nat) :
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
def charToHex (c : Char) :
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
Equations
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
instance instReprFin (n : Nat) :
Repr (Fin n)
Equations
Equations
Equations
Equations
Equations
Equations
instance instReprList {α : Type u_1} [inst : Repr α] :
Repr (List α)
Equations
  • One or more equations did not get rendered due to their size.
instance instReprList_1 {α : Type u_1} [inst : Repr α] [inst : ReprAtom α] :
Repr (List α)
Equations
  • One or more equations did not get rendered due to their size.