Documentation

Aesop.Search.SearchM

Equations
Instances For
    Instances For
      Equations
      • Aesop.SearchM.instInhabitedState = { default := { iteration := default, queue := default, maxRuleApplicationDepthReached := default } }
      Equations
      • Aesop.SearchM.instMonad = Monad.mk
      Equations
      Equations
      • Aesop.SearchM.instInhabited = { default := failure }
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • Aesop.SearchM.instMonadReaderContext = { read := MonadReaderOf.read }
      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.
      Instances For
        def Aesop.SearchM.run {Q : Type} [Aesop.Queue Q] {α : Type} (ruleSet : Aesop.LocalRuleSet) (options : Aesop.Options') (simpConfig : Lean.Meta.Simp.Config) (simpConfigStx? : Option Lean.Term) (goal : Lean.MVarId) (stats : Aesop.Stats) (x : Aesop.SearchM Q α) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          Equations
          Instances For
            Equations
            Instances For
              Equations
              Instances For
                Equations
                • Aesop.getIteration = do let __do_liftget pure __do_lift.iteration
                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
                        • Aesop.setMaxRuleApplicationDepthReached = modify fun (s : Aesop.SearchM.State Q) => { iteration := s.iteration, queue := s.queue, maxRuleApplicationDepthReached := true }
                        Instances For
                          Equations
                          • Aesop.wasMaxRuleApplicationDepthReached = do let __do_liftget pure __do_lift.maxRuleApplicationDepthReached
                          Instances For