Thu, 26 Jun 2025 17:25:29 +0200 |
haftmann |
append (rather than prepend) code equations: the order within a theory is maintained in the resulting code
|
file |
diff |
annotate
|
Mon, 21 Apr 2025 08:24:58 +0200 |
haftmann |
more efficient conversions for symbolic representations
|
file |
diff |
annotate
|
Tue, 15 Apr 2025 19:40:42 +0200 |
haftmann |
corrected operation
|
file |
diff |
annotate
|
Tue, 15 Apr 2025 19:40:39 +0200 |
haftmann |
tuned whitespace
|
file |
diff |
annotate
|
Sat, 05 Apr 2025 08:49:53 +0200 |
haftmann |
incorporate target-language integer implementation of bit shifts into Main
|
file |
diff |
annotate
|
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
|
Sun, 08 Oct 2017 22:28:20 +0200 |
haftmann |
avoid fact name clashes
|
file |
diff |
annotate
|
Sat, 24 Jun 2017 09:17:35 +0200 |
haftmann |
more direct construction of integer_of_num;
|
file |
diff |
annotate
|
Mon, 06 Feb 2017 20:56:38 +0100 |
haftmann |
computation preprocessing rules to allow literals as input for computations
|
file |
diff |
annotate
|
Mon, 09 Jan 2017 18:53:06 +0100 |
haftmann |
slightly generalized type class hierarchy concerning unit factors, to allow for lean polynomial normalization
|
file |
diff |
annotate
|
Sat, 17 Dec 2016 15:22:14 +0100 |
haftmann |
more fine-grained type class hierarchy for div and mod
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:06 +0200 |
haftmann |
eliminated irregular aliasses
|
file |
diff |
annotate
|
Sun, 16 Oct 2016 09:31:04 +0200 |
haftmann |
transfer rules for divides relation on integer and natural
|
file |
diff |
annotate
|
Wed, 12 Oct 2016 21:48:53 +0200 |
haftmann |
transfer lifting rule for numeral
|
file |
diff |
annotate
|
Mon, 26 Sep 2016 07:56:54 +0200 |
haftmann |
syntactic type class for operation mod named after mod;
|
file |
diff |
annotate
|
Sun, 29 May 2016 14:43:17 +0200 |
haftmann |
do not export abstract constructors in code_reflect
|
file |
diff |
annotate
|
Fri, 18 Dec 2015 14:23:11 +0100 |
Andreas Lochbihler |
add serialisation for abs on integer to target language operation
|
file |
diff |
annotate
|
Sun, 27 Sep 2015 10:11:15 +0200 |
haftmann |
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
|
file |
diff |
annotate
|
Sun, 27 Sep 2015 10:11:14 +0200 |
haftmann |
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
|
file |
diff |
annotate
|
Tue, 01 Sep 2015 22:32:58 +0200 |
wenzelm |
eliminated \<Colon>;
|
file |
diff |
annotate
|
Sat, 08 Aug 2015 10:51:33 +0200 |
haftmann |
direct bootstrap of integer division from natural division
|
file |
diff |
annotate
|
Sat, 18 Jul 2015 22:58:50 +0200 |
wenzelm |
isabelle update_cartouches;
|
file |
diff |
annotate
|
Tue, 23 Jun 2015 16:55:28 +0100 |
paulson |
Amalgamation of the class comm_semiring_1_diff_distrib into comm_semiring_1_cancel. Moving axiom le_add_diff_inverse2 from semiring_numeral_div to linordered_semidom.
|
file |
diff |
annotate
|
Mon, 01 Jun 2015 18:59:21 +0200 |
haftmann |
separate class for division operator, with particular syntax added in more specific classes
|
file |
diff |
annotate
|
Mon, 23 Mar 2015 19:05:14 +0100 |
haftmann |
distributivity of partial minus establishes desired properties of dvd in semirings
|
file |
diff |
annotate
|
Fri, 06 Feb 2015 17:57:03 +0100 |
haftmann |
default abstypes and default abstract equations make technical (no_code) annotation superfluous
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 18:21:45 +0100 |
wenzelm |
modernized header uniformly as section;
|
file |
diff |
annotate
|
Thu, 18 Sep 2014 18:48:54 +0200 |
haftmann |
always annotate potentially polymorphic Haskell numerals
|
file |
diff |
annotate
|
Thu, 18 Sep 2014 18:48:04 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Fri, 19 Sep 2014 13:27:04 +0200 |
blanchet |
keep obsolete interpretations in Main, to avoid merge trouble
|
file |
diff |
annotate
|
Thu, 18 Sep 2014 16:57:10 +0200 |
blanchet |
reintroduced an instantiation of 'size' for 'numerals'
|
file |
diff |
annotate
|
Thu, 18 Sep 2014 16:47:40 +0200 |
blanchet |
moved old 'size' generator together with 'old_datatype'
|
file |
diff |
annotate
|
Thu, 11 Sep 2014 18:54:36 +0200 |
blanchet |
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
|
file |
diff |
annotate
|
Fri, 04 Jul 2014 20:18:47 +0200 |
haftmann |
reduced name variants for assoc and commute on plus and mult
|
file |
diff |
annotate
|
Sun, 04 May 2014 18:14:58 +0200 |
blanchet |
renamed 'xxx_size' to 'size_xxx' for old datatype package
|
file |
diff |
annotate
|
Thu, 06 Mar 2014 15:40:33 +0100 |
blanchet |
renamed 'fun_rel' to 'rel_fun'
|
file |
diff |
annotate
|
Tue, 25 Feb 2014 19:07:14 +0100 |
kuncar |
unregister lifting setup following the best practice of Lifting
|
file |
diff |
annotate
|
Fri, 21 Feb 2014 00:09:56 +0100 |
blanchet |
adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
|
file |
diff |
annotate
|
Wed, 12 Feb 2014 10:59:25 +0100 |
Andreas Lochbihler |
merged
|
file |
diff |
annotate
|
Wed, 12 Feb 2014 09:06:04 +0100 |
Andreas Lochbihler |
make integer_of_char and char_of_integer work with NBE and code_simp
|
file |
diff |
annotate
|
Wed, 12 Feb 2014 08:35:57 +0100 |
blanchet |
adapted theories to 'xxx_case' to 'case_xxx'
|
file |
diff |
annotate
|
Wed, 12 Feb 2014 08:35:57 +0100 |
blanchet |
renamed '{prod,sum,bool,unit}_case' to 'case_...'
|
file |
diff |
annotate
|
Tue, 19 Nov 2013 10:05:53 +0100 |
haftmann |
eliminiated neg_numeral in favour of - (numeral _)
|
file |
diff |
annotate
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
|
file |
diff |
annotate
|
Sun, 23 Jun 2013 21:16:07 +0200 |
haftmann |
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
|
file |
diff |
annotate
|
Fri, 08 Mar 2013 13:21:06 +0100 |
kuncar |
patch Isabelle ditribution to conform to changes regarding the parametricity
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 08:31:31 +0100 |
haftmann |
two target language numeral types: integer and natural, as replacement for code_numeral;
|
file |
diff |
annotate
|
Fri, 19 Oct 2012 15:12:52 +0200 |
webertj |
Renamed {left,right}_distrib to distrib_{right,left}.
|
file |
diff |
annotate
|
Fri, 12 Oct 2012 18:58:20 +0200 |
wenzelm |
discontinued obsolete typedef (open) syntax;
|
file |
diff |
annotate
|
Mon, 23 Jul 2012 09:28:03 +0200 |
haftmann |
restrict unqualified imports from Haskell Prelude to a small set of fundamental operations
|
file |
diff |
annotate
|
Sun, 01 Apr 2012 16:09:58 +0200 |
huffman |
removed Nat_Numeral.thy, moving all theorems elsewhere
|
file |
diff |
annotate
|
Sun, 25 Mar 2012 20:15:39 +0200 |
huffman |
merged fork with new numeral representation (see NEWS)
|
file |
diff |
annotate
|
Fri, 24 Feb 2012 22:46:44 +0100 |
haftmann |
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
|
file |
diff |
annotate
|
Fri, 24 Feb 2012 09:40:02 +0100 |
haftmann |
given up disfruitful branch
|
file |
diff |
annotate
|
Thu, 23 Feb 2012 21:25:59 +0100 |
haftmann |
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
|
file |
diff |
annotate
|
Mon, 20 Feb 2012 12:37:17 +0100 |
huffman |
use qualified constant names instead of suffixes (from Florian Haftmann)
|
file |
diff |
annotate
|
Thu, 29 Dec 2011 10:47:55 +0100 |
haftmann |
attribute code_abbrev superseedes code_unfold_post
|
file |
diff |
annotate
|
Wed, 30 Nov 2011 16:27:10 +0100 |
wenzelm |
prefer typedef without extra definition and alternative name;
|
file |
diff |
annotate
|
Wed, 07 Sep 2011 09:02:58 -0700 |
huffman |
avoid using legacy theorem names
|
file |
diff |
annotate
|
Fri, 01 Oct 2010 14:15:49 +0200 |
haftmann |
use module integer for Eval
|
file |
diff |
annotate
|
Fri, 10 Sep 2010 10:21:25 +0200 |
haftmann |
Haskell == is infix, not infixl
|
file |
diff |
annotate
|