src/HOL/Code_Numeral.thy
Fri, 05 Apr 2024 21:21:02 +0200 wenzelm avoid Scala if-expressions and thus make it work both for -new-syntax or -old-syntax;
Wed, 21 Feb 2024 16:19:36 +0000 haftmann simplified specification of type class semiring_bits
Fri, 09 Feb 2024 16:43:43 +0000 haftmann simplified class specification
Tue, 06 Feb 2024 18:08:43 +0000 haftmann more lemmas and more correct lemma names
Mon, 29 Jan 2024 19:35:07 +0000 haftmann common type class for trivial properties on div/mod
Thu, 25 Jan 2024 11:19:03 +0000 haftmann rearranged and reformulated abstract classes for bit structures and operations
Sun, 14 Jan 2024 20:02:58 +0000 haftmann streamlined type class specification
Sun, 14 Jan 2024 20:02:55 +0000 haftmann consolidated lemma name
Sat, 13 Jan 2024 19:50:15 +0000 haftmann simplified specification of type class
Sat, 13 Jan 2024 19:50:12 +0000 haftmann consolidated name of lemma analogously to nat/int/word_bit_induct
Tue, 28 Nov 2023 17:39:26 +0000 haftmann de-duplicated specification of class ring_bit_operations
Thu, 23 Nov 2023 16:49:39 +0000 haftmann slightly more elementary characterization of unset_bit
Wed, 22 Nov 2023 17:50:36 +0000 haftmann base abstract specification of NOT on recursive equation rather than bit projection
Tue, 21 Nov 2023 19:19:16 +0000 haftmann more correct type annotation
Sun, 19 Nov 2023 15:45:22 +0000 haftmann operations AND, OR, XOR are specified by characteristic recursive equation
Sat, 11 Nov 2023 17:44:03 +0000 haftmann more specific name for type class
Thu, 09 Nov 2023 15:11:52 +0000 haftmann slightly less technical formulation of very specific type class
Thu, 09 Nov 2023 15:11:51 +0000 haftmann explicit type class for discrete linordered semidoms
Sat, 16 Sep 2023 06:38:44 +0000 haftmann reduced prominence of lemma names
Mon, 05 Sep 2022 16:39:23 +0200 haftmann clarified generic euclidean relation
Sun, 21 Aug 2022 06:18:23 +0000 haftmann simplified computation algorithm construction
Fri, 19 Aug 2022 05:49:17 +0000 haftmann tuned type signature
Mon, 13 Sep 2021 14:18:24 +0000 haftmann explicit predicate for confined bit range avoids cyclic rewriting in presence of extensionality rule for bit values (contributed by Thomas Sewell)
Tue, 03 Aug 2021 13:53:22 +0000 haftmann simplified hierarchy of type classes for bit operations
Mon, 02 Aug 2021 10:01:06 +0000 haftmann moved theory Bit_Operations into Main corpus
Sat, 20 Jun 2020 05:56:28 +0000 haftmann more class operations for the sake of efficient generated code
Sun, 08 Mar 2020 17:07:49 +0000 haftmann more frugal simp rules for bit operations; more pervasive use of bit selector
Sun, 09 Feb 2020 10:46:32 +0000 haftmann rule concerning bit (push_bit ...)
Sat, 01 Feb 2020 19:10:40 +0100 haftmann more specific class assumptions
Mon, 02 Dec 2019 17:15:16 +0000 haftmann tuned material
Sun, 01 Dec 2019 08:00:59 +0000 haftmann characterization of singleton bit operation
Sun, 17 Nov 2019 20:44:35 +0000 haftmann strengthened type class for bit operations
Sat, 09 Nov 2019 15:39:21 +0000 haftmann bit shifts as class operations
Wed, 23 Oct 2019 16:09:23 +0000 haftmann tuned syntax
Fri, 14 Jun 2019 08:34:27 +0000 haftmann slightly more specialized name for type class
Sat, 30 Mar 2019 15:37:22 +0100 haftmann irrelevant
Thu, 28 Mar 2019 21:24:55 +0100 wenzelm "export_code ... file_prefix ..." is the preferred way to produce output within the logical file-system within the theory context, as well as session exports;
Fri, 22 Mar 2019 19:18:08 +0000 haftmann improved code equations taken over from AFP
Sun, 10 Mar 2019 15:16:45 +0000 haftmann migrated from Nums to Zarith as library for OCaml integer arithmetic
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Tue, 24 Apr 2018 14:17:58 +0000 haftmann proper datatype for 8-bit characters
Fri, 20 Apr 2018 07:36:58 +0000 haftmann algebraic embeddings for bit operations
Tue, 20 Mar 2018 09:27:39 +0000 haftmann generalized
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Wed, 03 Jan 2018 11:06:13 +0100 blanchet kill old size infrastructure
Fri, 20 Oct 2017 07:46:10 +0200 haftmann added lemmas and tuned proofs
Mon, 09 Oct 2017 19:10:51 +0200 haftmann clarified parity
Mon, 09 Oct 2017 19:10:49 +0200 haftmann clarified uniqueness criterion for euclidean rings
Mon, 09 Oct 2017 19:10:47 +0200 haftmann tuned imports
Sun, 08 Oct 2017 22:28:22 +0200 haftmann euclidean rings need no normalization
Sun, 08 Oct 2017 22:28:22 +0200 haftmann one uniform type class for parity structures
Sun, 08 Oct 2017 22:28:21 +0200 haftmann abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
Sun, 08 Oct 2017 22:28:20 +0200 haftmann avoid fact name clashes
Sat, 24 Jun 2017 09:17:35 +0200 haftmann more direct construction of integer_of_num;
Mon, 06 Feb 2017 20:56:38 +0100 haftmann computation preprocessing rules to allow literals as input for computations
Mon, 09 Jan 2017 18:53:06 +0100 haftmann slightly generalized type class hierarchy concerning unit factors, to allow for lean polynomial normalization
Sat, 17 Dec 2016 15:22:14 +0100 haftmann more fine-grained type class hierarchy for div and mod
Sun, 16 Oct 2016 09:31:06 +0200 haftmann eliminated irregular aliasses
Sun, 16 Oct 2016 09:31:04 +0200 haftmann transfer rules for divides relation on integer and natural
Wed, 12 Oct 2016 21:48:53 +0200 haftmann transfer lifting rule for numeral
less more (0) -100 -60 tip