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;
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
Thu, 04 Apr 2013 18:48:40 +0200 Use Type.raw_match instead of Sign.typ_match
berghofe [Thu, 04 Apr 2013 18:48:40 +0200] rev 51675
Use Type.raw_match instead of Sign.typ_match
Fri, 05 Apr 2013 22:08:42 +0200 special constant to prevent eta-contraction of the check-phase syntax of case translations
traytel [Fri, 05 Apr 2013 22:08:42 +0200] rev 51674
special constant to prevent eta-contraction of the check-phase syntax of case translations
Tue, 22 Jan 2013 14:33:45 +0100 separate data used for case translation from the datatype package
traytel [Tue, 22 Jan 2013 14:33:45 +0100] rev 51673
separate data used for case translation from the datatype package
Tue, 22 Jan 2013 13:32:41 +0100 case translations performed in a separate check phase (with adjustments by traytel)
berghofe [Tue, 22 Jan 2013 13:32:41 +0100] rev 51672
case translations performed in a separate check phase (with adjustments by traytel)
Wed, 10 Apr 2013 13:10:38 +0200 formal proof context for axclass proofs;
wenzelm [Wed, 10 Apr 2013 13:10:38 +0200] rev 51671
formal proof context for axclass proofs; avoid global_simpset_of -- refer to simpset of proof context;
Wed, 10 Apr 2013 12:31:35 +0200 prefer local context;
wenzelm [Wed, 10 Apr 2013 12:31:35 +0200] rev 51670
prefer local context;
Wed, 10 Apr 2013 12:24:43 +0200 proper proof context;
wenzelm [Wed, 10 Apr 2013 12:24:43 +0200] rev 51669
proper proof context; removed historic comments;
Wed, 10 Apr 2013 11:51:56 +0200 tuned;
wenzelm [Wed, 10 Apr 2013 11:51:56 +0200] rev 51668
tuned;
Tue, 09 Apr 2013 21:39:55 +0200 merged
wenzelm [Tue, 09 Apr 2013 21:39:55 +0200] rev 51667
merged
Tue, 09 Apr 2013 21:22:15 +0200 add command timings (like document command status);
wenzelm [Tue, 09 Apr 2013 21:22:15 +0200] rev 51666
add command timings (like document command status);
Tue, 09 Apr 2013 21:14:00 +0200 tuned signature;
wenzelm [Tue, 09 Apr 2013 21:14:00 +0200] rev 51665
tuned signature;
Tue, 09 Apr 2013 20:34:15 +0200 public Isabelle_Process.xml_cache (thread-safe);
wenzelm [Tue, 09 Apr 2013 20:34:15 +0200] rev 51664
public Isabelle_Process.xml_cache (thread-safe); cache derived status messages;
Tue, 09 Apr 2013 20:27:27 +0200 tuned signature;
wenzelm [Tue, 09 Apr 2013 20:27:27 +0200] rev 51663
tuned signature;
Tue, 09 Apr 2013 20:16:52 +0200 just one timing protocol function, with 3 implementations: TTY/PG, PIDE/document, build;
wenzelm [Tue, 09 Apr 2013 20:16:52 +0200] rev 51662
just one timing protocol function, with 3 implementations: TTY/PG, PIDE/document, build;
Tue, 09 Apr 2013 15:59:02 +0200 clarified protocol_message undefinedness;
wenzelm [Tue, 09 Apr 2013 15:59:02 +0200] rev 51661
clarified protocol_message undefinedness;
Tue, 09 Apr 2013 15:40:34 +0200 quote by Alan Kay;
wenzelm [Tue, 09 Apr 2013 15:40:34 +0200] rev 51660
quote by Alan Kay;
Tue, 09 Apr 2013 15:37:23 +0200 more accurate documentation;
wenzelm [Tue, 09 Apr 2013 15:37:23 +0200] rev 51659
more accurate documentation;
Tue, 09 Apr 2013 15:29:25 +0200 discontinued Toplevel.no_timing complication -- also recovers timing of diagnostic commands, e.g. 'find_theorems';
wenzelm [Tue, 09 Apr 2013 15:29:25 +0200] rev 51658
discontinued Toplevel.no_timing complication -- also recovers timing of diagnostic commands, e.g. 'find_theorems'; print timing as tracing, to keep it out of the way in Proof General; no timing of control commands, especially relevant for Proof General;
Tue, 09 Apr 2013 13:55:28 +0200 more accurate documentation of "(structure)" mixfix;
wenzelm [Tue, 09 Apr 2013 13:55:28 +0200] rev 51657
more accurate documentation of "(structure)" mixfix;
Tue, 09 Apr 2013 13:24:00 +0200 more robust static structure reference, avoid dynamic Proof_Context.intern_skolem in Syntax_Phases.decode_term;
wenzelm [Tue, 09 Apr 2013 13:24:00 +0200] rev 51656
more robust static structure reference, avoid dynamic Proof_Context.intern_skolem in Syntax_Phases.decode_term;
Tue, 09 Apr 2013 13:20:09 +0200 tuned comment;
wenzelm [Tue, 09 Apr 2013 13:20:09 +0200] rev 51655
tuned comment;
Tue, 09 Apr 2013 12:56:26 +0200 just one syntax category "mixfix" -- check structure annotation semantically;
wenzelm [Tue, 09 Apr 2013 12:56:26 +0200] rev 51654
just one syntax category "mixfix" -- check structure annotation semantically;
Tue, 09 Apr 2013 12:29:36 +0200 tuned message;
wenzelm [Tue, 09 Apr 2013 12:29:36 +0200] rev 51653
tuned message;
Tue, 09 Apr 2013 16:32:04 +0200 handle case clashes on Mac file system by encoding goal numbers
blanchet [Tue, 09 Apr 2013 16:32:04 +0200] rev 51652
handle case clashes on Mac file system by encoding goal numbers
Tue, 09 Apr 2013 15:19:14 +0200 avoid duplicate "tcon_" names
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51651
avoid duplicate "tcon_" names
Tue, 09 Apr 2013 15:19:14 +0200 smoothly handle cyclic graphs
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51650
smoothly handle cyclic graphs
Tue, 09 Apr 2013 15:19:14 +0200 compile + fixed naming convention
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51649
compile + fixed naming convention
Tue, 09 Apr 2013 15:19:14 +0200 reverted accidental changes to theory file + updated wrt ML file
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51648
reverted accidental changes to theory file + updated wrt ML file
Tue, 09 Apr 2013 15:19:14 +0200 no need to filter tautologies anymore -- they are prefiltered by "all_facts"'
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51647
no need to filter tautologies anymore -- they are prefiltered by "all_facts"'
Tue, 09 Apr 2013 15:19:14 +0200 work on CASC LTB ISA exporter
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51646
work on CASC LTB ISA exporter
Tue, 09 Apr 2013 15:19:14 +0200 tuning
blanchet [Tue, 09 Apr 2013 15:19:14 +0200] rev 51645
tuning
Tue, 09 Apr 2013 15:07:35 +0200 add continuous_on rules for products
hoelzl [Tue, 09 Apr 2013 15:07:35 +0200] rev 51644
add continuous_on rules for products
Tue, 09 Apr 2013 14:13:13 +0200 fixed spelling
hoelzl [Tue, 09 Apr 2013 14:13:13 +0200] rev 51643
fixed spelling
Tue, 09 Apr 2013 14:04:47 +0200 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
hoelzl [Tue, 09 Apr 2013 14:04:47 +0200] rev 51642
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 remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
hoelzl [Tue, 09 Apr 2013 14:04:41 +0200] rev 51641
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 improved printing of exception CTERM (see also d0f0f37ec346);
wenzelm [Mon, 08 Apr 2013 21:01:59 +0200] rev 51640
improved printing of exception CTERM (see also d0f0f37ec346);
Mon, 08 Apr 2013 17:10:49 +0200 prefer pretty_exn where possible -- NB: low-level General.exnMessage may still be used elsewhere (e.g. by the ML compiler itself);
wenzelm [Mon, 08 Apr 2013 17:10:49 +0200] rev 51639
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 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;
wenzelm [Mon, 08 Apr 2013 16:06:54 +0200] rev 51638
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 discontinued odd magic number, which was once used for performance measurements;
wenzelm [Mon, 08 Apr 2013 15:44:09 +0200] rev 51637
discontinued odd magic number, which was once used for performance measurements;
Mon, 08 Apr 2013 15:35:48 +0200 document @{make_string}, cf. NEWS of Isabelle2009-2 (June 2010);
wenzelm [Mon, 08 Apr 2013 15:35:48 +0200] rev 51636
document @{make_string}, cf. NEWS of Isabelle2009-2 (June 2010);
Mon, 08 Apr 2013 14:28:37 +0200 merged
wenzelm [Mon, 08 Apr 2013 14:28:37 +0200] rev 51635
merged
Mon, 08 Apr 2013 14:18:39 +0200 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;
wenzelm [Mon, 08 Apr 2013 14:18:39 +0200] rev 51634
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 try to preserve original linearization
blanchet [Mon, 08 Apr 2013 14:16:00 +0200] rev 51633
try to preserve original linearization
Mon, 08 Apr 2013 12:27:13 +0200 use somewhat lighter encoding
blanchet [Mon, 08 Apr 2013 12:27:13 +0200] rev 51632
use somewhat lighter encoding
Mon, 08 Apr 2013 12:11:06 +0200 robustness w.r.t. unknown arguments
blanchet [Mon, 08 Apr 2013 12:11:06 +0200] rev 51631
robustness w.r.t. unknown arguments
Sun, 07 Apr 2013 15:08:34 +0200 cleaned
nipkow [Sun, 07 Apr 2013 15:08:34 +0200] rev 51630
cleaned
Sun, 07 Apr 2013 10:06:37 +0200 cleaned
nipkow [Sun, 07 Apr 2013 10:06:37 +0200] rev 51629
cleaned
Sat, 06 Apr 2013 18:42:55 +0200 tuned
nipkow [Sat, 06 Apr 2013 18:42:55 +0200] rev 51628
tuned
Fri, 05 Apr 2013 20:54:55 +0200 tuned signature -- agree with markup terminology;
wenzelm [Fri, 05 Apr 2013 20:54:55 +0200] rev 51627
tuned signature -- agree with markup terminology;
Fri, 05 Apr 2013 20:43:43 +0200 unified terminology with Markup.DOCUMENT_SOURCE in Scala, which is unused but displayed as "document source" entity in Isabelle/jEdit;
wenzelm [Fri, 05 Apr 2013 20:43:43 +0200] rev 51626
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 tuned document
nipkow [Fri, 05 Apr 2013 18:31:35 +0200] rev 51625
tuned document
Fri, 05 Apr 2013 15:13:25 +0200 tuned
nipkow [Fri, 05 Apr 2013 15:13:25 +0200] rev 51624
tuned
Thu, 04 Apr 2013 22:46:14 +0200 sup on multisets
haftmann [Thu, 04 Apr 2013 22:46:14 +0200] rev 51623
sup on multisets
Thu, 04 Apr 2013 22:29:59 +0200 convenient induction rule
haftmann [Thu, 04 Apr 2013 22:29:59 +0200] rev 51622
convenient induction rule
Thu, 04 Apr 2013 20:59:16 +0200 tuned README -- less buzzwords;
wenzelm [Thu, 04 Apr 2013 20:59:16 +0200] rev 51621
tuned README -- less buzzwords;
Thu, 04 Apr 2013 18:44:22 +0200 more conventional synchronized access to Options_Variable -- avoid Swing_Thread getting in the way, which might be absent in some environments (e.g. SWT);
wenzelm [Thu, 04 Apr 2013 18:44:22 +0200] rev 51620
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 added missing file;
wenzelm [Thu, 04 Apr 2013 18:25:47 +0200] rev 51619
added missing file;
Thu, 04 Apr 2013 18:20:00 +0200 tuned signature -- avoid intrusion of slightly odd Swing structures into pure Markup_Tree;
wenzelm [Thu, 04 Apr 2013 18:20:00 +0200] rev 51618
tuned signature -- avoid intrusion of slightly odd Swing structures into pure Markup_Tree;
Thu, 04 Apr 2013 18:06:48 +0200 tuned signature -- concentrate GUI tools;
wenzelm [Thu, 04 Apr 2013 18:06:48 +0200] rev 51617
tuned signature -- concentrate GUI tools;
Thu, 04 Apr 2013 17:58:47 +0200 tuned signature -- concentrate GUI tools;
wenzelm [Thu, 04 Apr 2013 17:58:47 +0200] rev 51616
tuned signature -- concentrate GUI tools;
Thu, 04 Apr 2013 17:47:28 +0200 separate module "GUI", to keep this out of the way of generic Isabelle_System operations, notably for non-Isabelle/jEdit applications;
wenzelm [Thu, 04 Apr 2013 17:47:28 +0200] rev 51615
separate module "GUI", to keep this out of the way of generic Isabelle_System operations, notably for non-Isabelle/jEdit applications; tuned signature;
Thu, 04 Apr 2013 17:33:04 +0200 separate module Isabelle_Font, to keep this out of the way of generic Isabelle_System operations, notably for non-Isabelle/jEdit applications;
wenzelm [Thu, 04 Apr 2013 17:33:04 +0200] rev 51614
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 tuned imports;
wenzelm [Thu, 04 Apr 2013 17:16:51 +0200] rev 51613
tuned imports;
Thu, 04 Apr 2013 12:06:23 +0200 added var_position in analogy to longid_position, for typing reports on input;
wenzelm [Thu, 04 Apr 2013 12:06:23 +0200] rev 51612
added var_position in analogy to longid_position, for typing reports on input; avoid duplicate token var report;
Thu, 04 Apr 2013 10:30:28 +0200 removed unnerving (esp in jedit) and pointless warning
nipkow [Thu, 04 Apr 2013 10:30:28 +0200] rev 51611
removed unnerving (esp in jedit) and pointless warning
Thu, 04 Apr 2013 08:10:20 +0200 tuned
nipkow [Thu, 04 Apr 2013 08:10:20 +0200] rev 51610
tuned
Wed, 03 Apr 2013 22:31:05 +0200 merged
wenzelm [Wed, 03 Apr 2013 22:31:05 +0200] rev 51609
merged
Wed, 03 Apr 2013 22:30:25 +0200 tuned;
wenzelm [Wed, 03 Apr 2013 22:30:25 +0200] rev 51608
tuned;
Wed, 03 Apr 2013 22:05:24 +0200 recover implicit thread position for status messages (cf. eca8acb42e4a);
wenzelm [Wed, 03 Apr 2013 22:05:24 +0200] rev 51607
recover implicit thread position for status messages (cf. eca8acb42e4a);
Wed, 03 Apr 2013 21:48:43 +0200 additional timing status for implicitly forked terminal proofs -- proper accounting for interactive Timing dockable etc.;
wenzelm [Wed, 03 Apr 2013 21:48:43 +0200] rev 51606
additional timing status for implicitly forked terminal proofs -- proper accounting for interactive Timing dockable etc.;
Wed, 03 Apr 2013 21:30:32 +0200 more explicit Goal.fork_params -- avoid implicit arguments via thread data;
wenzelm [Wed, 03 Apr 2013 21:30:32 +0200] rev 51605
more explicit Goal.fork_params -- avoid implicit arguments via thread data; actually fork terminal proofs in interactive mode (amending 8707df0b0255);
Wed, 03 Apr 2013 20:56:08 +0200 updated comment to 46b90bbc370d;
wenzelm [Wed, 03 Apr 2013 20:56:08 +0200] rev 51604
updated comment to 46b90bbc370d;
Wed, 03 Apr 2013 20:38:50 +0200 recovered proper transaction position for Goal.fork error reporting (lost in 8e9746e584c9);
wenzelm [Wed, 03 Apr 2013 20:38:50 +0200] rev 51603
recovered proper transaction position for Goal.fork error reporting (lost in 8e9746e584c9);
Wed, 03 Apr 2013 16:45:14 +0200 tuned -- Drule.comp_no_flatten includes Drule.incr_indexes already (NB: result should be deterministic by construction);
wenzelm [Wed, 03 Apr 2013 16:45:14 +0200] rev 51602
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 tuned output -- less bullets;
wenzelm [Wed, 03 Apr 2013 13:58:00 +0200] rev 51601
tuned output -- less bullets;
Wed, 03 Apr 2013 22:26:04 +0200 default implementation of multisets by list with reasonable coverage of operations on multisets
haftmann [Wed, 03 Apr 2013 22:26:04 +0200] rev 51600
default implementation of multisets by list with reasonable coverage of operations on multisets
Wed, 03 Apr 2013 22:26:04 +0200 optionalized very specific code setup for multisets
haftmann [Wed, 03 Apr 2013 22:26:04 +0200] rev 51599
optionalized very specific code setup for multisets
Wed, 03 Apr 2013 10:15:43 +0200 generalized lemma fold_image thanks to Peter Lammich
haftmann [Wed, 03 Apr 2013 10:15:43 +0200] rev 51598
generalized lemma fold_image thanks to Peter Lammich
Tue, 02 Apr 2013 20:19:38 +0200 tuned;
wenzelm [Tue, 02 Apr 2013 20:19:38 +0200] rev 51597
tuned;
Tue, 02 Apr 2013 16:29:40 +0200 NEWS for 635562bc14ef;
wenzelm [Tue, 02 Apr 2013 16:29:40 +0200] rev 51596
NEWS for 635562bc14ef;
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip