| Sat, 01 Oct 2016 19:29:48 +0200 | 
wenzelm | 
tuned proofs;
 | 
file |
diff |
annotate
 | 
| Sat, 01 Oct 2016 17:38:14 +0200 | 
wenzelm | 
Isar proof of Schroeder_Bernstein without using Hilbert_Choice (and metis);
 | 
file |
diff |
annotate
 | 
| Sat, 01 Oct 2016 17:16:35 +0200 | 
wenzelm | 
clarified lfp/gfp statements and proofs;
 | 
file |
diff |
annotate
 | 
| Sat, 01 Oct 2016 11:14:00 +0200 | 
wenzelm | 
added lemma;
 | 
file |
diff |
annotate
 | 
| Tue, 13 Sep 2016 20:51:14 +0200 | 
traytel | 
don't expose internal construction in the coinduction rule for mutual coinductive predicates
 | 
file |
diff |
annotate
 | 
| Tue, 02 Aug 2016 21:05:34 +0200 | 
wenzelm | 
misc tuning and modernization;
 | 
file |
diff |
annotate
 | 
| Fri, 29 Jul 2016 09:49:23 +0200 | 
Andreas Lochbihler | 
add lemmas contributed by Peter Gammie
 | 
file |
diff |
annotate
 | 
| Fri, 22 Jul 2016 11:00:43 +0200 | 
wenzelm | 
tuned proofs -- avoid unstructured calculation;
 | 
file |
diff |
annotate
 | 
| Tue, 05 Jul 2016 23:39:49 +0200 | 
wenzelm | 
misc tuning and modernization;
 | 
file |
diff |
annotate
 | 
| Mon, 28 Dec 2015 21:47:32 +0100 | 
wenzelm | 
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
 | 
file |
diff |
annotate
 | 
| Mon, 28 Dec 2015 17:43:30 +0100 | 
wenzelm | 
prefer symbols for "Union", "Inter";
 | 
file |
diff |
annotate
 | 
| Mon, 07 Dec 2015 10:38:04 +0100 | 
wenzelm | 
isabelle update_cartouches -c -t;
 | 
file |
diff |
annotate
 | 
| Tue, 06 Oct 2015 15:14:28 +0200 | 
wenzelm | 
fewer aliases for toplevel theorem statements;
 | 
file |
diff |
annotate
 | 
| Tue, 01 Sep 2015 22:32:58 +0200 | 
wenzelm | 
eliminated \<Colon>;
 | 
file |
diff |
annotate
 | 
| Sat, 18 Jul 2015 22:58:50 +0200 | 
wenzelm | 
isabelle update_cartouches;
 | 
file |
diff |
annotate
 | 
| Fri, 03 Jul 2015 08:26:34 +0200 | 
hoelzl | 
add named theorems order_continuous_intros; lfp/gfp_funpow; bounded variant for lfp/gfp transfer
 | 
file |
diff |
annotate
 | 
| Mon, 04 May 2015 18:49:51 +0200 | 
hoelzl | 
strengthened lfp_ordinal_induct; added dual gfp variant
 | 
file |
diff |
annotate
 | 
| Mon, 04 May 2015 18:04:01 +0200 | 
hoelzl | 
add rules for least/greatest fixed point calculus
 | 
file |
diff |
annotate
 | 
| Sun, 02 Nov 2014 18:21:45 +0100 | 
wenzelm | 
modernized header uniformly as section;
 | 
file |
diff |
annotate
 | 
| Wed, 29 Oct 2014 11:41:54 +0100 | 
wenzelm | 
modernized setup;
 | 
file |
diff |
annotate
 | 
| Thu, 11 Sep 2014 18:54:36 +0200 | 
blanchet | 
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
 | 
file |
diff |
annotate
 | 
| Fri, 05 Sep 2014 00:41:01 +0200 | 
blanchet | 
fixed infinite loops in 'register' functions + more uniform API
 | 
file |
diff |
annotate
 | 
