Documentation

Aesop.Search.SearchM

Instances For
    Equations
    Instances For
      Instances For
        structure Aesop.SearchM.State (Q : Type) [Queue Q] :
        • iteration : Iteration
        • queue : Q
        • maxRuleApplicationDepthReached : Bool
        Instances For
          def Aesop.SearchM.instInhabitedState.default {a✝ : Type} [Inhabited a✝] {a✝¹ : Queue a✝} :
          State a✝
          Equations
          Instances For
            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.
            def Aesop.SearchM.run' {Q : Type} [Queue Q] {α : Type} (ctx : Context) (σ : State Q) (tree : Tree) (x : SearchM Q α) :
            Equations
            Instances For
              def Aesop.SearchM.run {Q : Type} [Queue Q] {α : Type} (ruleSet : LocalRuleSet) (options : Options') (simpConfig : Lean.Meta.Simp.Config) (simpConfigStx? : Option Lean.Term) (goal : Lean.MVarId) (x : SearchM Q α) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                Equations
                Instances For
                  def Aesop.modifyTree {Q : Type} [Queue Q] :
                  (TreeTree)SearchM Q Unit
                  Equations
                  Instances For
                    Equations
                    Instances For
                      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.
                        Instances For
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            Equations
                            Instances For