src/HOL/HOLCF/Cfun.thy
Sat, 25 May 2013 15:37:53 +0200 syntax translations always depend on context;
Thu, 18 Apr 2013 17:07:01 +0200 simplifier uses proper Proof.context instead of historic type simpset;
Tue, 09 Oct 2012 17:33:46 +0200 removed support for set constant definitions in HOLCF {cpo,pcpo,domain}def commands;
Wed, 30 Nov 2011 17:30:01 +0100 prefer cpodef without extra definition;
Sun, 20 Nov 2011 21:07:06 +0100 eliminated obsolete "standard";
Fri, 08 Apr 2011 13:31:16 +0200 explicit structure Syntax_Trans;
Wed, 06 Apr 2011 23:04:00 +0200 separate structure Term_Position;
Tue, 05 Apr 2011 14:25:18 +0200 discontinued special treatment of structure Ast: no pervasive content, no inclusion in structure Syntax;
Tue, 29 Mar 2011 17:47:11 +0200 tuned headers;
Tue, 22 Mar 2011 20:44:47 +0100 more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
Tue, 22 Mar 2011 18:03:28 +0100 enable inner syntax source positions by default (controlled via configuration option);
Sat, 08 Jan 2011 11:18:09 -0800 use proper syntactic types for 'syntax' commands
Sat, 08 Jan 2011 10:02:43 -0800 make print translation for Abs_cfun consistent with other binders: prevent eta-contraction, but don't force eta-expansion
Tue, 04 Jan 2011 15:32:56 -0800 change some lemma names containing 'UU' to 'bottom'
Thu, 23 Dec 2010 11:52:26 -0800 replaced separate lemmas seq{1,2,3} with seq_simps
Mon, 20 Dec 2010 09:41:55 -0800 beta-reduction simproc uses lemma Abs_cfun_inverse2 instead of beta_cfun, to be more robust against eta-contraction
Mon, 06 Dec 2010 11:22:42 -0800 remove lemma cont_cfun;
Mon, 06 Dec 2010 10:08:33 -0800 rename lub_fun -> is_lub_fun, thelub_fun -> lub_fun
Mon, 06 Dec 2010 08:30:00 -0800 add lemmas lub_APP, lub_LAM
Tue, 30 Nov 2010 15:56:19 -0800 change cpodef-generated cont_Rep rules to cont2cont format
Sat, 27 Nov 2010 22:48:08 -0800 add lemma cont2cont_if_bottom
Sat, 27 Nov 2010 16:08:10 -0800 moved directory src/HOLCF to src/HOL/HOLCF;