| Sat, 12 Mar 2016 22:04:52 +0100 | 
haftmann | 
model characters directly as range 0..255
 | 
file |
diff |
annotate
 | 
| Thu, 18 Feb 2016 17:52:52 +0100 | 
haftmann | 
more direct bootstrap of char type, still retaining the nibble representation for syntax
 | 
file |
diff |
annotate
 | 
| Thu, 05 Nov 2015 10:39:49 +0100 | 
wenzelm | 
isabelle update_cartouches -c -t;
 | 
file |
diff |
annotate
 | 
| Tue, 01 Sep 2015 22:32:58 +0200 | 
wenzelm | 
eliminated \<Colon>;
 | 
file |
diff |
annotate
 | 
| Wed, 17 Jun 2015 11:03:05 +0200 | 
wenzelm | 
isabelle update_cartouches;
 | 
file |
diff |
annotate
 | 
| Sun, 02 Nov 2014 17:20:45 +0100 | 
wenzelm | 
modernized header;
 | 
file |
diff |
annotate
 | 
| Mon, 30 Jun 2014 08:00:36 +0200 | 
haftmann | 
qualified String.explode and String.implode
 | 
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, 27 Nov 2013 10:54:44 +0100 | 
Andreas Lochbihler | 
revert 4af7c82463d3 and document type class problem in Haskell
 | 
file |
diff |
annotate
 | 
| Wed, 20 Nov 2013 11:59:33 +0100 | 
Andreas Lochbihler | 
implement comparisons on String.literal by target-language comparisons
 | 
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, 26 Mar 2013 20:02:02 +0100 | 
wenzelm | 
tuned imports;
 | 
file |
diff |
annotate
 | 
| Fri, 15 Feb 2013 11:47:33 +0100 | 
haftmann | 
systematic conversions between nat and nibble/char;
 | 
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
 | 
| Mon, 02 May 2011 10:50:07 +0200 | 
bulwahn | 
adding code generation setup for String.implode and String.explode in OCaml (contributed by Andreas Lochbihler)
 | 
file |
diff |
annotate
 | 
| Fri, 08 Apr 2011 16:31:14 +0200 | 
bulwahn | 
deactivating other compilations in quickcheck_exhaustive momentarily that only interesting for my benchmarks and experiments
 | 
file |
diff |
annotate
 | 
| Tue, 05 Apr 2011 09:38:28 +0200 | 
bulwahn | 
removing bounded_forall code equation for characters when loading Code_Char
 | 
file |
diff |
annotate
 | 
| Fri, 10 Sep 2010 10:21:25 +0200 | 
haftmann | 
Haskell == is infix, not infixl
 | 
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
 | 
| Fri, 27 Aug 2010 19:34:23 +0200 | 
haftmann | 
renamed class/constant eq to equal; tuned some instantiations
 | 
file |
diff |
annotate
 | 
| Fri, 18 Jun 2010 15:03:20 +0200 | 
haftmann | 
avoid Scala legacy operations
 | 
file |
diff |
annotate
 | 
| Tue, 01 Jun 2010 10:30:53 +0200 | 
haftmann | 
added Scala code setup
 | 
file |
diff |
annotate
 | 
| Tue, 27 Oct 2009 15:32:20 +0100 | 
haftmann | 
added implode and explode
 | 
file |
diff |
annotate
 | 
| Wed, 23 Sep 2009 14:00:12 +0200 | 
haftmann | 
Code_Eval(uation)
 | 
file |
diff |
annotate
 | 
| Wed, 06 May 2009 19:09:14 +0200 | 
haftmann | 
confine term setup to Eval serialiser
 | 
file |
diff |
annotate
 | 
| Wed, 06 May 2009 16:01:05 +0200 | 
haftmann | 
confine term setup to Eval serialiser
 | 
file |
diff |
annotate
 | 
| Mon, 23 Mar 2009 08:14:24 +0100 | 
haftmann | 
Main is (Complex_Main) base entry point in library theories
 | 
file |
diff |
annotate
 | 
| Fri, 20 Feb 2009 10:14:31 +0100 | 
haftmann | 
dropped Id
 | 
file |
diff |
annotate
 | 
| Thu, 25 Sep 2008 09:28:03 +0200 | 
haftmann | 
discontinued special treatment of op = vs. eq_class.eq
 | 
file |
diff |
annotate
 | 
| Tue, 16 Sep 2008 16:13:09 +0200 | 
haftmann | 
a sophisticated char/nibble conversion combinator
 | 
file |
diff |
annotate
 | 
| Tue, 16 Sep 2008 09:21:24 +0200 | 
haftmann | 
evaluation using code generator
 | 
file |
diff |
annotate
 | 
| Tue, 02 Sep 2008 20:38:17 +0200 | 
haftmann | 
distributed literal code generation out of central infrastructure
 | 
file |
diff |
annotate
 | 
| Mon, 01 Sep 2008 10:18:37 +0200 | 
haftmann | 
restructured code generation of literals
 | 
file |
diff |
annotate
 | 
| Thu, 28 Aug 2008 22:09:20 +0200 | 
haftmann | 
restructured and split code serializer module
 | 
file |
diff |
annotate
 | 
| Mon, 07 Jul 2008 08:47:17 +0200 | 
haftmann | 
absolute imports of HOL/*.thy theories
 | 
file |
diff |
annotate
 | 
| Thu, 26 Jun 2008 10:07:01 +0200 | 
haftmann | 
established Plain theory and image
 | 
file |
diff |
annotate
 | 
| Fri, 25 Jan 2008 14:54:41 +0100 | 
haftmann | 
improved code theorem setup
 | 
file |
diff |
annotate
 | 
| Fri, 12 Oct 2007 10:26:18 +0200 | 
haftmann | 
added
 | 
file |
diff |
annotate
 |