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
Mon, 08 Apr 2013 12:27:13 +0200 blanchet use somewhat lighter encoding
Mon, 08 Apr 2013 12:11:06 +0200 blanchet robustness w.r.t. unknown arguments
Sun, 07 Apr 2013 15:08:34 +0200 nipkow cleaned
Sun, 07 Apr 2013 10:06:37 +0200 nipkow cleaned
Sat, 06 Apr 2013 18:42:55 +0200 nipkow tuned
Fri, 05 Apr 2013 20:54:55 +0200 wenzelm tuned signature -- agree with markup terminology;
Fri, 05 Apr 2013 20:43:43 +0200 wenzelm unified terminology with Markup.DOCUMENT_SOURCE in Scala, which is unused but displayed as "document source" entity in Isabelle/jEdit;
Fri, 05 Apr 2013 18:31:35 +0200 nipkow tuned document
Fri, 05 Apr 2013 15:13:25 +0200 nipkow tuned
Thu, 04 Apr 2013 22:46:14 +0200 haftmann sup on multisets
Thu, 04 Apr 2013 22:29:59 +0200 haftmann convenient induction rule
Thu, 04 Apr 2013 20:59:16 +0200 wenzelm tuned README -- less buzzwords;
Thu, 04 Apr 2013 18:44:22 +0200 wenzelm more conventional synchronized access to Options_Variable -- avoid Swing_Thread getting in the way, which might be absent in some environments (e.g. SWT);
Thu, 04 Apr 2013 18:25:47 +0200 wenzelm added missing file;
Thu, 04 Apr 2013 18:20:00 +0200 wenzelm tuned signature -- avoid intrusion of slightly odd Swing structures into pure Markup_Tree;
Thu, 04 Apr 2013 18:06:48 +0200 wenzelm tuned signature -- concentrate GUI tools;
Thu, 04 Apr 2013 17:58:47 +0200 wenzelm tuned signature -- concentrate GUI tools;
Thu, 04 Apr 2013 17:47:28 +0200 wenzelm separate module "GUI", to keep this out of the way of generic Isabelle_System operations, notably for non-Isabelle/jEdit applications;
Thu, 04 Apr 2013 17:33:04 +0200 wenzelm separate module Isabelle_Font, to keep this out of the way of generic Isabelle_System operations, notably for non-Isabelle/jEdit applications;
Thu, 04 Apr 2013 17:16:51 +0200 wenzelm tuned imports;
Thu, 04 Apr 2013 12:06:23 +0200 wenzelm added var_position in analogy to longid_position, for typing reports on input;
Thu, 04 Apr 2013 10:30:28 +0200 nipkow removed unnerving (esp in jedit) and pointless warning
Thu, 04 Apr 2013 08:10:20 +0200 nipkow tuned
Wed, 03 Apr 2013 22:31:05 +0200 wenzelm merged
Wed, 03 Apr 2013 22:30:25 +0200 wenzelm tuned;
Wed, 03 Apr 2013 22:05:24 +0200 wenzelm recover implicit thread position for status messages (cf. eca8acb42e4a);
Wed, 03 Apr 2013 21:48:43 +0200 wenzelm additional timing status for implicitly forked terminal proofs -- proper accounting for interactive Timing dockable etc.;
Wed, 03 Apr 2013 21:30:32 +0200 wenzelm more explicit Goal.fork_params -- avoid implicit arguments via thread data;
Wed, 03 Apr 2013 20:56:08 +0200 wenzelm updated comment to 46b90bbc370d;
Wed, 03 Apr 2013 20:38:50 +0200 wenzelm recovered proper transaction position for Goal.fork error reporting (lost in 8e9746e584c9);
Wed, 03 Apr 2013 16:45:14 +0200 wenzelm tuned -- Drule.comp_no_flatten includes Drule.incr_indexes already (NB: result should be deterministic by construction);
Wed, 03 Apr 2013 13:58:00 +0200 wenzelm tuned output -- less bullets;
Wed, 03 Apr 2013 22:26:04 +0200 haftmann default implementation of multisets by list with reasonable coverage of operations on multisets
Wed, 03 Apr 2013 22:26:04 +0200 haftmann optionalized very specific code setup for multisets
Wed, 03 Apr 2013 10:15:43 +0200 haftmann generalized lemma fold_image thanks to Peter Lammich
Tue, 02 Apr 2013 20:19:38 +0200 wenzelm tuned;
Tue, 02 Apr 2013 16:29:40 +0200 wenzelm NEWS for 635562bc14ef;
Tue, 02 Apr 2013 11:41:50 +0200 wenzelm more centralized command timing;
Tue, 02 Apr 2013 10:58:51 +0200 blanchet got rid of legacy smartness
Mon, 01 Apr 2013 17:42:29 +0200 nipkow added lemma
Sat, 30 Mar 2013 18:24:33 +0100 wenzelm merged
Sat, 30 Mar 2013 17:27:21 +0100 wenzelm amended uncond_skel to observe notion of cong_name properly -- may affect simplification with Free congs;
Sat, 30 Mar 2013 17:13:21 +0100 wenzelm more formal cong_name;
Sat, 30 Mar 2013 16:34:02 +0100 wenzelm timing status for forked diagnostic commands;
Sat, 30 Mar 2013 16:16:24 +0100 wenzelm tooltip of command keyword includes timing information;
Sat, 30 Mar 2013 16:15:26 +0100 wenzelm more operations on Time, Timing;
Fri, 29 Mar 2013 18:57:47 +0100 haftmann reverted slip introduced in f738e6dbd844
Sat, 30 Mar 2013 14:57:06 +0100 wenzelm added 'print_defn_rules' command;
Sat, 30 Mar 2013 13:40:19 +0100 wenzelm more item markup;
Sat, 30 Mar 2013 12:13:39 +0100 wenzelm item markup for Proof_Context.pretty_fact;
Sat, 30 Mar 2013 11:43:17 +0100 wenzelm obsolete, cf. Proof_Context.print_syntax;
Fri, 29 Mar 2013 22:26:25 +0100 wenzelm paint bullet bar within text layer -- thus it remains visible with active selection etc.;
Fri, 29 Mar 2013 22:14:27 +0100 wenzelm Pretty.item markup for improved readability of lists of items;
Fri, 29 Mar 2013 22:13:02 +0100 wenzelm tuned message;
Fri, 29 Mar 2013 11:32:07 +0100 haftmann convenience check for vain instantiation
Fri, 29 Mar 2013 13:32:53 +0100 wenzelm improved centering via strikethrough offset;
Thu, 28 Mar 2013 23:44:43 +0100 boehmes re-generated SMT certificates
Thu, 28 Mar 2013 23:44:41 +0100 boehmes new, simpler implementation of monomorphization;
Thu, 28 Mar 2013 22:42:18 +0100 wenzelm ghost bullet via markup, which is painted as bar under text (normally space);
Thu, 28 Mar 2013 16:11:48 +0100 kleing replace induction by hammer
Thu, 28 Mar 2013 15:47:03 +0100 wenzelm merged
Thu, 28 Mar 2013 15:37:39 +0100 wenzelm merged;
Thu, 28 Mar 2013 15:36:45 +0100 wenzelm basic support for Pretty.item, which is considered as logical markup and interpreted in Isabelle/Scala, but ignored elsewhere (TTY, latex etc.);
Thu, 28 Mar 2013 15:00:27 +0100 wenzelm maintain integer indentation during formatting -- it needs to be implemented by repeated spaces eventually;
Thu, 28 Mar 2013 14:47:37 +0100 wenzelm tuned;
Thu, 28 Mar 2013 14:01:56 +0100 wenzelm proper default browser info for interactive mode, notably thy_deps;
Thu, 28 Mar 2013 15:45:08 +0100 nipkow improved pretty printing for state set acom
Wed, 27 Mar 2013 22:36:03 +0100 ballarin Improvements to the print_dependencies command.
Wed, 27 Mar 2013 21:25:33 +0100 wenzelm discontinued obsolete parallel_proofs_reuse_timing;
Wed, 27 Mar 2013 21:13:02 +0100 wenzelm merged
Wed, 27 Mar 2013 21:07:10 +0100 wenzelm separate isatest with skip_proofs, to give some impression of performance without most of the proofs;
Wed, 27 Mar 2013 21:12:49 +0100 wenzelm merged
Wed, 27 Mar 2013 20:57:05 +0100 wenzelm extra checkpoint to avoid stale theory in skip_proof context, e.g. in 'instance' proof;
Wed, 27 Mar 2013 19:32:44 +0100 wenzelm tuned;
Wed, 27 Mar 2013 18:04:21 +0100 wenzelm allow build with skip_proofs enabled -- disable it for sessions that would fail due to embedded diagnostic commands, for example;
Wed, 27 Mar 2013 17:58:07 +0100 wenzelm more robust access Toplevel.proof_of -- prefer warning via Toplevel.unknown_proof over hard crash (notably for skipped proofs);
Wed, 27 Mar 2013 17:55:21 +0100 wenzelm more liberal handling of skipped proofs;
Wed, 27 Mar 2013 17:53:29 +0100 wenzelm explicit Toplevel.is_skipped_proof;
Wed, 27 Mar 2013 16:46:52 +0100 wenzelm separate option editor_skip_proofs, to avoid accidental change of preferences for skip_proofs, which would invalidate batch builds;
Wed, 27 Mar 2013 16:38:25 +0100 wenzelm more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
Wed, 27 Mar 2013 14:50:30 +0100 wenzelm clarified Skip_Proof.cheat_tac: more standard tactic;
Wed, 27 Mar 2013 14:19:18 +0100 wenzelm tuned signature and module arrangement;
Wed, 27 Mar 2013 14:08:03 +0100 wenzelm tuned;
Wed, 27 Mar 2013 11:54:53 +0100 wenzelm tuned GUI;
Wed, 27 Mar 2013 10:55:05 +0100 haftmann centralized various multiset operations in theory multiset;
Tue, 26 Mar 2013 22:09:39 +0100 haftmann avoid odd foundational terms after interpretation;
Tue, 26 Mar 2013 21:53:56 +0100 haftmann more uniform style for interpretation and sublocale declarations
Tue, 26 Mar 2013 20:55:21 +0100 wenzelm merged
Tue, 26 Mar 2013 20:37:32 +0100 wenzelm tuned session specification;
Tue, 26 Mar 2013 20:36:32 +0100 wenzelm tuned proof;
Tue, 26 Mar 2013 20:02:02 +0100 wenzelm tuned imports;
Tue, 26 Mar 2013 19:43:31 +0100 wenzelm tuned proofs;
Tue, 26 Mar 2013 20:49:57 +0100 haftmann explicit sublocale dependency for Min/Max yields more appropriate Min/Max prefix for a couple of facts
Tue, 26 Mar 2013 15:10:28 +0100 wenzelm merged
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip