src/HOL/List.thy
Tue, 28 Jan 2025 21:42:04 +0100 nipkow extracted the ^^ subtheory for modularity reasons
Mon, 20 Jan 2025 22:19:54 +0100 nipkow introduced/overloaded power operator ^^ lists
Mon, 23 Dec 2024 19:38:16 +0100 Lukas Bartl Rename "suggest_of" to "instantiate"
Wed, 08 Jan 2025 05:37:40 +0100 nipkow added lemmas
Thu, 02 Jan 2025 08:37:55 +0100 haftmann refined syntax for code_reserved
Sun, 15 Dec 2024 14:59:57 +0100 wenzelm more syntax bundles, e.g. to explore terms without notation;
Fri, 01 Nov 2024 14:10:52 +0000 paulson Library material from Eberl's Parallel_Shear_Sort
Tue, 29 Oct 2024 10:26:06 +0100 nipkow more attribute tuning
Tue, 29 Oct 2024 07:41:52 +0100 nipkow tuned attributes
Mon, 28 Oct 2024 18:48:14 +0100 nipkow added lemmas
Fri, 18 Oct 2024 14:20:09 +0200 wenzelm more inner-syntax markup;
Tue, 08 Oct 2024 17:26:31 +0200 wenzelm clarified bundles for list syntax;
Tue, 08 Oct 2024 12:10:35 +0200 wenzelm more inner-syntax markup;
Sat, 05 Oct 2024 14:58:36 +0200 wenzelm first-class support for "unbundle no foobar_syntax" -- avoid redundant "bundle no_foobar_syntax" definitions;
Tue, 01 Oct 2024 21:35:31 +0200 wenzelm more robust 'no_syntax' via bundles;
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);
Mon, 30 Sep 2024 13:00:42 +0200 wenzelm less markup: prefer "notatation" over "entity";
Mon, 23 Sep 2024 21:09:23 +0200 wenzelm more inner syntax markup: HOL;
Mon, 23 Sep 2024 13:32:38 +0200 wenzelm standardize mixfix annotations via "isabelle update -u mixfix_cartouches -l Pure HOL" --- 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 15:02:19 +0200 wenzelm more markup for syntax consts;
Sat, 24 Aug 2024 23:44:05 +0100 paulson Some tidying
Sun, 04 Aug 2024 17:39:47 +0200 wenzelm tuned: more explicit dest_Const_name and dest_Const_type;
Sun, 04 Aug 2024 13:24:54 +0200 wenzelm tuned: more explicit dest_Type_name and dest_Type_args;
Fri, 02 Aug 2024 18:25:18 +0200 nipkow got rid of references to system-generated names
Thu, 27 Jun 2024 11:59:12 +0200 Fabian Huch tuned comment;
Mon, 10 Jun 2024 08:25:55 +0200 desharna renamed theorems
Sat, 23 Mar 2024 18:55:38 +0100 desharna redefined wf as an abbreviation for "wf_on UNIV"
Tue, 13 Feb 2024 17:18:50 +0000 paulson A few lemmas brought in from AFP entries
Wed, 10 Jan 2024 15:30:13 +0100 nipkow added and removed lemmas
Thu, 26 Oct 2023 20:41:42 +0200 nipkow added lemma
Thu, 19 Oct 2023 21:38:09 +0200 wenzelm tuned signature;
Thu, 19 Oct 2023 17:06:39 +0200 wenzelm clarified signature;
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;
Wed, 01 Mar 2023 21:05:09 +0000 paulson A little bit more tidying up
Mon, 20 Feb 2023 13:55:58 +0100 nipkow Backed out changeset bafdc56654cf
Mon, 13 Feb 2023 16:07:41 +0100 nipkow move map_of to List
Mon, 19 Dec 2022 16:00:49 +0100 desharna strengthened and renamed lemmas preorder.transp_(ge|gr|le|less)
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, 08 Nov 2022 08:41:29 +0100 nipkow retain derived lemma for better findability
Mon, 07 Nov 2022 22:16:37 +0100 nipkow generalized sorted_sort_id to sort_key_id_if_sorted
Wed, 26 Oct 2022 17:22:12 +0100 paulson A couple of new theorems. Also additional coercions to the complex numbers
Fri, 14 Oct 2022 10:35:07 +0200 nipkow more List lemmas (partly by Jeremy Sylvestre)
Wed, 22 Jun 2022 08:15:10 +0000 haftmann Executable lexords.
Wed, 22 Jun 2022 08:15:09 +0000 haftmann Less warnings.
Mon, 30 May 2022 20:58:45 +0200 nipkow Added lemmas
Wed, 04 May 2022 07:20:20 +0200 nipkow added lemma
Mon, 07 Mar 2022 15:28:53 +0100 nipkow more count_list lemmas
Sun, 06 Mar 2022 22:13:18 +0100 nipkow added count_list lemmas
Wed, 29 Dec 2021 08:07:51 +0100 nipkow added lemma
Wed, 17 Nov 2021 16:13:00 +0100 nipkow added lemmas
Wed, 10 Nov 2021 08:36:50 +0100 nipkow added lemma
Tue, 09 Nov 2021 16:17:13 +0100 nipkow tuned attributes to avoid looping
Mon, 08 Nov 2021 19:56:15 +0100 nipkow added eq_iff_swap for creating symmetric variants of thms; applied it in List.
Sat, 02 Oct 2021 20:31:46 +0200 wenzelm trim whitespace;
Mon, 02 Aug 2021 10:01:06 +0000 haftmann moved theory Bit_Operations into Main corpus
Thu, 08 Jul 2021 08:42:36 +0200 desharna added opaque_combs and renamed hide_lams to opaque_lifting
Tue, 01 Jun 2021 19:46:34 +0200 nipkow More general fold function for maps
less more (0) -300 -100 -60 tip