Documentation

Init.Data.AC

Instances For
    structure Lean.Data.AC.Variable {α : Sort u} (op : ααα) :
    Instances For
      structure Lean.Data.AC.Context (α : Sort u) :
      Instances For
        class Lean.Data.AC.ContextInformation (α : Sort u) :
        Sort (max 1 u)
        Instances
          class Lean.Data.AC.EvalInformation (α : Sort u) (β : Sort v) :
          Sort (max (max 1 u) v)
          • arbitrary : αβ
          • evalOp : αβββ
          • evalVar : αNatβ
          Instances
            Equations
            • ctx.var idx = ctx.vars.getD idx { value := ctx.arbitrary, neutral := none }
            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.
              Equations
              Instances For
                Equations
                Instances For
                  Equations
                  Instances For
                    Equations
                    Instances For
                      Equations
                      Instances For
                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          noncomputable def Lean.Data.AC.List.two_step_induction {motive : List NatSort u} (l : List Nat) (empty : motive []) (single : (a : Nat) → motive [a]) (step : (a b : Nat) → (l : List Nat) → motive (b :: l)motive (a :: b :: l)) :
                          motive l
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            theorem Lean.Data.AC.Context.evalList_append {α : Sort u_1} (ctx : Lean.Data.AC.Context α) (l r : List Nat) (h₁ : l []) (h₂ : r []) :
                            Lean.Data.AC.evalList α ctx (l.append r) = ctx.op (Lean.Data.AC.evalList α ctx l) (Lean.Data.AC.evalList α ctx r)