Thu, 18 Apr 2013 21:31:24 +0200 merged
wenzelm [Thu, 18 Apr 2013 21:31:24 +0200] rev 51719
merged
Thu, 18 Apr 2013 21:10:12 +0200 tuned signature;
wenzelm [Thu, 18 Apr 2013 21:10:12 +0200] rev 51718
tuned signature;
Thu, 18 Apr 2013 17:07:01 +0200 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm [Thu, 18 Apr 2013 17:07:01 +0200] rev 51717
simplifier uses proper Proof.context instead of historic type simpset;
Thu, 18 Apr 2013 20:18:50 +0200 merged
nipkow [Thu, 18 Apr 2013 20:18:50 +0200] rev 51716
merged
Thu, 18 Apr 2013 20:18:37 +0200 avoided map_of in def of fun_rep (but still needed for efficient code)
nipkow [Thu, 18 Apr 2013 20:18:37 +0200] rev 51715
avoided map_of in def of fun_rep (but still needed for efficient code)
Thu, 18 Apr 2013 18:57:02 +0200 spelling
haftmann [Thu, 18 Apr 2013 18:57:02 +0200] rev 51714
spelling
Thu, 18 Apr 2013 18:55:23 +0200 spelling
haftmann [Thu, 18 Apr 2013 18:55:23 +0200] rev 51713
spelling
Wed, 17 Apr 2013 21:23:35 +0200 tuned
nipkow [Wed, 17 Apr 2013 21:23:35 +0200] rev 51712
tuned
Wed, 17 Apr 2013 21:11:01 +0200 complete revision: finally got rid of annoying L-predicate
nipkow [Wed, 17 Apr 2013 21:11:01 +0200] rev 51711
complete revision: finally got rid of annoying L-predicate
Wed, 17 Apr 2013 20:53:26 +0200 moved leastness lemma
nipkow [Wed, 17 Apr 2013 20:53:26 +0200] rev 51710
moved leastness lemma
Tue, 16 Apr 2013 17:54:14 +0200 proper prolog command-line instead of hashbang, which might switch to invalid executable and thus fail (notably on lxbroy2);
wenzelm [Tue, 16 Apr 2013 17:54:14 +0200] rev 51709
proper prolog command-line instead of hashbang, which might switch to invalid executable and thus fail (notably on lxbroy2); speculative update for yap (untested);
Mon, 15 Apr 2013 22:51:55 +0200 use automatic type coerctions in Sqrt example
hoelzl [Mon, 15 Apr 2013 22:51:55 +0200] rev 51708
use automatic type coerctions in Sqrt example
Mon, 15 Apr 2013 12:03:16 +0200 make SML/NJ happy;
wenzelm [Mon, 15 Apr 2013 12:03:16 +0200] rev 51707
make SML/NJ happy;
Mon, 15 Apr 2013 10:41:03 +0200 not all Nitpick 'constructors' are injective -- careful
blanchet [Mon, 15 Apr 2013 10:41:03 +0200] rev 51706
not all Nitpick 'constructors' are injective -- careful
Sun, 14 Apr 2013 21:54:45 +1000 added another definition snipped
kleing [Sun, 14 Apr 2013 21:54:45 +1000] rev 51705
added another definition snipped
Fri, 12 Apr 2013 17:56:51 +0200 actually fail on prolog errors -- such as swipl startup failure due to missing shared libraries -- assuming it normally produces clean return code 0;
wenzelm [Fri, 12 Apr 2013 17:56:51 +0200] rev 51704
actually fail on prolog errors -- such as swipl startup failure due to missing shared libraries -- assuming it normally produces clean return code 0;
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;
(0) -30000 -10000 -3000 -1000 -300 -100 -50 -28 +28 +50 +100 +300 +1000 +3000 +10000 +30000 tip