src/HOL/Wellfounded.thy
Tue, 26 Mar 2024 09:31:34 +0100 desharna added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
Mon, 25 Mar 2024 19:27:53 +0100 desharna added lemma wf_on_iff_wf
Mon, 25 Mar 2024 19:27:32 +0100 desharna changed number of consumed assumptions of wf_on_induct and wfp_on_induct
Sat, 23 Mar 2024 18:55:38 +0100 desharna redefined wf as an abbreviation for "wf_on UNIV"
Thu, 21 Mar 2024 11:24:03 +0100 desharna redefined wfP as an abbreviation for "wfp_on UNIV"
Wed, 20 Mar 2024 21:13:49 +0100 desharna added lemma wellorder.wfp_on_less[simp]
Sun, 17 Mar 2024 19:45:07 +0100 desharna added alias wfp for wfP
Sun, 17 Mar 2024 12:34:11 +0100 desharna added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
Sun, 17 Mar 2024 09:05:44 +0100 desharna tuned proofs
Sun, 17 Mar 2024 09:03:18 +0100 desharna added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
Sat, 16 Mar 2024 09:05:17 +0100 desharna added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
Wed, 01 Feb 2023 20:21:33 +0100 wenzelm isabelle update -u cite -l "";
Mon, 19 Dec 2022 16:20:57 +0100 desharna added lemma trans_on_lex_prod[simp]
Mon, 19 Dec 2022 12:00:56 +0100 desharna added lemma refl_lex_prod[simp]
Mon, 19 Dec 2022 11:26:56 +0100 desharna added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
Mon, 19 Dec 2022 11:25:37 +0100 desharna added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
Mon, 19 Dec 2022 11:23:28 +0100 desharna added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
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 18:56:28 +0100 desharna rewrite proofs using to_pred attribute on existing lemmas
Mon, 21 Nov 2022 14:11:30 +0100 desharna introduced predicates irrefl_on and irreflp_on, and redefined irrefl and irreflp as abbreviations
Wed, 12 Oct 2022 14:37:03 +0200 desharna added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
Fri, 22 Jul 2022 14:39:56 +0200 Fabian Huch tuned (some HOL lints, by Yecine Megdiche);
Thu, 06 Jan 2022 17:45:07 +0100 desharna added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
Sun, 28 Nov 2021 19:12:48 +0100 desharna added wfP_less to wellorder and wfP_less_multiset
Fri, 21 Aug 2020 12:42:57 +0100 paulson reversing all the lex crap
Wed, 19 Aug 2020 12:58:28 +0100 paulson Another go with lex: now lexordp back in class ord
Tue, 18 Aug 2020 17:38:51 +0100 paulson lexicographic ordering: new simp setup to prioritise the simpler "less_than" case
Mon, 17 Aug 2020 15:42:38 +0100 paulson S Holub's proposed generalisation of the lexicographic product of two orderings
Thu, 11 Jun 2020 16:13:53 +0100 paulson fixed the utterly weird definitions of asym / asymp, and added many asym lemmas
Mon, 11 May 2020 11:15:41 +0100 paulson the Uniq quantifier
Fri, 17 Apr 2020 20:55:53 +0100 paulson New theory Library/List_Lenlexorder.thy, a type class instantiation for well-ordering lists
Sat, 14 Mar 2020 15:58:51 +0000 paulson tidied up a few little proofs
Tue, 28 Jan 2020 14:59:54 +0000 paulson Tidied up some messy proofs
Mon, 27 Jan 2020 14:32:43 +0000 paulson A few lemmas connected with orderings
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Sat, 10 Nov 2018 07:57:19 +0000 haftmann clarified status of legacy input abbreviations
Tue, 17 Jul 2018 22:18:27 +0100 paulson more de-applying
Thu, 24 May 2018 16:38:24 +0200 nipkow tuned
Thu, 24 May 2018 07:59:41 +0200 nipkow By Andrei Popescu based on an initial version by Kasper F. Brandt
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Mon, 30 Oct 2017 21:52:31 +0100 blanchet added 'mlex_iff' lemma and simplified proof
Wed, 21 Dec 2016 21:26:26 +0100 haftmann dropped aliasses
Sat, 01 Oct 2016 19:30:21 +0200 wenzelm tuned;
Sun, 18 Sep 2016 20:33:48 +0200 wenzelm tuned proofs;
Fri, 05 Aug 2016 18:14:28 +0200 wenzelm misc tuning and modernization;
Sun, 31 Jul 2016 22:56:18 +0200 wenzelm misc tuning and modernization;
Mon, 23 May 2016 12:48:24 +0200 wenzelm proper document source;
Mon, 23 May 2016 12:18:16 +0200 wenzelm misc tuning and modernization;
Tue, 17 May 2016 17:05:35 +0200 eberlm Moved material from AFP/Randomised_Social_Choice to distribution
Thu, 12 May 2016 09:34:07 +0200 haftmann a quasi-recursive characterization of the multiset order (by Christian Sternagel)
Mon, 28 Dec 2015 17:43:30 +0100 wenzelm prefer symbols for "Union", "Inter";
Sun, 27 Dec 2015 22:07:17 +0100 wenzelm discontinued ASCII replacement syntax <*>;
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 13 Oct 2015 09:21:15 +0200 haftmann prod_case as canonical name for product type eliminator
Tue, 06 Oct 2015 15:14:28 +0200 wenzelm fewer aliases for toplevel theorem statements;
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Wed, 17 Jun 2015 14:35:50 +0100 paulson New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
Mon, 27 Apr 2015 15:02:51 +0200 nipkow new lemma
Wed, 25 Mar 2015 10:44:57 +0100 wenzelm prefer local fixes;
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
less more (0) -100 -60 tip