Commit 2023-01-16 08:13 5a1c5bb7

View on Github →

feat: port Data.Finset.Basic (#1555)

Estimated changes

added theorem Finset.Insert.comm
added theorem Finset.Nonempty.bex
added theorem Finset.Nonempty.mono
added theorem Finset.Subset.antisymm
added theorem Finset.Subset.refl
added theorem Finset.Subset.trans
added theorem Finset.Superset.trans
added def Finset.attach
added theorem Finset.attach_empty
added theorem Finset.attach_val
added theorem Finset.bind_toFinset
added theorem Finset.bot_eq_empty
added theorem Finset.bunionᵢ_congr
added theorem Finset.bunionᵢ_empty
added theorem Finset.bunionᵢ_inter
added theorem Finset.bunionᵢ_mono
added theorem Finset.bunionᵢ_val
added def Finset.choose
added def Finset.chooseX
added theorem Finset.choose_mem
added theorem Finset.choose_property
added theorem Finset.choose_spec
added def Finset.coeEmb
added theorem Finset.coe_bunionᵢ
added theorem Finset.coe_coeEmb
added theorem Finset.coe_cons
added theorem Finset.coe_empty
added theorem Finset.coe_eq_empty
added theorem Finset.coe_eq_pair
added theorem Finset.coe_erase
added theorem Finset.coe_filter
added theorem Finset.coe_inj
added theorem Finset.coe_injective
added theorem Finset.coe_insert
added theorem Finset.coe_inter
added theorem Finset.coe_mem
added theorem Finset.coe_nonempty
added theorem Finset.coe_pair
added theorem Finset.coe_range
added theorem Finset.coe_sdiff
added theorem Finset.coe_singleton
added theorem Finset.coe_sort_coe
added theorem Finset.coe_ssubset
added theorem Finset.coe_subset
added theorem Finset.coe_symmDiff
added theorem Finset.coe_toList
added theorem Finset.coe_union
added def Finset.cons
added theorem Finset.cons_eq_insert
added theorem Finset.cons_induction
added theorem Finset.cons_subset
added theorem Finset.cons_val
added theorem Finset.dedup_eq_self
added def Finset.disjUnion
added theorem Finset.disjUnion_comm
added theorem Finset.disjUnion_empty
added theorem Finset.disjoint_coe
added theorem Finset.disjoint_filter
added theorem Finset.disjoint_iff_ne
added theorem Finset.disjoint_left
added theorem Finset.disjoint_right
added theorem Finset.disjoint_sdiff
added theorem Finset.disjoint_val
added theorem Finset.empty_disjUnion
added theorem Finset.empty_inter
added theorem Finset.empty_sdiff
added theorem Finset.empty_ssubset
added theorem Finset.empty_subset
added theorem Finset.empty_toList
added theorem Finset.empty_union
added theorem Finset.empty_val
added theorem Finset.eq_of_veq
added def Finset.erase
added theorem Finset.erase_bunionᵢ
added theorem Finset.erase_cons
added theorem Finset.erase_empty
added theorem Finset.erase_eq_self
added theorem Finset.erase_idem
added theorem Finset.erase_inj
added theorem Finset.erase_injOn'
added theorem Finset.erase_injOn
added theorem Finset.erase_insert
added theorem Finset.erase_ne_self
added theorem Finset.erase_singleton
added theorem Finset.erase_ssubset
added theorem Finset.erase_subset
added theorem Finset.erase_val
added theorem Finset.ext
added theorem Finset.ext_iff
added def Finset.filter
added theorem Finset.filter_and
added theorem Finset.filter_congr
added theorem Finset.filter_cons
added theorem Finset.filter_empty
added theorem Finset.filter_eq'
added theorem Finset.filter_eq
added theorem Finset.filter_eq_self
added theorem Finset.filter_erase
added theorem Finset.filter_false
added theorem Finset.filter_filter
added theorem Finset.filter_insert
added theorem Finset.filter_inter
added theorem Finset.filter_ne'
added theorem Finset.filter_ne
added theorem Finset.filter_not
added theorem Finset.filter_or
added theorem Finset.filter_ssubset
added theorem Finset.filter_subset
added theorem Finset.filter_true
added theorem Finset.filter_union
added theorem Finset.filter_val
added theorem Finset.forall_mem_cons
added theorem Finset.induction_on'
added theorem Finset.inf_eq_inter
added theorem Finset.insert_def
added theorem Finset.insert_eq
added theorem Finset.insert_eq_self
added theorem Finset.insert_erase
added theorem Finset.insert_idem
added theorem Finset.insert_inj
added theorem Finset.insert_inj_on
added theorem Finset.insert_ne_empty
added theorem Finset.insert_ne_self
added theorem Finset.insert_nonempty
added theorem Finset.insert_subset
added theorem Finset.insert_union
added theorem Finset.insert_val'
added theorem Finset.insert_val
added theorem Finset.inter_assoc
added theorem Finset.inter_bunionᵢ
added theorem Finset.inter_comm
added theorem Finset.inter_empty
added theorem Finset.inter_filter
added theorem Finset.inter_left_comm
added theorem Finset.inter_left_idem
added theorem Finset.inter_sdiff
added theorem Finset.inter_self
added theorem Finset.inter_val
added theorem Finset.inter_val_nd
added theorem Finset.le_eq_subset
added theorem Finset.le_iff_subset
added theorem Finset.lt_eq_subset
added theorem Finset.lt_iff_ssubset
added theorem Finset.mem_attach
added theorem Finset.mem_bunionᵢ
added theorem Finset.mem_coe
added theorem Finset.mem_cons
added theorem Finset.mem_cons_self
modified theorem Finset.mem_def
added theorem Finset.mem_disjUnion
added theorem Finset.mem_erase
added theorem Finset.mem_filter
added theorem Finset.mem_insert
added theorem Finset.mem_insert_coe
added theorem Finset.mem_insert_self
added theorem Finset.mem_inter
added theorem Finset.mem_mk
added theorem Finset.mem_of_subset
added theorem Finset.mem_range
added theorem Finset.mem_range_le
added theorem Finset.mem_sdiff
added theorem Finset.mem_singleton
added theorem Finset.mem_symmDiff
added theorem Finset.mem_toList
added theorem Finset.mem_union
added theorem Finset.mem_union_left
added theorem Finset.mem_union_right
added theorem Finset.mem_val
added theorem Finset.mk_coe
added theorem Finset.mk_cons
added theorem Finset.mk_zero
added theorem Finset.ne_empty_of_mem
added theorem Finset.ne_of_mem_erase
added theorem Finset.nodup_toList
added theorem Finset.nonempty_cons
added theorem Finset.nonempty_mk
added theorem Finset.not_mem_empty
added theorem Finset.not_mem_erase
added theorem Finset.not_mem_mono
added theorem Finset.not_mem_union
added theorem Finset.not_subset
added theorem Finset.pair_comm
added theorem Finset.pairwise_cons'
added theorem Finset.pairwise_cons
added def Finset.piecewise
added theorem Finset.piecewise_cases
added theorem Finset.piecewise_coe
added theorem Finset.piecewise_congr
added theorem Finset.piecewise_empty
added def Finset.range
added theorem Finset.range_add_one
added theorem Finset.range_filter_eq
added theorem Finset.range_mono
added theorem Finset.range_one
added theorem Finset.range_subset
added theorem Finset.range_succ
added theorem Finset.range_val
added theorem Finset.range_zero
added theorem Finset.sdiff_disjoint
added theorem Finset.sdiff_empty
added theorem Finset.sdiff_eq_filter
added theorem Finset.sdiff_eq_self
added theorem Finset.sdiff_erase
added theorem Finset.sdiff_idem
added theorem Finset.sdiff_insert
added theorem Finset.sdiff_nonempty
added theorem Finset.sdiff_self
added theorem Finset.sdiff_ssubset
added theorem Finset.sdiff_subset
added theorem Finset.sdiff_val
added theorem Finset.setOf_mem
added theorem Finset.singleton_inj
added theorem Finset.singleton_val
added theorem Finset.ssubset_cons
added theorem Finset.ssubset_def
added theorem Finset.ssubset_iff
added theorem Finset.ssubset_insert
added theorem Finset.subset_cons
added theorem Finset.subset_def
added theorem Finset.subset_empty
added theorem Finset.subset_erase
added theorem Finset.subset_iff
added theorem Finset.subset_insert
added theorem Finset.subset_inter
added theorem Finset.subset_sdiff
added theorem Finset.sup_eq_union
added theorem Finset.toList_cons
added theorem Finset.toList_empty
added theorem Finset.toList_eq_nil
added theorem Finset.toList_insert
added theorem Finset.toList_toFinset
added def Finset.toSet
added theorem Finset.union_assoc
added theorem Finset.union_comm
added theorem Finset.union_empty
added theorem Finset.union_insert
added theorem Finset.union_left_comm
added theorem Finset.union_left_idem
added theorem Finset.union_self
added theorem Finset.union_subset
added theorem Finset.union_val
added theorem Finset.union_val_nd
added theorem Finset.val_eq_zero
added theorem Finset.val_inj
added theorem Finset.val_injective
added theorem Finset.val_le_iff
added theorem Finset.val_lt_iff
added theorem Finset.val_toFinset
added theorem List.coe_toFinset
added theorem List.mem_toFinset
added theorem List.toFinset.ext
added theorem List.toFinset.ext_iff
added def List.toFinset
added theorem List.toFinset_append
added theorem List.toFinset_coe
added theorem List.toFinset_cons
added theorem List.toFinset_eq
added theorem List.toFinset_inter
added theorem List.toFinset_nil
added theorem List.toFinset_reverse
added theorem List.toFinset_surj_on
added theorem List.toFinset_union
added theorem List.toFinset_val
added theorem Multiset.mem_toFinset
added theorem Multiset.toFinset_add
added theorem Multiset.toFinset_cons
added theorem Multiset.toFinset_eq
added theorem Multiset.toFinset_val
added theorem Multiset.toFinset_zero
added theorem coe_notMemRangeEquiv
added def notMemRangeEquiv