Mathlib Changelog
v3
Changelog
About
Github
Mathlib v3 is deprecated.
Go to Mathlib v4
Commit
2019-04-18 22:33
c1aff1b5
View on Github →
style(tactic/omega): whitespace and minor tweaks missed the PR review cycle
Estimated changes
Modified
src/data/list/basic.lean
modified
theorem
list.func.add_nil
modified
theorem
list.func.equiv_of_eq
modified
theorem
list.func.equiv_symm
modified
theorem
list.func.forall_val_of_forall_mem
modified
theorem
list.func.get_map'
modified
theorem
list.func.get_map
modified
theorem
list.func.get_neg
modified
theorem
list.func.get_nil
modified
theorem
list.func.get_pointwise
modified
theorem
list.func.get_sub
modified
theorem
list.func.length_add
modified
theorem
list.func.length_neg
modified
theorem
list.func.length_pointwise
modified
theorem
list.func.length_sub
modified
theorem
list.func.nil_add
modified
theorem
list.func.nil_pointwise
modified
theorem
list.func.nil_sub
modified
theorem
list.func.pointwise_nil
modified
theorem
list.func.sub_nil
Modified
src/tactic/omega/coeffs.lean
modified
theorem
omega.coeffs.val_between_map_div
modified
theorem
omega.coeffs.val_except_update_set
Modified
src/tactic/omega/eq_elim.lean
Modified
src/tactic/omega/find_ees.lean
added
structure
omega.ee_state
Modified
src/tactic/omega/int/dnf.lean
Modified
src/tactic/omega/int/form.lean
Modified
src/tactic/omega/int/main.lean
Modified
src/tactic/omega/int/preterm.lean
Modified
src/tactic/omega/misc.lean
Modified
src/tactic/omega/nat/dnf.lean
Modified
src/tactic/omega/nat/form.lean
modified
def
omega.nat.form.equiv
modified
def
omega.nat.form.fresh_index
modified
def
omega.nat.form.holds
modified
def
omega.nat.form.implies
modified
def
omega.nat.form.neg_free
modified
def
omega.nat.form.repr
modified
def
omega.nat.form.sat
modified
def
omega.nat.form.sub_free
modified
def
omega.nat.form.valid
modified
inductive
omega.nat.form
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
src/tactic/omega/nat/neg_elim.lean
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.le_and_le_iff_eq
modified
def
omega.nat.neg_elim_core
modified
theorem
omega.nat.neg_free_neg_elim
modified
theorem
omega.nat.neg_free_neg_elim_core
modified
def
omega.nat.nnf
modified
def
omega.nat.push_neg
modified
theorem
omega.nat.push_neg_equiv
Modified
src/tactic/omega/nat/preterm.lean
modified
def
omega.nat.canonize
modified
def
omega.nat.preterm.fresh_index
modified
def
omega.nat.preterm.repr
modified
def
omega.nat.preterm.sub_free
modified
def
omega.nat.preterm.val
modified
theorem
omega.nat.preterm.val_add
modified
theorem
omega.nat.preterm.val_sub
modified
theorem
omega.nat.val_canonize
Modified
src/tactic/omega/nat/sub_elim.lean
Modified
src/tactic/omega/term.lean
added
def
omega.term.to_string
Modified
test/omega.lean