Documentation

Lean.Util.PtrSet

structure Lean.Ptr (α : Type u) :
  • value : α
Instances For
    unsafe instance Lean.instHashablePtr {α : Type u_1} :
    Equations
    unsafe instance Lean.instBEqPtr {α : Type u_1} :
    Equations
    unsafe def Lean.PtrSet (α : Type) :

    Set of pointers. It is a low-level auxiliary datastructure used for traversing DAGs.

    Equations
    Instances For
      unsafe def Lean.mkPtrSet {α : Type} (capacity : optParam Nat 64) :
      Equations
      Instances For
        @[inline, reducible]
        unsafe abbrev Lean.PtrSet.insert {α : Type} (s : Lean.PtrSet α) (a : α) :
        Equations
        Instances For
          @[inline, reducible]
          unsafe abbrev Lean.PtrSet.contains {α : Type} (s : Lean.PtrSet α) (a : α) :
          Equations
          Instances For