Documentation

Aesop.Script.ScriptM

@[reducible, inline]
abbrev Aesop.ScriptT (m : TypeType) (α : Type) :
Equations
Instances For
    def Aesop.ScriptT.run {m : TypeType} {α : Type} [Monad m] [MonadLiftT (ST IO.RealWorld) m] (x : ScriptT m α) :
    Equations
    Instances For
      @[reducible, inline]
      abbrev Aesop.ScriptM (α : Type) :
      Equations
      Instances For
        Equations
        Instances For
          def Aesop.withScriptStep {α : Type} (preGoal : Lean.MVarId) (postGoals : αArray Lean.MVarId) (success : αBool) (tacticBuilder : αScript.TacticBuilder) (x : Lean.MetaM α) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def Aesop.withOptScriptStep {α : Type} (preGoal : Lean.MVarId) (postGoals : αArray Lean.MVarId) (tacticBuilder : αScript.TacticBuilder) (x : Lean.MetaM (Option α)) :
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For