Thu, 09 Jan 2025 08:33:11 +0100 |
haftmann |
direct symbolic implementations of and, or, xor on integer
|
file |
diff |
annotate
|
Sat, 04 Jan 2025 20:24:12 +0100 |
haftmann |
delegate computation to integer thoroughly
|
file |
diff |
annotate
|
Sat, 04 Jan 2025 14:41:30 +0100 |
haftmann |
optionally use shift operations on target numerals for efficient execution
|
file |
diff |
annotate
|
Sat, 04 Jan 2025 14:25:56 +0100 |
haftmann |
some bit operations on target numerals
|
file |
diff |
annotate
|
Thu, 02 Jan 2025 08:37:55 +0100 |
haftmann |
refined syntax for code_reserved
|
file |
diff |
annotate
|
Sat, 28 Dec 2024 21:20:33 +0100 |
nipkow |
Backed out changeset 0ca0a47235e5 (produced Code check failed for Haskell?)
|
file |
diff |
annotate
|
Mon, 23 Dec 2024 21:58:26 +0100 |
haftmann |
some bit operations on target numerals
|
file |
diff |
annotate
|
Thu, 19 Dec 2024 15:13:33 +0100 |
haftmann |
more default simp rules
|
file |
diff |
annotate
|
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;
|
file |
diff |
annotate
|
Wed, 21 Feb 2024 16:19:36 +0000 |
haftmann |
simplified specification of type class semiring_bits
|
file |
diff |
annotate
|
Fri, 09 Feb 2024 16:43:43 +0000 |
haftmann |
simplified class specification
|
file |
diff |
annotate
|
Tue, 06 Feb 2024 18:08:43 +0000 |
haftmann |
more lemmas and more correct lemma names
|
file |
diff |
annotate
|
Mon, 29 Jan 2024 19:35:07 +0000 |
haftmann |
common type class for trivial properties on div/mod
|
file |
diff |
annotate
|
Thu, 25 Jan 2024 11:19:03 +0000 |
haftmann |
rearranged and reformulated abstract classes for bit structures and operations
|
file |
diff |
annotate
|
Sun, 14 Jan 2024 20:02:58 +0000 |
haftmann |
streamlined type class specification
|
file |
diff |
annotate
|
Sun, 14 Jan 2024 20:02:55 +0000 |
haftmann |
consolidated lemma name
|
file |
diff |
annotate
|
Sat, 13 Jan 2024 19:50:15 +0000 |
haftmann |
simplified specification of type class
|
file |
diff |
annotate
|
Sat, 13 Jan 2024 19:50:12 +0000 |
haftmann |
consolidated name of lemma analogously to nat/int/word_bit_induct
|
file |
diff |
annotate
|
Tue, 28 Nov 2023 17:39:26 +0000 |
haftmann |
de-duplicated specification of class ring_bit_operations
|
file |
diff |
annotate
|
Thu, 23 Nov 2023 16:49:39 +0000 |
haftmann |
slightly more elementary characterization of unset_bit
|
file |
diff |
annotate
|
Wed, 22 Nov 2023 17:50:36 +0000 |
haftmann |
base abstract specification of NOT on recursive equation rather than bit projection
|
file |
diff |
annotate
|
Tue, 21 Nov 2023 19:19:16 +0000 |
haftmann |
more correct type annotation
|
file |
diff |
annotate
|
Sun, 19 Nov 2023 15:45:22 +0000 |
haftmann |
operations AND, OR, XOR are specified by characteristic recursive equation
|
file |
diff |
annotate
|
Sat, 11 Nov 2023 17:44:03 +0000 |
haftmann |
more specific name for type class
|
file |
diff |
annotate
|
Thu, 09 Nov 2023 15:11:52 +0000 |
haftmann |
slightly less technical formulation of very specific type class
|
file |
diff |
annotate
|
Thu, 09 Nov 2023 15:11:51 +0000 |
haftmann |
explicit type class for discrete linordered semidoms
|
file |
diff |
annotate
|
Sat, 16 Sep 2023 06:38:44 +0000 |
haftmann |
reduced prominence of lemma names
|
file |
diff |
annotate
|
Mon, 05 Sep 2022 16:39:23 +0200 |
haftmann |
clarified generic euclidean relation
|
file |
diff |
annotate
|
Sun, 21 Aug 2022 06:18:23 +0000 |
haftmann |
simplified computation algorithm construction
|
file |
diff |
annotate
|
Fri, 19 Aug 2022 05:49:17 +0000 |
haftmann |
tuned type signature
|
file |
diff |
annotate
|
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)
|
file |
diff |
annotate
|
Tue, 03 Aug 2021 13:53:22 +0000 |
haftmann |
simplified hierarchy of type classes for bit operations
|
file |
diff |
annotate
|
Mon, 02 Aug 2021 10:01:06 +0000 |
haftmann |
moved theory Bit_Operations into Main corpus
|
file |
diff |
annotate
|
Sat, 20 Jun 2020 05:56:28 +0000 |
haftmann |
more class operations for the sake of efficient generated code
|
file |
diff |
annotate
|
Sun, 08 Mar 2020 17:07:49 +0000 |
haftmann |
more frugal simp rules for bit operations; more pervasive use of bit selector
|
file |
diff |
annotate
|
Sun, 09 Feb 2020 10:46:32 +0000 |
haftmann |
rule concerning bit (push_bit ...)
|
file |
diff |
annotate
|
Sat, 01 Feb 2020 19:10:40 +0100 |
haftmann |
more specific class assumptions
|
file |
diff |
annotate
|
Mon, 02 Dec 2019 17:15:16 +0000 |
haftmann |
tuned material
|
file |
diff |
annotate
|
Sun, 01 Dec 2019 08:00:59 +0000 |
haftmann |
characterization of singleton bit operation
|
file |
diff |
annotate
|
Sun, 17 Nov 2019 20:44:35 +0000 |
haftmann |
strengthened type class for bit operations
|
file |
diff |
annotate
|
Sat, 09 Nov 2019 15:39:21 +0000 |
haftmann |
bit shifts as class operations
|
file |
diff |
annotate
|
Wed, 23 Oct 2019 16:09:23 +0000 |
haftmann |
tuned syntax
|
file |
diff |
annotate
|
Fri, 14 Jun 2019 08:34:27 +0000 |
haftmann |
slightly more specialized name for type class
|
file |
diff |
annotate
|
Sat, 30 Mar 2019 15:37:22 +0100 |
haftmann |
irrelevant
|
file |
diff |
annotate
|
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;
|
file |
diff |
annotate
|
Fri, 22 Mar 2019 19:18:08 +0000 |
haftmann |
improved code equations taken over from AFP
|
file |
diff |
annotate
|
Sun, 10 Mar 2019 15:16:45 +0000 |
haftmann |
migrated from Nums to Zarith as library for OCaml integer arithmetic
|
file |
diff |
annotate
|
Fri, 04 Jan 2019 23:22:53 +0100 |
wenzelm |
isabelle update -u control_cartouches;
|
file |
diff |
annotate
|
Tue, 24 Apr 2018 14:17:58 +0000 |
haftmann |
proper datatype for 8-bit characters
|
file |
diff |
annotate
|
Fri, 20 Apr 2018 07:36:58 +0000 |
haftmann |
algebraic embeddings for bit operations
|
file |
diff |
annotate
|
Tue, 20 Mar 2018 09:27:39 +0000 |
haftmann |
generalized
|
file |
diff |
annotate
|
Wed, 10 Jan 2018 15:25:09 +0100 |
nipkow |
ran isabelle update_op on all sources
|
file |
diff |
annotate
|
Wed, 03 Jan 2018 11:06:13 +0100 |
blanchet |
kill old size infrastructure
|
file |
diff |
annotate
|
Fri, 20 Oct 2017 07:46:10 +0200 |
haftmann |
added lemmas and tuned proofs
|
file |
diff |
annotate
|
Mon, 09 Oct 2017 19:10:51 +0200 |
haftmann |
clarified parity
|
file |
diff |
annotate
|
Mon, 09 Oct 2017 19:10:49 +0200 |
haftmann |
clarified uniqueness criterion for euclidean rings
|
file |
diff |
annotate
|
Mon, 09 Oct 2017 19:10:47 +0200 |
haftmann |
tuned imports
|
file |
diff |
annotate
|
Sun, 08 Oct 2017 22:28:22 +0200 |
haftmann |
euclidean rings need no normalization
|
file |
diff |
annotate
|
Sun, 08 Oct 2017 22:28:22 +0200 |
haftmann |
one uniform type class for parity structures
|
file |
diff |
annotate
|
Sun, 08 Oct 2017 22:28:21 +0200 |
haftmann |
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
|
file |
diff |
annotate
|