Documentation

Lean.Meta.Tactic.AC.Main

@[reducible, inline]
Equations
Instances For
    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
      • 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
          Instances For
            @[match_pattern]
            def Lean.Meta.AC.bin (op l r : Expr) :
            Equations
            Instances For
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                In order to prevent the kernel trying to reduce the atoms of the expression, we abstract the proof over them. But ac_rfl proofs are not completely abstract in the value of the atoms – it recognizes neutral elements. So we have to abstract over these proofs as well.

                Equations
                Instances For
                  @[irreducible]
                  def Lean.Meta.AC.abstractAtoms.go (preContext : PreContext) (atoms : Array Expr) (k : Array (Expr × Option Expr)MetaM Expr) (α : Expr) (u : Level) (i : Nat) (acc : Array (Expr × Option Expr)) (vars args : Array Expr) :
                  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
                          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
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For

                                  Implementation of the ac_nf tactic when operating on the main goal.

                                  Equations
                                  Instances For

                                    Implementation of the ac_nf tactic when operating on a hypothesis.

                                    Equations
                                    Instances For
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For