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
|
Sat, 19 Sep 2009 07:38:03 +0200 |
haftmann |
inter and union are mere abbreviations for inf and sup
|
file |
diff |
annotate
|
Wed, 23 Sep 2009 12:03:47 +0200 |
haftmann |
stripped legacy ML bindings
|
file |
diff |
annotate
|
Wed, 16 Sep 2009 13:43:05 +0200 |
haftmann |
Inter and Union are mere abbreviations for Inf and Sup
|
file |
diff |
annotate
|
Mon, 06 Jul 2009 14:19:13 +0200 |
haftmann |
moved Inductive.myinv to Fun.inv; tuned
|
file |
diff |
annotate
|
Tue, 23 Jun 2009 16:27:12 +0200 |
haftmann |
tuned interfaces of datatype module
|
file |
diff |
annotate
|
Tue, 23 Jun 2009 12:09:30 +0200 |
haftmann |
uniformly capitialized names for subdirectories
|
file |
diff |
annotate
|
Fri, 19 Jun 2009 17:23:21 +0200 |
haftmann |
discontinued ancient tradition to suffix certain ML module names with "_package"
|
file |
diff |
annotate
|
Wed, 10 Jun 2009 15:04:33 +0200 |
haftmann |
separate directory for datatype package
|
file |
diff |
annotate
|
Wed, 31 Dec 2008 20:31:36 +0100 |
wenzelm |
eliminated OldTerm.add_term_free_names;
|
file |
diff |
annotate
|
Wed, 31 Dec 2008 18:53:16 +0100 |
wenzelm |
moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
|
file |
diff |
annotate
|
Wed, 07 May 2008 10:56:35 +0200 |
berghofe |
Instantiated some rules to avoid problems with HO unification.
|
file |
diff |
annotate
|
Wed, 30 Jan 2008 10:57:44 +0100 |
haftmann |
Theorem Inductive.lfp_ordinal_induct generalized to complete lattices
|
file |
diff |
annotate
|
Thu, 06 Dec 2007 15:10:09 +0100 |
haftmann |
added new primrec package
|
file |
diff |
annotate
|
Wed, 05 Dec 2007 14:15:45 +0100 |
haftmann |
simplified infrastructure for code generator operational equality
|
file |
diff |
annotate
|
Fri, 30 Nov 2007 20:13:03 +0100 |
haftmann |
adjustions to due to instance target
|
file |
diff |
annotate
|
Mon, 08 Oct 2007 22:03:25 +0200 |
haftmann |
integrated FixedPoint into Inductive
|
file |
diff |
annotate
|
Thu, 04 Oct 2007 19:54:46 +0200 |
haftmann |
tuned datatype_codegen setup
|
file |
diff |
annotate
|
Wed, 26 Sep 2007 19:17:55 +0200 |
wenzelm |
removed dead code;
|
file |
diff |
annotate
|
Tue, 25 Sep 2007 12:16:08 +0200 |
haftmann |
datatype interpretators for size and datatype_realizer
|
file |
diff |
annotate
|
Tue, 18 Sep 2007 07:46:00 +0200 |
haftmann |
introduced generic concepts for theory interpretators
|
file |
diff |
annotate
|
Tue, 18 Sep 2007 07:36:38 +0200 |
haftmann |
separated code for inductive sequences from inductive_codegen.ML
|
file |
diff |
annotate
|
Mon, 20 Aug 2007 18:10:13 +0200 |
nipkow |
Final mods for list comprehension
|
file |
diff |
annotate
|
Wed, 11 Jul 2007 10:59:23 +0200 |
berghofe |
Added new package for inductive sets.
|
file |
diff |
annotate
|
Tue, 10 Jul 2007 17:30:49 +0200 |
haftmann |
clarified import
|
file |
diff |
annotate
|
Tue, 03 Jul 2007 15:23:11 +0200 |
nipkow |
Fixed problem with patterns in lambdas
|
file |
diff |
annotate
|
Mon, 02 Jul 2007 23:14:06 +0200 |
nipkow |
Added pattern maatching for lambda abstraction
|
file |
diff |
annotate
|
Thu, 14 Jun 2007 18:33:31 +0200 |
wenzelm |
tuned proofs: avoid implicit prems;
|
file |
diff |
annotate
|
Wed, 09 May 2007 07:53:06 +0200 |
haftmann |
moved recfun_codegen.ML to Code_Generator.thy
|
file |
diff |
annotate
|
Mon, 07 May 2007 00:49:59 +0200 |
wenzelm |
simplified DataFun interfaces;
|
file |
diff |
annotate
|
Tue, 24 Apr 2007 15:18:42 +0200 |
berghofe |
Added datatype_case.
|
file |
diff |
annotate
|
Wed, 31 Jan 2007 16:05:10 +0100 |
haftmann |
dropped lemma duplicates in HOL.thy
|
file |
diff |
annotate
|
Fri, 13 Oct 2006 18:12:58 +0200 |
berghofe |
Added new package for inductive definitions, moved old package
|
file |
diff |
annotate
|
Tue, 19 Sep 2006 15:22:35 +0200 |
haftmann |
added auxiliary lemma for code generation 2
|
file |
diff |
annotate
|
Tue, 09 May 2006 10:09:37 +0200 |
haftmann |
added DatatypeHooks
|
file |
diff |
annotate
|
Thu, 22 Dec 2005 00:28:34 +0100 |
wenzelm |
updated auxiliary facts for induct method;
|
file |
diff |
annotate
|
Wed, 03 Aug 2005 14:48:13 +0200 |
avigad |
import FixedPoint instead of Gfp
|
file |
diff |
annotate
|
Fri, 17 Jun 2005 16:12:49 +0200 |
haftmann |
migrated theory headers to new format
|
file |
diff |
annotate
|
Wed, 18 Aug 2004 11:09:40 +0200 |
nipkow |
import -> imports
|
file |
diff |
annotate
|
Mon, 16 Aug 2004 14:22:27 +0200 |
nipkow |
New theory header syntax.
|
file |
diff |
annotate
|
Mon, 21 Jun 2004 10:25:57 +0200 |
kleing |
Merged in license change from Isabelle2004
|
file |
diff |
annotate
|
Wed, 13 Nov 2002 15:25:17 +0100 |
berghofe |
Added InductiveRealizer package.
|
file |
diff |
annotate
|
Wed, 07 Aug 2002 16:48:20 +0200 |
berghofe |
Added file Tools/datatype_realizer.ML
|
file |
diff |
annotate
|
Thu, 21 Feb 2002 20:09:48 +0100 |
wenzelm |
include theory Record (tuned dependencies);
|
file |
diff |
annotate
|
Mon, 10 Dec 2001 15:17:49 +0100 |
berghofe |
Moved code generator setup from Recdef to Inductive.
|
file |
diff |
annotate
|
Sat, 03 Nov 2001 01:33:54 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Wed, 31 Oct 2001 01:21:01 +0100 |
wenzelm |
use induct_rulify2;
|
file |
diff |
annotate
|
Thu, 18 Oct 2001 20:59:59 +0200 |
wenzelm |
moved InductMethod.setup to theory HOL;
|
file |
diff |
annotate
|
Thu, 04 Oct 2001 15:43:17 +0200 |
wenzelm |
generic induct_method.ML;
|
file |
diff |
annotate
|
Sun, 22 Jul 2001 21:30:21 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Fri, 20 Jul 2001 22:00:06 +0200 |
wenzelm |
private "myinv" (uses "The" instead of "Eps");
|
file |
diff |
annotate
|
Tue, 22 May 2001 15:10:06 +0200 |
berghofe |
Inductive definitions are now introduced earlier in the theory hierarchy.
|
file |
diff |
annotate
|
Tue, 30 Jan 2001 18:57:24 +0100 |
oheimb |
added if_def2
|
file |
diff |
annotate
|
Fri, 22 Dec 2000 18:23:41 +0100 |
wenzelm |
added inductive_conj;
|
file |
diff |
annotate
|
Fri, 10 Nov 2000 19:03:55 +0100 |
wenzelm |
simplified atomize;
|
file |
diff |
annotate
|
Mon, 06 Nov 2000 22:49:16 +0100 |
wenzelm |
inductive_atomize, inductive_rulify;
|
file |
diff |
annotate
|
Mon, 23 Oct 2000 22:12:04 +0200 |
wenzelm |
declare trancl rules;
|
file |
diff |
annotate
|
Thu, 12 Oct 2000 18:38:23 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Wed, 15 Mar 2000 23:41:42 +0100 |
berghofe |
Added setup for primrec theory data.
|
file |
diff |
annotate
|
Sat, 04 Mar 2000 13:25:09 +0100 |
wenzelm |
require NatDef;
|
file |
diff |
annotate
|
Sun, 27 Feb 2000 15:23:28 +0100 |
wenzelm |
early setup of induct_method;
|
file |
diff |
annotate
|