Documentation

Lean.Meta.Tactic.Simp.BuiltinSimprocs.Char

@[inline]
def Char.reduceUnary {α : Type u_1} [Lean.ToExpr α] (declName : Lake.Name) (op : Charα) (arity : optParam Nat 1) (e : Lean.Expr) :
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[inline]
    def Char.reduceBinPred (declName : Lake.Name) (arity : Nat) (op : CharCharBool) (e : Lean.Expr) :
    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
        Equations
        Instances For
          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
                  Instances For

                    Return .done for Char values. We don't want to unfold in the symbolic evaluator. In regular simp, we want to prevent the nested raw literal from being converted into a OfNat.ofNat application. TODO: cleanup

                    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