Documentation

Mathlib.Util.Export

A rudimentary export format, adapted from with support for lean 4 kernel primitives.

structure Lean.Export.Alloc (α : Type u_1) [BEq α] [Hashable α] :
Type u_1
Instances For
    instance Lean.Export.instInhabitedAlloc :
    {a : Type u_1} → {a_1 : BEq a} → {a_2 : Hashable a} → Inhabited (Lean.Export.Alloc a)
    Equations
    • Lean.Export.instInhabitedAlloc = { default := { map := default, next := default } }
    Equations
    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.
    Equations
    • One or more equations did not get rendered due to their size.
    @[inline, reducible]
    abbrev Lean.ExportM (α : Type) :
    Equations
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        Instances For
          Equations
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              Equations
              Instances For
                Equations
                Instances For