Mathlib Changelog
v3
Changelog
About
Github
Mathlib v3 is deprecated.
Go to Mathlib v4
Commit
2020-02-28 18:23
19a9bdc2
View on Github →
fix(tactic/omega): reify nonconstant ints and nats (
#1748
)
Estimated changes
Modified
archive/imo1988_q6.lean
Modified
docs/tactics.md
Modified
scripts/nolints.txt
Modified
src/tactic/omega/clause.lean
Modified
src/tactic/omega/coeffs.lean
Modified
src/tactic/omega/eq_elim.lean
Modified
src/tactic/omega/find_ees.lean
Modified
src/tactic/omega/find_scalars.lean
Modified
src/tactic/omega/int/dnf.lean
modified
theorem
omega.int.clauses_sat_dnf_core
modified
def
omega.int.dnf
modified
def
omega.int.dnf_core
modified
theorem
omega.int.implies_neg_elim
modified
def
omega.int.is_nnf
modified
theorem
omega.int.is_nnf_nnf
modified
theorem
omega.int.is_nnf_push_neg
modified
def
omega.int.neg_elim
modified
def
omega.int.neg_free
modified
theorem
omega.int.neg_free_neg_elim
modified
def
omega.int.nnf
modified
theorem
omega.int.nnf_equiv
modified
def
omega.int.push_neg
modified
theorem
omega.int.unsat_of_clauses_unsat
Modified
src/tactic/omega/int/form.lean
deleted
def
omega.int.form.equiv
deleted
def
omega.int.form.fresh_index
deleted
def
omega.int.form.holds
deleted
def
omega.int.form.implies
deleted
def
omega.int.form.repr
deleted
def
omega.int.form.sat
deleted
theorem
omega.int.form.sat_of_implies_of_sat
deleted
theorem
omega.int.form.sat_or
deleted
def
omega.int.form.unsat
deleted
def
omega.int.form.valid
deleted
inductive
omega.int.form
added
def
omega.int.preform.equiv
added
def
omega.int.preform.fresh_index
added
def
omega.int.preform.holds
added
def
omega.int.preform.implies
added
def
omega.int.preform.repr
added
def
omega.int.preform.sat
added
theorem
omega.int.preform.sat_of_implies_of_sat
added
theorem
omega.int.preform.sat_or
added
def
omega.int.preform.unsat
added
def
omega.int.preform.valid
added
inductive
omega.int.preform
modified
def
omega.int.univ_close
modified
theorem
omega.int.univ_close_of_valid
modified
theorem
omega.int.valid_of_unsat_not
Modified
src/tactic/omega/int/main.lean
modified
theorem
omega.int.univ_close_of_unsat_clausify
Modified
src/tactic/omega/int/preterm.lean
Modified
src/tactic/omega/lin_comb.lean
Modified
src/tactic/omega/main.lean
Modified
src/tactic/omega/misc.lean
Modified
src/tactic/omega/nat/dnf.lean
modified
def
omega.nat.dnf
modified
def
omega.nat.dnf_core
modified
theorem
omega.nat.exists_clause_holds
modified
theorem
omega.nat.exists_clause_sat
modified
theorem
omega.nat.unsat_of_unsat_dnf
Modified
src/tactic/omega/nat/form.lean
deleted
def
omega.nat.form.equiv
deleted
def
omega.nat.form.fresh_index
deleted
def
omega.nat.form.holds
deleted
theorem
omega.nat.form.holds_constant
deleted
def
omega.nat.form.implies
deleted
def
omega.nat.form.neg_free
deleted
def
omega.nat.form.repr
deleted
def
omega.nat.form.sat
deleted
theorem
omega.nat.form.sat_of_implies_of_sat
deleted
theorem
omega.nat.form.sat_or
deleted
def
omega.nat.form.sub_free
deleted
def
omega.nat.form.unsat
deleted
def
omega.nat.form.valid
deleted
inductive
omega.nat.form
added
def
omega.nat.preform.equiv
added
def
omega.nat.preform.fresh_index
added
def
omega.nat.preform.holds
added
theorem
omega.nat.preform.holds_constant
added
def
omega.nat.preform.implies
added
def
omega.nat.preform.neg_free
added
def
omega.nat.preform.repr
added
def
omega.nat.preform.sat
added
theorem
omega.nat.preform.sat_of_implies_of_sat
added
theorem
omega.nat.preform.sat_or
added
def
omega.nat.preform.sub_free
added
def
omega.nat.preform.unsat
added
def
omega.nat.preform.valid
added
inductive
omega.nat.preform
modified
def
omega.nat.univ_close
modified
theorem
omega.nat.univ_close_of_valid
modified
theorem
omega.nat.valid_of_unsat_not
Modified
src/tactic/omega/nat/main.lean
modified
theorem
omega.nat.univ_close_of_unsat_neg_elim_not
Modified
src/tactic/omega/nat/neg_elim.lean
modified
theorem
omega.nat.implies_neg_elim
modified
theorem
omega.nat.implies_neg_elim_core
modified
def
omega.nat.is_nnf
modified
theorem
omega.nat.is_nnf_nnf
modified
theorem
omega.nat.is_nnf_push_neg
modified
def
omega.nat.neg_elim
modified
def
omega.nat.neg_elim_core
modified
theorem
omega.nat.neg_free_neg_elim
modified
def
omega.nat.nnf
modified
theorem
omega.nat.nnf_equiv
modified
def
omega.nat.push_neg
Modified
src/tactic/omega/nat/preterm.lean
Modified
src/tactic/omega/nat/sub_elim.lean
deleted
def
omega.nat.form.sub_subst
deleted
def
omega.nat.form.sub_terms
modified
def
omega.nat.is_diff
added
def
omega.nat.preform.sub_subst
added
def
omega.nat.preform.sub_terms
modified
theorem
omega.nat.sat_sub_elim
modified
def
omega.nat.sub_elim
modified
def
omega.nat.sub_elim_core
modified
def
omega.nat.sub_fresh_index
modified
theorem
omega.nat.unsat_of_unsat_sub_elim
Modified
src/tactic/omega/prove_unsats.lean
Modified
src/tactic/omega/term.lean
Modified
test/omega.lean