Documentation

Aesop.Index

structure Aesop.Index (α : Type) :
Instances For
    instance Aesop.instInhabitedIndex {a✝ : Type} :
    Equations
    def Aesop.Index.trace {α : Type} [ToString (Rule α)] (ri : Index α) (traceOpt : TraceOption) :
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      def Aesop.Index.merge {α : Type} (ri₁ ri₂ : Index α) :
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[specialize #[]]
        partial def Aesop.Index.add {α : Type} (r : Rule α) (imode : IndexingMode) (ri : Index α) :
        def Aesop.Index.unindex {α : Type} (ri : Index α) (p : Rule αBool) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[always_inline]
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def Aesop.Index.foldM {α : Type} {m : Type u_1 → Type u_1} {σ : Type u_1} [Monad m] (ri : Index α) (f : σRule αm σ) (init : σ) :
            m σ
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[inline]
              def Aesop.Index.fold {α : Type} {σ : Type u_1} (ri : Index α) (f : σRule ασ) (init : σ) :
              σ
              Equations
              Instances For
                @[specialize #[]]
                def Aesop.Index.applicableRules {α : Type} [Ord α] (ri : Index α) (goal : Lean.MVarId) (include? : Rule αBool) :
                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[inline]
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For