Mon, 01 Oct 2012 17:29:00 +0200 wenzelm tuned proofs;
Mon, 01 Oct 2012 16:37:22 +0200 wenzelm report sort assignment of visible type variables;
Mon, 01 Oct 2012 12:05:05 +0200 wenzelm more robust File.eq, and thus File.copy of "~~/lib/logo/isabelle.gif";
Mon, 01 Oct 2012 11:04:30 +0200 blanchet fixed recursor definition for datatypes with inner products (e.g. "'a trm" from the lambda-term example)
Mon, 01 Oct 2012 10:46:30 +0200 blanchet tweaked corecursor/coiterator tactic
Mon, 01 Oct 2012 10:34:58 +0200 blanchet changed the type of the recursor for nested recursion
Sun, 30 Sep 2012 23:45:03 +0200 blanchet fixed quick-and-dirty mode
Sun, 30 Sep 2012 22:02:34 +0200 blanchet tuning
Sun, 30 Sep 2012 12:08:16 +0200 traytel use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
Sun, 30 Sep 2012 12:04:47 +0200 traytel got rid of subst_tac alias
Sun, 30 Sep 2012 12:04:13 +0200 traytel tuned tactic
Sat, 29 Sep 2012 21:59:08 +0200 wenzelm tuned proofs;
Sat, 29 Sep 2012 21:24:20 +0200 wenzelm tuned proofs;
Sat, 29 Sep 2012 20:13:50 +0200 wenzelm proper handling of constraints stemming from idtyp_ast_tr';
Sat, 29 Sep 2012 19:28:03 +0200 wenzelm enable show_markup by default (approx. double output size);
Sat, 29 Sep 2012 18:23:46 +0200 wenzelm more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
Sat, 29 Sep 2012 16:51:04 +0200 wenzelm explicit show_types takes preferenced over show_markup;
Sat, 29 Sep 2012 16:35:31 +0200 wenzelm ignore wrapped markup elements in Proof General;
Sat, 29 Sep 2012 16:17:46 +0200 wenzelm turn constraints into Isabelle_Markup.typing, depending on show_markup options;
Sat, 29 Sep 2012 16:15:18 +0200 wenzelm treat wrapped markup elements as raw markup delimiters;
Sat, 29 Sep 2012 13:43:23 +0200 wenzelm tuned signature;
Fri, 28 Sep 2012 23:45:15 +0200 wenzelm tuned proofs;
Fri, 28 Sep 2012 23:40:48 +0200 wenzelm tuned proofs;
Fri, 28 Sep 2012 23:02:49 +0200 wenzelm tuned proofs;
Fri, 28 Sep 2012 23:02:39 +0200 wenzelm tuned;
Fri, 28 Sep 2012 22:53:18 +0200 wenzelm support for wrapped XML elements, which allows to preserve full markup tree information in to_XML/from_XML conversion;
Fri, 28 Sep 2012 17:06:07 +0200 wenzelm merged
Fri, 28 Sep 2012 16:59:53 +0200 wenzelm eliminated dead code;
Fri, 28 Sep 2012 16:51:58 +0200 wenzelm smarter handling of tracing messages;
Fri, 28 Sep 2012 15:45:03 +0200 wenzelm display number of tracing messages;
Fri, 28 Sep 2012 15:25:49 +0200 wenzelm tuned signature;
Fri, 28 Sep 2012 15:05:16 +0200 wenzelm tuned proofs;
Fri, 28 Sep 2012 15:23:32 +0200 blanchet simplified simpset
Fri, 28 Sep 2012 15:14:11 +0200 blanchet fixed simplification of prod and sum relators to avoid issues with e.g. codata ('a, 'b) k = K "'a + 'b"
Fri, 28 Sep 2012 13:16:10 +0200 traytel tuned tactic
Fri, 28 Sep 2012 11:46:57 +0200 wenzelm updated keywords using proper "isabelle update_keywords";
Fri, 28 Sep 2012 11:31:51 +0200 traytel tuned tactic
Fri, 28 Sep 2012 09:38:07 +0200 traytel tuned tactic
Fri, 28 Sep 2012 09:21:27 +0200 blanchet merge
Fri, 28 Sep 2012 09:12:50 +0200 blanchet renamed ML file in preparation for next step
Fri, 28 Sep 2012 09:12:50 +0200 blanchet killed temporary "data_raw" and "codata_raw" now that the examples have been ported to "data" and "codata"
Fri, 28 Sep 2012 09:12:50 +0200 blanchet modernized example, exploiting "rep_compat" option
Fri, 28 Sep 2012 09:12:50 +0200 blanchet compatibility option to use "rep_datatype"
Fri, 28 Sep 2012 09:12:50 +0200 blanchet tuned message
Fri, 28 Sep 2012 09:12:49 +0200 blanchet modernized example
Fri, 28 Sep 2012 09:17:30 +0200 traytel tuned tactics
Fri, 28 Sep 2012 08:59:54 +0200 nipkow second usage of const_typ
Fri, 28 Sep 2012 08:39:48 +0200 nipkow new antiquotation const_typ
Fri, 28 Sep 2012 08:09:28 +0200 nipkow tuned printing of _ in latex
Thu, 27 Sep 2012 20:30:32 +0200 kuncar mk_readable_rsp_thm_eq is more robust now
Thu, 27 Sep 2012 20:30:30 +0200 kuncar new get function for non-symmetric relator_eq & tuned
Thu, 27 Sep 2012 19:35:29 +0200 wenzelm merged
Thu, 27 Sep 2012 18:58:15 +0200 traytel tuned tactic; got rid of substs_tac alias
Thu, 27 Sep 2012 18:39:17 +0200 blanchet use a nicer scheme to indexify names
Thu, 27 Sep 2012 18:25:41 +0200 traytel tuned tactic
Thu, 27 Sep 2012 18:01:33 +0200 traytel type of the bound of a BNF depends at most on dead type variables
Thu, 27 Sep 2012 17:54:35 +0200 blanchet repaired signature
Thu, 27 Sep 2012 17:00:54 +0200 blanchet lower the defaults for the number of bits, based on an example by Lukas Bulwahn
Thu, 27 Sep 2012 17:00:54 +0200 blanchet modernized examples
Thu, 27 Sep 2012 12:08:38 +0200 nipkow merged
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip