blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49682
removed dead params and dead code
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49681
changed type of corecursor for the nested recursion case
blanchet [Tue, 02 Oct 2012 01:00:18 +0200] rev 49680
made (co)rec tactic more robust when the simplifier succeeds early
wenzelm [Mon, 01 Oct 2012 20:38:57 +0200] rev 49679
tuned;
wenzelm [Mon, 01 Oct 2012 20:35:09 +0200] rev 49678
removed unused module Blob;
wenzelm [Mon, 01 Oct 2012 20:17:30 +0200] rev 49677
more direct message header: eliminated historic encoding via single letter;
wenzelm [Mon, 01 Oct 2012 20:16:37 +0200] rev 49676
tuned whitespace;
wenzelm [Mon, 01 Oct 2012 17:29:00 +0200] rev 49675
tuned proofs;
wenzelm [Mon, 01 Oct 2012 16:37:22 +0200] rev 49674
report sort assignment of visible type variables;
wenzelm [Mon, 01 Oct 2012 12:05:05 +0200] rev 49673
more robust File.eq, and thus File.copy of "~~/lib/logo/isabelle.gif";
blanchet [Mon, 01 Oct 2012 11:04:30 +0200] rev 49672
fixed recursor definition for datatypes with inner products (e.g. "'a trm" from the lambda-term example)
blanchet [Mon, 01 Oct 2012 10:46:30 +0200] rev 49671
tweaked corecursor/coiterator tactic
blanchet [Mon, 01 Oct 2012 10:34:58 +0200] rev 49670
changed the type of the recursor for nested recursion
blanchet [Sun, 30 Sep 2012 23:45:03 +0200] rev 49669
fixed quick-and-dirty mode
blanchet [Sun, 30 Sep 2012 22:02:34 +0200] rev 49668
tuning
traytel [Sun, 30 Sep 2012 12:08:16 +0200] rev 49667
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
traytel [Sun, 30 Sep 2012 12:04:47 +0200] rev 49666
got rid of subst_tac alias
traytel [Sun, 30 Sep 2012 12:04:13 +0200] rev 49665
tuned tactic
wenzelm [Sat, 29 Sep 2012 21:59:08 +0200] rev 49664
tuned proofs;
wenzelm [Sat, 29 Sep 2012 21:24:20 +0200] rev 49663
tuned proofs;
wenzelm [Sat, 29 Sep 2012 20:13:50 +0200] rev 49662
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm [Sat, 29 Sep 2012 19:28:03 +0200] rev 49661
enable show_markup by default (approx. double output size);
wenzelm [Sat, 29 Sep 2012 18:23:46 +0200] rev 49660
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm [Sat, 29 Sep 2012 16:51:04 +0200] rev 49659
explicit show_types takes preferenced over show_markup;
wenzelm [Sat, 29 Sep 2012 16:35:31 +0200] rev 49658
ignore wrapped markup elements in Proof General;
wenzelm [Sat, 29 Sep 2012 16:17:46 +0200] rev 49657
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
proper recursion in standard_format;
wenzelm [Sat, 29 Sep 2012 16:15:18 +0200] rev 49656
treat wrapped markup elements as raw markup delimiters;
wenzelm [Sat, 29 Sep 2012 13:43:23 +0200] rev 49655
tuned signature;