src/HOL/List.thy
Thu, 12 Jun 2025 08:03:05 +0200 haftmann reorganized more code-only operations
Mon, 09 Jun 2025 22:14:38 +0200 haftmann more qualified auxiliary operations
Thu, 05 Jun 2025 15:18:27 +0000 haftmann prefer already existing operation to calculate minimum
Wed, 04 Jun 2025 19:43:13 +0000 haftmann tuned syntax
Sat, 31 May 2025 21:51:08 +0200 haftmann generic executable ranges
Fri, 30 May 2025 08:02:55 +0200 haftmann explicit abort for big lattice operations over non-empty sets
Fri, 30 May 2025 08:02:54 +0200 haftmann prefer explicit operation to make generated code more abstract
Fri, 30 May 2025 07:48:17 +0200 haftmann tuned theory structure
Fri, 30 May 2025 07:47:03 +0200 haftmann qualify can_select auxiliary operations
Wed, 28 May 2025 17:49:22 +0200 haftmann more modern qualification of auxiliary operations
Thu, 22 May 2025 19:59:43 +0200 nipkow added lemmas
Fri, 09 May 2025 14:15:10 +0200 nipkow added lemma
Sun, 04 May 2025 20:50:01 +0200 haftmann new lemma
Sun, 30 Mar 2025 13:50:06 +0200 haftmann tuned namespace organisation
Tue, 11 Mar 2025 10:20:44 +0100 desharna changed definition of refl_on
Wed, 05 Mar 2025 15:34:01 +0100 nipkow more take/drop/While lemmas (by Martin Desharnais)
Wed, 19 Feb 2025 10:12:35 +0100 nipkow added lemma
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
less more (0) -300 -100 -60 tip