blanchet [Tue, 17 Sep 2013 01:11:37 +0200] rev 53679
merge
blanchet [Tue, 17 Sep 2013 01:09:51 +0200] rev 53678
return right theorems
blanchet [Tue, 17 Sep 2013 00:48:01 +0200] rev 53677
more (co)data docs
huffman [Fri, 13 Sep 2013 14:57:20 -0700] rev 53676
tuned proofs about 'convex'
blanchet [Tue, 17 Sep 2013 00:39:51 +0200] rev 53675
more (co)data docs
wenzelm [Tue, 17 Sep 2013 00:13:20 +0200] rev 53674
tuned proofs;
wenzelm [Mon, 16 Sep 2013 23:08:02 +0200] rev 53673
treat all dummy type variables separately (in contrast to fca432074fb2);
wenzelm [Mon, 16 Sep 2013 23:04:13 +0200] rev 53672
removed dead code (see also 69d4543811d0);
wenzelm [Mon, 16 Sep 2013 19:30:33 +0200] rev 53671
merged
wenzelm [Mon, 16 Sep 2013 19:27:20 +0200] rev 53670
tuned signature;
wenzelm [Mon, 16 Sep 2013 17:42:05 +0200] rev 53669
more antiquotations -- avoid unchecked string literals;
wenzelm [Mon, 16 Sep 2013 17:18:56 +0200] rev 53668
more explicit exception pattern (NB: unqualified exceptions without arguments are in danger of becoming catch-all patterns by accident);
wenzelm [Mon, 16 Sep 2013 17:13:38 +0200] rev 53667
distinguish Proof.context vs. local_theory semantically, with corresponding naming conventions;
some notes about missing ML interface;
wenzelm [Mon, 16 Sep 2013 17:04:28 +0200] rev 53666
tuned white space;
avoid "object-oriented English";
wenzelm [Mon, 16 Sep 2013 16:50:49 +0200] rev 53665
adhoc check of ML sources, in addition to thy files already covered in Thy_Load;
wenzelm [Mon, 16 Sep 2013 16:46:52 +0200] rev 53664
proper Isabelle symbols -- no UTF8 here;
wenzelm [Mon, 16 Sep 2013 14:21:07 +0200] rev 53663
proper Cygwin mirror for Isabelle2013-1;
wenzelm [Mon, 16 Sep 2013 13:56:02 +0200] rev 53662
explicit test of quick_and_dirty, which is rarely used in practice;
wenzelm [Mon, 16 Sep 2013 13:54:58 +0200] rev 53661
updated to cygwin-20130916;
wenzelm [Mon, 16 Sep 2013 13:22:02 +0200] rev 53660
more CHECKLIST;
wenzelm [Mon, 16 Sep 2013 13:11:32 +0200] rev 53659
updated cygwin snapshot;
wenzelm [Mon, 16 Sep 2013 12:51:33 +0200] rev 53658
updated to smlnj 110.76;
wenzelm [Mon, 16 Sep 2013 12:37:54 +0200] rev 53657
prefer high-level ML_System.share_common_data, ML_System.save_state -- except for bootstrap images (RAW, Pure);
wenzelm [Mon, 16 Sep 2013 11:46:24 +0200] rev 53656
more NEWS;
panny [Mon, 16 Sep 2013 16:48:08 +0200] rev 53655
merge
panny [Mon, 16 Sep 2013 15:03:23 +0200] rev 53654
prove simp theorems for newly generated definitions
kuncar [Mon, 16 Sep 2013 15:30:20 +0200] rev 53653
example using restoring Transfer/Lifting context
kuncar [Mon, 16 Sep 2013 15:30:20 +0200] rev 53652
use lifting_forget for deregistering numeric types as a quotient type
kuncar [Mon, 16 Sep 2013 15:30:17 +0200] rev 53651
restoring Transfer/Lifting context
kuncar [Mon, 16 Sep 2013 11:54:57 +0200] rev 53650
make ML function for deleting quotients public
kuncar [Mon, 16 Sep 2013 11:54:57 +0200] rev 53649
public access to the raw transfer rules - for restoring transferring
wenzelm [Mon, 16 Sep 2013 11:22:06 +0200] rev 53648
another move to avoid sporadic kill of poly, which is presumably due to resource management on lxbroy2, lxbroy3 etc.;