src/HOL/Library/Multiset.thy
Mon, 09 Jun 2025 22:14:38 +0200 haftmann more qualified auxiliary operations
Thu, 29 May 2025 14:17:09 +0200 haftmann added lemma
Fri, 02 May 2025 17:24:43 +0200 haftmann executable sorted_list_of_multiset
Tue, 22 Apr 2025 15:41:34 +0200 Manuel Eberl removed possible problematic dependency in HOL-Library.Multiset
Tue, 22 Apr 2025 14:14:00 +0200 Manuel Eberl HOL-Library: multisets of a given size
Tue, 04 Mar 2025 16:58:46 +0100 desharna added attribute "simp" to filter_mset_eq_mempty_iff
Tue, 04 Mar 2025 16:38:21 +0100 desharna removed lemma size_multiset_sum_mset[simp]
Tue, 04 Mar 2025 16:37:14 +0100 desharna added lemma size_mset_sum_mset_conv[simp] (thanks to Manuel Eberl)
Tue, 04 Mar 2025 16:07:55 +0100 desharna added lemma filter_mset_eq_mempty_iff (thanks to Manuel Eberl)
Tue, 04 Mar 2025 15:19:08 +0100 desharna renamed lemma filter_image_mset to filter_mset_image_mset
Tue, 04 Mar 2025 13:10:47 +0100 desharna added lemma sum_mset_image_mset_mono_strong
Tue, 04 Mar 2025 13:10:31 +0100 desharna added lemmas filter_mset_mono_strong, filter_mset_sum_list, set_mset_sum_list[simp] (thanks to Manuel Eberl)
Fri, 06 Dec 2024 20:26:33 +0100 wenzelm clarified renaming of bounds, using Syntax_Trans.variant_bounds: avoid structures and fixed variables with syntax;
Mon, 04 Nov 2024 11:21:19 +0100 wenzelm tuned proofs;
Sun, 03 Nov 2024 22:29:07 +0100 wenzelm tuned proofs;
Fri, 01 Nov 2024 14:10:52 +0000 paulson Library material from Eberl's Parallel_Shear_Sort
Sat, 19 Oct 2024 22:57:43 +0200 wenzelm tuned proofs;
Sat, 19 Oct 2024 19:00:19 +0200 wenzelm more type information;
Fri, 18 Oct 2024 14:20:09 +0200 wenzelm more inner-syntax markup;
Wed, 09 Oct 2024 23:38:29 +0200 wenzelm more inner-syntax markup;
Tue, 01 Oct 2024 20:39:16 +0200 wenzelm drop somewhat pointless 'syntax_consts' declarations;
Mon, 30 Sep 2024 23:32:26 +0200 wenzelm clarified syntax: use outer block (with indent);
Mon, 30 Sep 2024 20:30:59 +0200 wenzelm clarified inner-syntax markup, notably for enumerations: prefer "notation=mixfix" over "entity" via 'syntax_consts' (see also 70076ba563d2);
Fri, 20 Sep 2024 19:51:08 +0200 wenzelm standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
Wed, 28 Aug 2024 22:54:45 +0200 wenzelm more specific "args" syntax, to support more markup for syntax consts;
Sun, 25 Aug 2024 21:10:01 +0200 wenzelm more markup for syntax consts;
Mon, 08 Jul 2024 10:14:22 +0200 desharna added lemma image_mset_diff_if_inj
Mon, 08 Jul 2024 10:08:07 +0200 desharna added lemma minus_add_mset_if_not_in_lhs[simp]
Tue, 11 Jun 2024 10:27:35 +0200 desharna tuned proof
Mon, 10 Jun 2024 21:32:24 +0200 desharna renamed lemmas
Mon, 10 Jun 2024 14:09:55 +0200 desharna renamed theorems
Sat, 08 Jun 2024 14:57:14 +0200 desharna renamed lemmas
Fri, 12 Apr 2024 09:58:32 +0100 paulson Tidying ugly proofs
Fri, 29 Mar 2024 19:28:59 +0100 Manuel Eberl moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Sat, 23 Mar 2024 18:55:38 +0100 desharna redefined wf as an abbreviation for "wf_on UNIV"
Wed, 06 Mar 2024 10:39:45 +0100 blanchet more multiset lemmas
Mon, 05 Feb 2024 10:06:34 +0100 desharna added lemmas Multiset.transp_on_multp and Multiset.trans_on_mult
Tue, 23 May 2023 21:43:36 +0200 wenzelm more uniform simproc_setup: avoid vacuous abstraction over morphism, which sometimes captures context values in its functional closure;
Mon, 08 May 2023 11:24:46 +0200 desharna added lemmas count_minus_inter_lt_count_minus_inter_iff and minus_inter_eq_minus_inter_iff
Wed, 12 Apr 2023 19:56:05 +0200 desharna added lemma multp_image_mset_image_msetI
Mon, 20 Mar 2023 18:33:56 +0100 desharna reordered assumption and tuned proof of Multiset.bex_least_element and Multiset.bex_greatest_element
Fri, 17 Mar 2023 13:56:54 +0100 desharna added lemma multp_repeat_mset_repeat_msetI
Mon, 23 Jan 2023 14:34:07 +0100 desharna added lemmas total_on_mult, total_mult, totalp_on_multp, and totalp_multp
Thu, 22 Dec 2022 21:55:51 +0100 desharna merged
Tue, 20 Dec 2022 09:34:37 +0100 desharna used transp_on in assumptions of lemmas Multiset.bex_(least|greatest)_element
Mon, 19 Dec 2022 16:00:49 +0100 desharna strengthened and renamed lemmas preorder.transp_(ge|gr|le|less)
Tue, 20 Dec 2022 18:20:19 +0100 blanchet added lifting_forget as suggested by Peter Lammich
Sun, 18 Dec 2022 14:03:43 +0100 desharna added predicates asym_on and asymp_on and redefined asym and asymp to be abbreviations
Tue, 06 Dec 2022 19:17:05 +0100 desharna Strengthened multiset lemmas w.r.t. irrefl and irreflp
Wed, 07 Dec 2022 10:11:58 +0100 desharna stated goals of some lemmas explicitely to prevent silent changes
Wed, 23 Nov 2022 09:57:59 +0100 desharna strengthened and renamed irreflp_greater[simp] and irreflp_less[simp]
Fri, 28 Oct 2022 15:39:35 +0200 desharna added lemmas multp_mono_strong and mult_mono_strong
Thu, 20 Oct 2022 14:43:29 +0200 desharna tuned proof
Sat, 15 Oct 2022 16:34:19 +0200 desharna added lemma wfP_subset_mset[simp]
Mon, 27 Jun 2022 15:54:18 +0200 traytel strict bounds for BNFs (by Jan van Brügge)
Tue, 21 Jun 2022 14:21:55 +0200 desharna added lemmas monotone{,_on}_multp_multp_image_mset
Mon, 13 Jun 2022 20:02:00 +0200 desharna added lemmas image_mset_eq_{image_mset_plus,plus,plus_image_mset}D, and multp_image_mset_image_msetD
Sat, 28 May 2022 10:45:45 +0200 desharna added lemmas Multiset.bex_{least,greatest}_element
Mon, 23 May 2022 10:13:08 +0200 desharna added lemma image_mset_filter_mset_swap
Fri, 20 May 2022 11:08:33 +0200 desharna added lemmas filter_mset_cong{0,}
less more (0) -300 -100 -60 tip