Thu, 18 Apr 2013 20:18:50 +0200 nipkow merged
Thu, 18 Apr 2013 20:18:37 +0200 nipkow avoided map_of in def of fun_rep (but still needed for efficient code)
Thu, 18 Apr 2013 18:57:02 +0200 haftmann spelling
Thu, 18 Apr 2013 18:55:23 +0200 haftmann spelling
Wed, 17 Apr 2013 21:23:35 +0200 nipkow tuned
Wed, 17 Apr 2013 21:11:01 +0200 nipkow complete revision: finally got rid of annoying L-predicate
Wed, 17 Apr 2013 20:53:26 +0200 nipkow moved leastness lemma
Tue, 16 Apr 2013 17:54:14 +0200 wenzelm proper prolog command-line instead of hashbang, which might switch to invalid executable and thus fail (notably on lxbroy2);
Mon, 15 Apr 2013 22:51:55 +0200 hoelzl use automatic type coerctions in Sqrt example
Mon, 15 Apr 2013 12:03:16 +0200 wenzelm make SML/NJ happy;
Mon, 15 Apr 2013 10:41:03 +0200 blanchet not all Nitpick 'constructors' are injective -- careful
Sun, 14 Apr 2013 21:54:45 +1000 kleing added another definition snipped
Fri, 12 Apr 2013 17:56:51 +0200 wenzelm 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 wenzelm modifiers for classical wrappers operate on Proof.context instead of claset;
Fri, 12 Apr 2013 17:02:55 +0200 wenzelm removed historic comments;
Fri, 12 Apr 2013 15:30:38 +0200 wenzelm tuned exceptions -- avoid composing error messages in low-level situations;
Fri, 12 Apr 2013 14:54:14 +0200 wenzelm tuned signature;
Fri, 12 Apr 2013 12:20:51 +0200 wenzelm proper identifiers -- avoid crash of case translations;
Fri, 12 Apr 2013 08:27:43 +0200 nipkow reduced duplication
Thu, 11 Apr 2013 16:58:54 +0200 traytel do not add case translation syntax in rep_datatype compatibility mode
Thu, 11 Apr 2013 16:39:01 +0200 traytel run type inference on input to wrap_data
Thu, 11 Apr 2013 16:03:11 +0200 traytel installed case translations in BNF package
Thu, 11 Apr 2013 15:10:22 +0200 nipkow tuned
Wed, 10 Apr 2013 21:46:28 +0200 wenzelm more antiquotations;
Wed, 10 Apr 2013 21:20:35 +0200 wenzelm tuned pretty layout: avoid nested Pretty.string_of, which merely happens to work with Isabelle/jEdit since formatting is delegated to Scala side;
Wed, 10 Apr 2013 20:58:01 +0200 wenzelm updated keywords;
Wed, 10 Apr 2013 20:06:36 +0200 wenzelm merged
Wed, 10 Apr 2013 19:14:47 +0200 wenzelm merged
Wed, 10 Apr 2013 17:27:38 +0200 wenzelm obsolete -- tools should refer to proper Proof.context;
Wed, 10 Apr 2013 17:17:16 +0200 wenzelm discontinued obsolete ML antiquotation @{claset};
Wed, 10 Apr 2013 17:02:47 +0200 wenzelm added ML antiquotation @{theory_context};
Wed, 10 Apr 2013 15:30:19 +0200 wenzelm more standard module name Axclass (according to file name);
Wed, 10 Apr 2013 19:52:19 +0200 traytel made SML/NJ happy
Wed, 10 Apr 2013 18:51:21 +0200 hoelzl 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 traytel NEWS and CONTRIBUTORS
Wed, 10 Apr 2013 17:49:16 +0200 traytel declaration attribute for case combinators
Tue, 09 Apr 2013 18:27:49 +0200 berghofe Handle dummy patterns in parse translation rather than check phase
Sat, 06 Apr 2013 01:42:07 +0200 traytel disallow coercions to interfere with case translations
Fri, 05 Apr 2013 22:08:42 +0200 traytel allow redundant cases in the list comprehension translation
Fri, 05 Apr 2013 22:08:42 +0200 traytel recur in the expression to be matched (do not rely on repetitive execution of a check phase);
Fri, 05 Apr 2013 22:08:42 +0200 traytel tuned whitespace
Thu, 04 Apr 2013 18:48:40 +0200 berghofe Use Type.raw_match instead of Sign.typ_match
Fri, 05 Apr 2013 22:08:42 +0200 traytel special constant to prevent eta-contraction of the check-phase syntax of case translations
Tue, 22 Jan 2013 14:33:45 +0100 traytel separate data used for case translation from the datatype package
Tue, 22 Jan 2013 13:32:41 +0100 berghofe case translations performed in a separate check phase (with adjustments by traytel)
Wed, 10 Apr 2013 13:10:38 +0200 wenzelm formal proof context for axclass proofs;
Wed, 10 Apr 2013 12:31:35 +0200 wenzelm prefer local context;
Wed, 10 Apr 2013 12:24:43 +0200 wenzelm proper proof context;
Wed, 10 Apr 2013 11:51:56 +0200 wenzelm tuned;
Tue, 09 Apr 2013 21:39:55 +0200 wenzelm merged
Tue, 09 Apr 2013 21:22:15 +0200 wenzelm add command timings (like document command status);
Tue, 09 Apr 2013 21:14:00 +0200 wenzelm tuned signature;
Tue, 09 Apr 2013 20:34:15 +0200 wenzelm public Isabelle_Process.xml_cache (thread-safe);
Tue, 09 Apr 2013 20:27:27 +0200 wenzelm tuned signature;
Tue, 09 Apr 2013 20:16:52 +0200 wenzelm just one timing protocol function, with 3 implementations: TTY/PG, PIDE/document, build;
Tue, 09 Apr 2013 15:59:02 +0200 wenzelm clarified protocol_message undefinedness;
Tue, 09 Apr 2013 15:40:34 +0200 wenzelm quote by Alan Kay;
Tue, 09 Apr 2013 15:37:23 +0200 wenzelm more accurate documentation;
Tue, 09 Apr 2013 15:29:25 +0200 wenzelm discontinued Toplevel.no_timing complication -- also recovers timing of diagnostic commands, e.g. 'find_theorems';
Tue, 09 Apr 2013 13:55:28 +0200 wenzelm more accurate documentation of "(structure)" mixfix;
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 tip