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;
Tue, 09 Apr 2013 13:24:00 +0200 wenzelm more robust static structure reference, avoid dynamic Proof_Context.intern_skolem in Syntax_Phases.decode_term;
Tue, 09 Apr 2013 13:20:09 +0200 wenzelm tuned comment;
Tue, 09 Apr 2013 12:56:26 +0200 wenzelm just one syntax category "mixfix" -- check structure annotation semantically;
Tue, 09 Apr 2013 12:29:36 +0200 wenzelm tuned message;
Tue, 09 Apr 2013 16:32:04 +0200 blanchet handle case clashes on Mac file system by encoding goal numbers
Tue, 09 Apr 2013 15:19:14 +0200 blanchet avoid duplicate "tcon_" names
Tue, 09 Apr 2013 15:19:14 +0200 blanchet smoothly handle cyclic graphs
Tue, 09 Apr 2013 15:19:14 +0200 blanchet compile + fixed naming convention
Tue, 09 Apr 2013 15:19:14 +0200 blanchet reverted accidental changes to theory file + updated wrt ML file
Tue, 09 Apr 2013 15:19:14 +0200 blanchet no need to filter tautologies anymore -- they are prefiltered by "all_facts"'
Tue, 09 Apr 2013 15:19:14 +0200 blanchet work on CASC LTB ISA exporter
Tue, 09 Apr 2013 15:19:14 +0200 blanchet tuning
Tue, 09 Apr 2013 15:07:35 +0200 hoelzl add continuous_on rules for products
Tue, 09 Apr 2013 14:13:13 +0200 hoelzl fixed spelling
Tue, 09 Apr 2013 14:04:47 +0200 hoelzl move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
Tue, 09 Apr 2013 14:04:41 +0200 hoelzl remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
Mon, 08 Apr 2013 21:01:59 +0200 wenzelm improved printing of exception CTERM (see also d0f0f37ec346);
Mon, 08 Apr 2013 17:10:49 +0200 wenzelm prefer pretty_exn where possible -- NB: low-level General.exnMessage may still be used elsewhere (e.g. by the ML compiler itself);
Mon, 08 Apr 2013 16:06:54 +0200 wenzelm more defensive representation of forced break within PolyML.PrettyBreak -- avoid accidental blowup if low-level operations are used, notably PolyML.makestring or its variant General.exnMessage;
Mon, 08 Apr 2013 15:44:09 +0200 wenzelm discontinued odd magic number, which was once used for performance measurements;
Mon, 08 Apr 2013 15:35:48 +0200 wenzelm document @{make_string}, cf. NEWS of Isabelle2009-2 (June 2010);
Mon, 08 Apr 2013 14:28:37 +0200 wenzelm merged
Mon, 08 Apr 2013 14:18:39 +0200 wenzelm more general Thy_Load.import_name, e.g. relevant for Isabelle/eclipse -- NB: Thy_Load serves as main hub for funny overriding to adapt to provers and editors;
Mon, 08 Apr 2013 14:16:00 +0200 blanchet try to preserve original linearization
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 tip