| Mon, 01 Sep 2014 16:17:46 +0200 | 
blanchet | 
renamed modules defining old datatypes, as a step towards having 'datatype_new' take 'datatype's place
 | 
file |
diff |
annotate
 | 
| Fri, 14 Mar 2014 15:41:29 +0100 | 
wenzelm | 
discontinued somewhat pointless "thy_script" keyword kind;
 | 
file |
diff |
annotate
 | 
| Thu, 20 Feb 2014 15:14:37 +0100 | 
noschinl | 
less flex-flex pairs
 | 
file |
diff |
annotate
 | 
| Wed, 19 Feb 2014 08:34:33 +0100 | 
blanchet | 
moved 'primrec' up (for real this time) and removed temporary 'old_primrec'
 | 
file |
diff |
annotate
 | 
| Mon, 17 Feb 2014 13:31:42 +0100 | 
blanchet | 
renamed old 'primrec' to 'old_primrec' (until the new 'primrec' can be moved above 'Nat' in the theory dependencies)
 | 
file |
diff |
annotate
 | 
| 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
 | 
| Sat, 17 Dec 2011 12:42:10 +0100 | 
wenzelm | 
clarified modules that contribute to datatype package;
 | 
file |
diff |
annotate
 | 
| Fri, 16 Dec 2011 12:03:33 +0100 | 
wenzelm | 
prefer Name.context operations;
 | 
file |
diff |
annotate
 | 
| Fri, 16 Dec 2011 10:52:35 +0100 | 
wenzelm | 
clarified modules that contribute to datatype package;
 | 
file |
diff |
annotate
 | 
| Thu, 15 Dec 2011 18:08:40 +0100 | 
wenzelm | 
clarified module dependencies: Datatype_Data, Datatype_Case, Rep_Datatype;
 | 
file |
diff |
annotate
 | 
| Thu, 15 Dec 2011 17:37:14 +0100 | 
wenzelm | 
separate rep_datatype.ML;
 | 
file |
diff |
annotate
 | 
| Sat, 10 Sep 2011 10:29:24 +0200 | 
haftmann | 
renamed theory Complete_Lattice to Complete_Lattices, in accordance with Lattices, Orderings etc.
 | 
file |
diff |
annotate
 | 
| Mon, 27 Jun 2011 17:04:04 +0200 | 
krauss | 
new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
 | 
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
 | 
| Wed, 08 Dec 2010 14:52:23 +0100 | 
haftmann | 
tuned
 | 
file |
diff |
annotate
 | 
| Tue, 28 Sep 2010 15:39:59 +0200 | 
haftmann | 
dropped old primrec package
 | 
file |
diff |
annotate
 | 
| Thu, 10 Jun 2010 12:24:02 +0200 | 
haftmann | 
moved inductive_codegen to place where product type is available; tuned structure name
 | 
file |
diff |
annotate
 | 
| Thu, 11 Feb 2010 23:00:22 +0100 | 
wenzelm | 
modernized translations;
 | 
file |
diff |
annotate
 | 
| Mon, 30 Nov 2009 11:42:49 +0100 | 
haftmann | 
modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML
 | 
file |
diff |
annotate
 | 
| Mon, 30 Nov 2009 08:08:31 +0100 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 | 
| Fri, 27 Nov 2009 08:41:10 +0100 | 
haftmann | 
renamed former datatype.ML to datatype_data.ML; datatype.ML provides uniform view on datatype.ML and datatype_rep_proofs.ML
 | 
file |
diff |
annotate
 | 
| Wed, 25 Nov 2009 11:16:57 +0100 | 
haftmann | 
bootstrap datatype_rep_proofs in Datatype.thy (avoids unchecked dynamic name references)
 | 
file |
diff |
annotate
 | 
| Fri, 27 Nov 2009 16:26:04 +0100 | 
berghofe | 
Streamlined setup for monotonicity rules (no longer requires classical rules).
 | 
file |
diff |
annotate
 | 
| Wed, 23 Sep 2009 14:00:43 +0200 | 
haftmann | 
merged
 | 
file |
diff |
annotate
 |