wenzelm [Wed, 10 Apr 2013 21:46:28 +0200] rev 51693
more antiquotations;
wenzelm [Wed, 10 Apr 2013 21:20:35 +0200] rev 51692
tuned pretty layout: avoid nested Pretty.string_of, which merely happens to work with Isabelle/jEdit since formatting is delegated to Scala side;
declare command "print_case_translations" where it is actually defined;
wenzelm [Wed, 10 Apr 2013 20:58:01 +0200] rev 51691
updated keywords;
wenzelm [Wed, 10 Apr 2013 20:06:36 +0200] rev 51690
merged
wenzelm [Wed, 10 Apr 2013 19:14:47 +0200] rev 51689
merged
wenzelm [Wed, 10 Apr 2013 17:27:38 +0200] rev 51688
obsolete -- tools should refer to proper Proof.context;
wenzelm [Wed, 10 Apr 2013 17:17:16 +0200] rev 51687
discontinued obsolete ML antiquotation @{claset};
wenzelm [Wed, 10 Apr 2013 17:02:47 +0200] rev 51686
added ML antiquotation @{theory_context};
wenzelm [Wed, 10 Apr 2013 15:30:19 +0200] rev 51685
more standard module name Axclass (according to file name);
traytel [Wed, 10 Apr 2013 19:52:19 +0200] rev 51684
made SML/NJ happy
hoelzl [Wed, 10 Apr 2013 18:51:21 +0200] rev 51683
generalize Borel-set properties from real/ereal/ordered_euclidean_spaces to order_topology and real_normed_vector
traytel [Wed, 10 Apr 2013 17:49:16 +0200] rev 51682
NEWS and CONTRIBUTORS
traytel [Wed, 10 Apr 2013 17:49:16 +0200] rev 51681
declaration attribute for case combinators
berghofe [Tue, 09 Apr 2013 18:27:49 +0200] rev 51680
Handle dummy patterns in parse translation rather than check phase
traytel [Sat, 06 Apr 2013 01:42:07 +0200] rev 51679
disallow coercions to interfere with case translations
traytel [Fri, 05 Apr 2013 22:08:42 +0200] rev 51678
allow redundant cases in the list comprehension translation