Documentation

Std.Tactic.BVDecide.LRAT.Internal.Clause

An inductive datatype used specifically for the output of the reduce function. The intended meaning of each constructor is explained in the docstring of the reduce function.

Instances For

    Typeclass for clauses. An instance [Clause α β] indicates that β is the type of a clause with variables of type α.

    Instances
      theorem Std.Tactic.BVDecide.LRAT.Internal.Clause.ofArray_eq {α : outParam (Type u)} {β : Type v} [self : Std.Tactic.BVDecide.LRAT.Internal.Clause α β] (arr : Array (Std.Sat.Literal α)) :
      (∀ (i j : Fin arr.size), i jarr[i] arr[j])∀ (c : β), Std.Tactic.BVDecide.LRAT.Internal.Clause.ofArray arr = some cStd.Tactic.BVDecide.LRAT.Internal.Clause.toList c = arr.toList
      Equations
      • Std.Tactic.BVDecide.LRAT.Internal.Clause.instEntailsLiteral = { eval := fun (p : αBool) (l : Std.Sat.Literal α) => p l.fst = l.snd }
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        Equations
        • Std.Tactic.BVDecide.LRAT.Internal.Clause.instInhabited = { default := Std.Tactic.BVDecide.LRAT.Internal.Clause.empty }

        The DefaultClause structure is primarily a list of literals. The additional field nodupkey is included to ensure that not_tautology is provable (which is needed to prove sat_of_insertRup and sat_of_insertRat in LRAT.Formula.Internal.RupAddSound and LRAT.Formula.Internal.RatAddSound). The additional field nodup is included to ensure that delete can be implemented by simply calling erase on the clause field. Without nodup, it would be necessary to iterate through the entire clause field and erase all instances of the literal to be deleted, since there would potentially be more than one.

        In principle, one could combine nodupkey and nodup to instead have one additional field that stipulates that ∀ l1 : PosFin numVarsSucc, ∀ l2 : PosFin numVarsSucc, l1.1 ≠ l2.1. This would work just as well, and the only reason that DefaultClause is structured in this manner is that the nodup field was only included in a later stage of the verification process when it became clear that it was needed.

        Instances For
          Equations
          • Std.Tactic.BVDecide.LRAT.Internal.instBEqDefaultClause = { beq := Std.Tactic.BVDecide.LRAT.Internal.beqDefaultClause✝ }
          Equations
          • One or more equations did not get rendered due to their size.
          Equations
          • Std.Tactic.BVDecide.LRAT.Internal.DefaultClause.empty = { clause := [], nodupkey := , nodup := }
          Instances For
            theorem Std.Tactic.BVDecide.LRAT.Internal.DefaultClause.empty_eq {n : Nat} :
            Std.Tactic.BVDecide.LRAT.Internal.DefaultClause.empty.toList = []

            Attempts to add the literal (idx, b) to clause c. Returns none if doing so would make c a tautology.

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

              The reduce function takes in a clause c and takes in an array of assignments and attempts to eliminate every literal in the clause that is not compatible with the assignments argument.

              • If reduce returns encounteredBoth, then this means that the assignments array has a both Assignment and is therefore fundamentally unsatisfiable.
              • If reduce returns reducedToEmpty, then this means that every literal in c is incompatible with assignments. In other words, this means that the conjunction of assignments and c is unsatisfiable.
              • If reduce returns reducedToUnit l, then this means that every literal in c is incompatible with assignments except for l. In other words, this means that the conjunction of assignments and c entail l.
              • If reduce returns reducedToNonunit, then this means that there are multiple literals in c that are compatible with assignments. This is a failure condition for confirmRupHint (in LRAT.Formula.Implementation.lean) which calls reduce.
              Equations
              Instances For