Mon, 02 Dec 2013 20:31:54 +0100 |
blanchet |
generalized datatype code generation code so that it works with old-style and new-style (co)datatypes (as long as they are not local)
|
file |
diff |
annotate
|
Tue, 12 Nov 2013 13:47:24 +0100 |
blanchet |
moved 'Ctr_Sugar' further up the theory hierarchy, so that 'Datatype' can use it
|
file |
diff |
annotate
|
Sat, 25 May 2013 15:37:53 +0200 |
wenzelm |
syntax translations always depend on context;
|
file |
diff |
annotate
|
Wed, 10 Apr 2013 21:20:35 +0200 |
wenzelm |
tuned pretty layout: avoid nested Pretty.string_of, which merely happens to work with Isabelle/jEdit since formatting is delegated to Scala side;
|
file |
diff |
annotate
|
Sat, 06 Apr 2013 01:42:07 +0200 |
traytel |
disallow coercions to interfere with case translations
|
file |
diff |
annotate
|
Fri, 05 Apr 2013 22:08:42 +0200 |
traytel |
allow redundant cases in the list comprehension translation
|
file |
diff |
annotate
|
Fri, 05 Apr 2013 22:08:42 +0200 |
traytel |
special constant to prevent eta-contraction of the check-phase syntax of case translations
|
file |
diff |
annotate
|
Tue, 22 Jan 2013 14:33:45 +0100 |
traytel |
separate data used for case translation from the datatype package
|
file |
diff |
annotate
|
Tue, 22 Jan 2013 13:32:41 +0100 |
berghofe |
case translations performed in a separate check phase (with adjustments by traytel)
|
file |
diff |
annotate
|
Fri, 30 Nov 2012 22:55:02 +0100 |
wenzelm |
added 'print_inductives' command;
|
file |
diff |
annotate
|
Wed, 22 Aug 2012 22:55:41 +0200 |
wenzelm |
prefer ML_file over old uses;
|
file |
diff |
annotate
|
Thu, 19 Jul 2012 19:38:39 +0200 |
haftmann |
removed ML module DSeq which was a part of the ancient code generator (cf. 58e33a125f32)
|
file |
diff |
annotate
|
Thu, 15 Mar 2012 22:08:53 +0100 |
wenzelm |
declare command keywords via theory header, including strict checking outside Pure;
|
file |
diff |
annotate
|
Thu, 15 Mar 2012 19:02:34 +0100 |
wenzelm |
declare minor keywords via theory header;
|
file |
diff |
annotate
|
Wed, 28 Dec 2011 20:03:13 +0100 |
wenzelm |
reverted some changes for set->predicate transition, according to "hg log -u berghofe -r Isabelle2007:Isabelle2008";
|
file |
diff |
annotate
|