Fri, 12 Apr 2013 17:21:51 +0200 modifiers for classical wrappers operate on Proof.context instead of claset;
wenzelm [Fri, 12 Apr 2013 17:21:51 +0200] rev 51703
modifiers for classical wrappers operate on Proof.context instead of claset;
Fri, 12 Apr 2013 17:02:55 +0200 removed historic comments;
wenzelm [Fri, 12 Apr 2013 17:02:55 +0200] rev 51702
removed historic comments;
Fri, 12 Apr 2013 15:30:38 +0200 tuned exceptions -- avoid composing error messages in low-level situations;
wenzelm [Fri, 12 Apr 2013 15:30:38 +0200] rev 51701
tuned exceptions -- avoid composing error messages in low-level situations;
Fri, 12 Apr 2013 14:54:14 +0200 tuned signature;
wenzelm [Fri, 12 Apr 2013 14:54:14 +0200] rev 51700
tuned signature; tuned comments;
Fri, 12 Apr 2013 12:20:51 +0200 proper identifiers -- avoid crash of case translations;
wenzelm [Fri, 12 Apr 2013 12:20:51 +0200] rev 51699
proper identifiers -- avoid crash of case translations;
Fri, 12 Apr 2013 08:27:43 +0200 reduced duplication
nipkow [Fri, 12 Apr 2013 08:27:43 +0200] rev 51698
reduced duplication
Thu, 11 Apr 2013 16:58:54 +0200 do not add case translation syntax in rep_datatype compatibility mode
traytel [Thu, 11 Apr 2013 16:58:54 +0200] rev 51697
do not add case translation syntax in rep_datatype compatibility mode
Thu, 11 Apr 2013 16:39:01 +0200 run type inference on input to wrap_data
traytel [Thu, 11 Apr 2013 16:39:01 +0200] rev 51696
run type inference on input to wrap_data
Thu, 11 Apr 2013 16:03:11 +0200 installed case translations in BNF package
traytel [Thu, 11 Apr 2013 16:03:11 +0200] rev 51695
installed case translations in BNF package
Thu, 11 Apr 2013 15:10:22 +0200 tuned
nipkow [Thu, 11 Apr 2013 15:10:22 +0200] rev 51694
tuned
Wed, 10 Apr 2013 21:46:28 +0200 more antiquotations;
wenzelm [Wed, 10 Apr 2013 21:46:28 +0200] rev 51693
more antiquotations;
Wed, 10 Apr 2013 21:20:35 +0200 tuned pretty layout: avoid nested Pretty.string_of, which merely happens to work with Isabelle/jEdit since formatting is delegated to Scala side;
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;
Wed, 10 Apr 2013 20:58:01 +0200 updated keywords;
wenzelm [Wed, 10 Apr 2013 20:58:01 +0200] rev 51691
updated keywords;
Wed, 10 Apr 2013 20:06:36 +0200 merged
wenzelm [Wed, 10 Apr 2013 20:06:36 +0200] rev 51690
merged
Wed, 10 Apr 2013 19:14:47 +0200 merged
wenzelm [Wed, 10 Apr 2013 19:14:47 +0200] rev 51689
merged
Wed, 10 Apr 2013 17:27:38 +0200 obsolete -- tools should refer to proper Proof.context;
wenzelm [Wed, 10 Apr 2013 17:27:38 +0200] rev 51688
obsolete -- tools should refer to proper Proof.context;
Wed, 10 Apr 2013 17:17:16 +0200 discontinued obsolete ML antiquotation @{claset};
wenzelm [Wed, 10 Apr 2013 17:17:16 +0200] rev 51687
discontinued obsolete ML antiquotation @{claset};
Wed, 10 Apr 2013 17:02:47 +0200 added ML antiquotation @{theory_context};
wenzelm [Wed, 10 Apr 2013 17:02:47 +0200] rev 51686
added ML antiquotation @{theory_context};
Wed, 10 Apr 2013 15:30:19 +0200 more standard module name Axclass (according to file name);
wenzelm [Wed, 10 Apr 2013 15:30:19 +0200] rev 51685
more standard module name Axclass (according to file name);
Wed, 10 Apr 2013 19:52:19 +0200 made SML/NJ happy
traytel [Wed, 10 Apr 2013 19:52:19 +0200] rev 51684
made SML/NJ happy
Wed, 10 Apr 2013 18:51:21 +0200 generalize Borel-set properties from real/ereal/ordered_euclidean_spaces to order_topology and real_normed_vector
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
Wed, 10 Apr 2013 17:49:16 +0200 NEWS and CONTRIBUTORS
traytel [Wed, 10 Apr 2013 17:49:16 +0200] rev 51682
NEWS and CONTRIBUTORS
Wed, 10 Apr 2013 17:49:16 +0200 declaration attribute for case combinators
traytel [Wed, 10 Apr 2013 17:49:16 +0200] rev 51681
declaration attribute for case combinators
Tue, 09 Apr 2013 18:27:49 +0200 Handle dummy patterns in parse translation rather than check phase
berghofe [Tue, 09 Apr 2013 18:27:49 +0200] rev 51680
Handle dummy patterns in parse translation rather than check phase
Sat, 06 Apr 2013 01:42:07 +0200 disallow coercions to interfere with case translations
traytel [Sat, 06 Apr 2013 01:42:07 +0200] rev 51679
disallow coercions to interfere with case translations
Fri, 05 Apr 2013 22:08:42 +0200 allow redundant cases in the list comprehension translation
traytel [Fri, 05 Apr 2013 22:08:42 +0200] rev 51678
allow redundant cases in the list comprehension translation
Fri, 05 Apr 2013 22:08:42 +0200 recur in the expression to be matched (do not rely on repetitive execution of a check phase);
traytel [Fri, 05 Apr 2013 22:08:42 +0200] rev 51677
recur in the expression to be matched (do not rely on repetitive execution of a check phase); separate ML-interface function that is not recurring (strip_case)
Fri, 05 Apr 2013 22:08:42 +0200 tuned whitespace
traytel [Fri, 05 Apr 2013 22:08:42 +0200] rev 51676
tuned whitespace
(0) -30000 -10000 -3000 -1000 -300 -100 -50 -28 +28 +50 +100 +300 +1000 +3000 +10000 +30000 tip