Mathlib Changelog
v3
Changelog
About
Github
Mathlib v3 is deprecated.
Go to Mathlib v4
Commit
2017-11-19 00:41
f9de1839
View on Github →
feat(data/multiset): working on multisets, fix rcases bug
Estimated changes
Modified
algebra/functions.lean
added
theorem
max_min_distrib_left
added
theorem
max_min_distrib_right
added
theorem
min_max_distrib_left
added
theorem
min_max_distrib_right
Modified
analysis/topology/uniform_space.lean
Modified
data/list/basic.lean
added
theorem
list.bag_inter_nil
added
theorem
list.bag_inter_sublist_left
added
theorem
list.cons_bag_inter_of_neg
added
theorem
list.cons_bag_inter_of_pos
added
theorem
list.length_bind
added
theorem
list.length_join
added
theorem
list.mem_bag_inter
added
theorem
list.mem_erase_of_ne
deleted
theorem
list.mem_erase_of_ne_of_mem
added
theorem
list.nil_bag_inter
added
theorem
list.nth_range'
added
theorem
list.nth_range
deleted
def
list.permutations_aux.F
deleted
def
list.permutations_aux.eqn_1
deleted
def
list.permutations_aux.eqn_2
added
def
list.permutations_aux.rec
modified
def
list.permutations_aux2
modified
def
list.permutations_aux
added
theorem
list.permutations_aux_cons
added
theorem
list.permutations_aux_nil
added
theorem
list.sum_const_nat
Modified
data/list/perm.lean
added
theorem
list.foldr_permutations_aux2
added
theorem
list.length_foldr_permutations_aux2'
added
theorem
list.length_foldr_permutations_aux2
added
theorem
list.length_permutations
added
theorem
list.length_permutations_aux2
added
theorem
list.length_permutations_aux
added
theorem
list.mem_foldr_permutations_aux2
added
theorem
list.mem_permutations
added
theorem
list.mem_permutations_aux2'
added
theorem
list.mem_permutations_aux2
added
theorem
list.mem_permutations_aux_of_perm
added
theorem
list.mem_permutations_of_perm_lemma
added
theorem
list.perm_bag_inter_left
added
theorem
list.perm_bag_inter_right
modified
theorem
list.perm_diff_right
added
theorem
list.perm_nil
added
theorem
list.perm_of_mem_permutations
added
theorem
list.perm_of_mem_permutations_aux
added
theorem
list.permutations_aux2_append
added
theorem
list.permutations_aux2_fst
added
theorem
list.permutations_aux2_snd_cons
added
theorem
list.permutations_aux2_snd_nil
Modified
data/multiset/basic.lean
added
theorem
multiset.add_bind
added
theorem
multiset.add_product
added
def
multiset.bind
added
theorem
multiset.coe_bind
modified
theorem
multiset.coe_eq_coe
modified
theorem
multiset.coe_foldl
modified
theorem
multiset.coe_foldr
added
theorem
multiset.coe_map
added
theorem
multiset.coe_prod
added
theorem
multiset.coe_product
added
theorem
multiset.cons_bind
added
theorem
multiset.cons_inter_of_neg
added
theorem
multiset.cons_inter_of_pos
added
theorem
multiset.cons_product
added
theorem
multiset.foldl_add
added
theorem
multiset.foldl_cons
added
theorem
multiset.foldl_zero
added
theorem
multiset.foldr_add
added
theorem
multiset.foldr_cons
added
theorem
multiset.foldr_zero
added
def
multiset.inter
modified
theorem
multiset.inter_comm
added
theorem
multiset.inter_le_left
added
theorem
multiset.inter_le_right
added
theorem
multiset.inter_zero
added
theorem
multiset.join_add
added
theorem
multiset.join_cons
added
theorem
multiset.join_zero
added
theorem
multiset.le_inter
modified
theorem
multiset.le_union_left
modified
theorem
multiset.le_union_right
added
theorem
multiset.map_add
added
theorem
multiset.map_cons
added
theorem
multiset.map_map
added
theorem
multiset.map_zero
added
theorem
multiset.mem_erase_of_ne
modified
theorem
multiset.mem_erase_of_ne_of_mem
added
theorem
multiset.prod_add
added
theorem
multiset.prod_cons
added
theorem
multiset.prod_eq_foldl
deleted
def
multiset.prod_eq_foldl
added
theorem
multiset.prod_eq_foldr
deleted
def
multiset.prod_eq_foldr
added
theorem
multiset.prod_zero
added
def
multiset.product
added
theorem
multiset.product_add
deleted
def
multiset.sum
modified
theorem
multiset.union_comm
added
theorem
multiset.zero_bind
added
theorem
multiset.zero_inter
added
theorem
multiset.zero_product
Modified
data/quot.lean
deleted
theorem
quot_mk_image_univ_eq
added
theorem
quotient.eq
Modified
data/set/basic.lean
added
theorem
set.quot_mk_image_univ_eq
Modified
order/boolean_algebra.lean
Modified
order/lattice.lean
added
theorem
lattice.sup_le_sup_left
added
theorem
lattice.sup_le_sup_right
Modified
tactic/rcases.lean
Modified
theories/set_theory.lean
modified
inductive
pSet.definable