Fri, 24 Mar 2023 18:30:17 +0000 |
haftmann |
more uniform approach towards satisfied applications
|
file |
diff |
annotate
|
Thu, 09 Feb 2023 13:50:09 +0100 |
stuebinm |
explicit range types in abstractions
|
file |
diff |
annotate
|
Sun, 12 Feb 2023 06:45:59 +0000 |
haftmann |
somehow more clear terminology
|
file |
diff |
annotate
|
Wed, 06 Jul 2022 13:08:33 +0200 |
wenzelm |
minor performance tuning: avoid redundant BigInt construction;
|
file |
diff |
annotate
|
Sun, 17 Jan 2021 00:16:14 +0100 |
wenzelm |
updated to scala-2.13: its ArraySeq implementation is not usable here (requires scala.relection.ClassTag);
|
file |
diff |
annotate
|
Sat, 19 Jan 2019 07:19:16 +0000 |
haftmann |
self-contained code modules for Haskell
|
file |
diff |
annotate
|
Sat, 05 Jan 2019 17:24:33 +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
|
Wed, 10 Jan 2018 15:25:09 +0100 |
nipkow |
ran isabelle update_op on all sources
|
file |
diff |
annotate
|
Fri, 18 Aug 2017 20:47:47 +0200 |
wenzelm |
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
|
file |
diff |
annotate
|
Tue, 20 Jun 2017 13:07:47 +0200 |
haftmann |
avoid ancient [code, code del] antipattern
|
file |
diff |
annotate
|
Thu, 26 May 2016 17:51:22 +0200 |
wenzelm |
isabelle update_cartouches -c -t;
|
file |
diff |
annotate
|
Fri, 01 Jan 2016 14:44:52 +0100 |
wenzelm |
more symbols;
|
file |
diff |
annotate
|
Mon, 09 Nov 2015 15:48:17 +0100 |
wenzelm |
qualifier is mandatory by default;
|
file |
diff |
annotate
|
Wed, 04 Nov 2015 08:13:52 +0100 |
ballarin |
Keyword 'rewrites' identifies rewrite morphisms.
|
file |
diff |
annotate
|
Fri, 05 Dec 2014 19:35:36 +0100 |
haftmann |
allow multiple inheritance of targets
|
file |
diff |
annotate
|
Wed, 26 Nov 2014 20:05:34 +0100 |
wenzelm |
renamed "pairself" to "apply2", in accordance to @{apply 2};
|
file |
diff |
annotate
|
Sat, 22 Nov 2014 11:36:00 +0100 |
wenzelm |
named_theorems: multiple args;
|
file |
diff |
annotate
|
Sat, 08 Nov 2014 09:16:47 +0100 |
haftmann |
less space-wasting serialization setup: highest cell of array has been unused so far
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 18:21:45 +0100 |
wenzelm |
modernized header uniformly as section;
|
file |
diff |
annotate
|
Thu, 02 Oct 2014 11:33:04 +0200 |
haftmann |
tuned Heap_Monad.successE
|
file |
diff |
annotate
|
Thu, 18 Sep 2014 18:48:04 +0200 |
haftmann |
tuned data structure
|
file |
diff |
annotate
|
Thu, 11 Sep 2014 19:32:36 +0200 |
blanchet |
updated news
|
file |
diff |
annotate
|
Tue, 09 Sep 2014 20:51:36 +0200 |
blanchet |
use 'datatype_new' (soon to be renamed 'datatype') in Isabelle's libraries
|
file |
diff |
annotate
|
Sat, 16 Aug 2014 18:08:55 +0200 |
wenzelm |
updated to named_theorems;
|
file |
diff |
annotate
|
Mon, 30 Jun 2014 08:00:36 +0200 |
haftmann |
qualified String.explode and String.implode
|
file |
diff |
annotate
|
Sun, 09 Feb 2014 21:37:27 +0100 |
haftmann |
dropped legacy finally
|
file |
diff |
annotate
|
Sat, 25 Jan 2014 23:50:49 +0100 |
haftmann |
prefer explicit code symbol type over ad-hoc name mangling
|
file |
diff |
annotate
|
Thu, 05 Dec 2013 09:20:32 +0100 |
Andreas Lochbihler |
restrict admissibility to non-empty chains to allow more syntax-directed proof rules
|
file |
diff |
annotate
|
Mon, 02 Sep 2013 16:28:11 +0200 |
Andreas Lochbihler |
move admissible out of class ccpo to avoid unnecessary class predicate in foundational theorems
|
file |
diff |
annotate
|
Wed, 24 Jul 2013 17:15:59 +0200 |
krauss |
derive specialized version of full fixpoint induction (with admissibility)
|
file |
diff |
annotate
|
Fri, 12 Jul 2013 16:19:05 +0200 |
wenzelm |
localized and modernized adhoc-overloading (patch by Christian Sternagel);
|
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
|
Tue, 18 Jun 2013 15:35:53 +0200 |
lammich |
Added parantheses to code_type for heap monad
|
file |
diff |
annotate
|
Fri, 22 Mar 2013 00:39:16 +0100 |
krauss |
added rudimentary induction rule for partial_function (heap)
|
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
|
Tue, 05 Jun 2012 07:10:51 +0200 |
haftmann |
prefer sys.error over plain error in Scala to avoid deprecation warning
|
file |
diff |
annotate
|
Tue, 05 Jun 2012 07:05:56 +0200 |
haftmann |
prefer records with speaking labels over deeply nested tuples
|
file |
diff |
annotate
|
Thu, 29 Dec 2011 10:47:55 +0100 |
haftmann |
attribute code_abbrev superseedes code_unfold_post; tuned names and spacing
|
file |
diff |
annotate
|
Fri, 28 Oct 2011 23:41:16 +0200 |
wenzelm |
tuned Named_Thms: proper binding;
|
file |
diff |
annotate
|
Fri, 21 Oct 2011 11:17:14 +0200 |
bulwahn |
replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
|
file |
diff |
annotate
|
Wed, 07 Sep 2011 13:51:37 +0200 |
bulwahn |
adapting Imperative HOL serializer to changes of the iterm datatype in the code generator
|
file |
diff |
annotate
|
Fri, 12 Aug 2011 14:45:50 -0700 |
huffman |
make more HOL theories work with separate set type
|
file |
diff |
annotate
|
Thu, 09 Jun 2011 16:34:49 +0200 |
wenzelm |
discontinued Name.variant to emphasize that this is old-style / indirect;
|
file |
diff |
annotate
|
Mon, 23 May 2011 21:34:37 +0200 |
krauss |
also manage induction rule;
|
file |
diff |
annotate
|
Mon, 23 May 2011 10:58:21 +0200 |
krauss |
separate initializations for different modes of partial_function -- generation of induction rules will be non-uniform
|
file |
diff |
annotate
|
Wed, 29 Dec 2010 17:34:41 +0100 |
wenzelm |
explicit file specifications -- avoid secondary load path;
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 09:37:39 +0100 |
haftmann |
renamed slightly ambivalent crel to effect
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 14:03:02 +0200 |
haftmann |
tuned structure of theory
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 13:49:49 +0200 |
haftmann |
remove term_of equations for Heap type explicitly
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 12:19:02 +0200 |
krauss |
added Heap monad instance of partial_function package
|
file |
diff |
annotate
|
Mon, 13 Sep 2010 11:13:15 +0200 |
nipkow |
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
|
file |
diff |
annotate
|
Thu, 09 Sep 2010 14:38:14 +0200 |
bulwahn |
changing String.literal to a type instead of a datatype
|
file |
diff |
annotate
|
Tue, 07 Sep 2010 10:05:19 +0200 |
nipkow |
expand_fun_eq -> ext_iff
|
file |
diff |
annotate
|
Wed, 01 Sep 2010 15:51:49 +0200 |
haftmann |
Graph.map, in analogy to Table.map
|
file |
diff |
annotate
|
Wed, 01 Sep 2010 11:09:50 +0200 |
haftmann |
do not print object frame around Scala includes -- this is in the responsibility of the user
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 12:19:49 +0200 |
haftmann |
prevent line breaks after Scala symbolic operators
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 10:16:22 +0200 |
haftmann |
code_include Scala: qualify module nmae
|
file |
diff |
annotate
|
Fri, 13 Aug 2010 14:45:07 +0200 |
haftmann |
lemma execute_bind_case
|
file |
diff |
annotate
|
Thu, 12 Aug 2010 09:00:19 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|