Sun, 14 Oct 2012 19:16:32 +0200 extending the setcomprehension_pointfree simproc to handle nesting disjunctions, conjunctions and negations (with contributions from Rafal Kolanski, NICTA); tuned
bulwahn [Sun, 14 Oct 2012 19:16:32 +0200] rev 49849
extending the setcomprehension_pointfree simproc to handle nesting disjunctions, conjunctions and negations (with contributions from Rafal Kolanski, NICTA); tuned
Sat, 13 Oct 2012 21:09:20 +0200 more informative error of initial/terminal proof steps;
wenzelm [Sat, 13 Oct 2012 21:09:20 +0200] rev 49848
more informative error of initial/terminal proof steps;
Sat, 13 Oct 2012 19:53:04 +0200 some attempts to unify/simplify pretty_goal;
wenzelm [Sat, 13 Oct 2012 19:53:04 +0200] rev 49847
some attempts to unify/simplify pretty_goal;
Sat, 13 Oct 2012 18:04:11 +0200 refined Proof.the_finished_goal with more informative error;
wenzelm [Sat, 13 Oct 2012 18:04:11 +0200] rev 49846
refined Proof.the_finished_goal with more informative error; more permissive Method.all_assm_tac: do not insist in solving by assumption here to postpone failure; clarified Method.finish_text: no Thm.no_prems filtering here to postpone failure;
Sat, 13 Oct 2012 16:19:16 +0200 tuned signature;
wenzelm [Sat, 13 Oct 2012 16:19:16 +0200] rev 49845
tuned signature;
Sat, 13 Oct 2012 00:08:36 +0200 improved adhoc height for small fonts;
wenzelm [Sat, 13 Oct 2012 00:08:36 +0200] rev 49844
improved adhoc height for small fonts;
Fri, 12 Oct 2012 23:38:48 +0200 further refinement of jEdit line range, avoiding lack of final \n;
wenzelm [Fri, 12 Oct 2012 23:38:48 +0200] rev 49843
further refinement of jEdit line range, avoiding lack of final \n;
Fri, 12 Oct 2012 22:53:20 +0200 more uniform tooltip color;
wenzelm [Fri, 12 Oct 2012 22:53:20 +0200] rev 49842
more uniform tooltip color;
Fri, 12 Oct 2012 22:10:45 +0200 more NEWS;
wenzelm [Fri, 12 Oct 2012 22:10:45 +0200] rev 49841
more NEWS;
Fri, 12 Oct 2012 21:51:25 +0200 merged
wenzelm [Fri, 12 Oct 2012 21:51:25 +0200] rev 49840
merged
Fri, 12 Oct 2012 15:52:55 +0200 disambiguated grammar
traytel [Fri, 12 Oct 2012 15:52:55 +0200] rev 49839
disambiguated grammar
Fri, 12 Oct 2012 15:52:45 +0200 tuned proofs
traytel [Fri, 12 Oct 2012 15:52:45 +0200] rev 49838
tuned proofs
Fri, 12 Oct 2012 14:57:56 +0200 tuned
nipkow [Fri, 12 Oct 2012 14:57:56 +0200] rev 49837
tuned
Fri, 12 Oct 2012 21:39:58 +0200 simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm [Fri, 12 Oct 2012 21:39:58 +0200] rev 49836
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
Fri, 12 Oct 2012 21:22:35 +0200 discontinued typedef with alternative name;
wenzelm [Fri, 12 Oct 2012 21:22:35 +0200] rev 49835
discontinued typedef with alternative name;
Fri, 12 Oct 2012 18:58:20 +0200 discontinued obsolete typedef (open) syntax;
wenzelm [Fri, 12 Oct 2012 18:58:20 +0200] rev 49834
discontinued obsolete typedef (open) syntax;
Fri, 12 Oct 2012 15:08:29 +0200 discontinued typedef with implicit set_def;
wenzelm [Fri, 12 Oct 2012 15:08:29 +0200] rev 49833
discontinued typedef with implicit set_def;
Fri, 12 Oct 2012 14:05:30 +0200 merged
wenzelm [Fri, 12 Oct 2012 14:05:30 +0200] rev 49832
merged
Fri, 12 Oct 2012 12:21:01 +0200 increading indexes to avoid clashes in the set_comprehension_pointfree simproc
bulwahn [Fri, 12 Oct 2012 12:21:01 +0200] rev 49831
increading indexes to avoid clashes in the set_comprehension_pointfree simproc
Fri, 12 Oct 2012 13:55:13 +0200 no special treatment of errors inside goal forks without transaction id, to avoid duplication in plain build with sequential log, for example;
wenzelm [Fri, 12 Oct 2012 13:55:13 +0200] rev 49830
no special treatment of errors inside goal forks without transaction id, to avoid duplication in plain build with sequential log, for example;
Fri, 12 Oct 2012 13:46:41 +0200 do not treat interrupt as error here, to avoid confusion in log etc.;
wenzelm [Fri, 12 Oct 2012 13:46:41 +0200] rev 49829
do not treat interrupt as error here, to avoid confusion in log etc.;
Fri, 12 Oct 2012 11:03:23 +0200 more basic ML compiler messages -- avoid conflict of 638cefe3ee99 and cb7264721c91 concerning Protocol.message_positions;
wenzelm [Fri, 12 Oct 2012 11:03:23 +0200] rev 49828
more basic ML compiler messages -- avoid conflict of 638cefe3ee99 and cb7264721c91 concerning Protocol.message_positions;
Thu, 11 Oct 2012 23:10:49 +0200 refined separator: FBreak needs to be free for proper breaking, extra space at end helps to work around last-line oddity in jEdit;
wenzelm [Thu, 11 Oct 2012 23:10:49 +0200] rev 49827
refined separator: FBreak needs to be free for proper breaking, extra space at end helps to work around last-line oddity in jEdit;
Thu, 11 Oct 2012 21:02:19 +0200 merged
wenzelm [Thu, 11 Oct 2012 21:02:19 +0200] rev 49826
merged
Thu, 11 Oct 2012 14:38:58 +0200 cleanup borel_measurable_positive_integral_(fst|snd)
hoelzl [Thu, 11 Oct 2012 14:38:58 +0200] rev 49825
cleanup borel_measurable_positive_integral_(fst|snd)
Thu, 11 Oct 2012 11:56:43 +0200 msetprod based directly on Multiset.fold;
haftmann [Thu, 11 Oct 2012 11:56:43 +0200] rev 49824
msetprod based directly on Multiset.fold; pretty syntax for msetprod_image
Thu, 11 Oct 2012 11:56:43 +0200 avoid global interpretation
haftmann [Thu, 11 Oct 2012 11:56:43 +0200] rev 49823
avoid global interpretation
Thu, 11 Oct 2012 11:56:42 +0200 simplified construction of fold combinator on multisets;
haftmann [Thu, 11 Oct 2012 11:56:42 +0200] rev 49822
simplified construction of fold combinator on multisets; more coherent name for fold combinator on multisets
Thu, 11 Oct 2012 20:38:02 +0200 clarified output token markup (see also bc22daeed49e);
wenzelm [Thu, 11 Oct 2012 20:38:02 +0200] rev 49821
clarified output token markup (see also bc22daeed49e);
Thu, 11 Oct 2012 19:25:36 +0200 refined aprop_tr' -- retain entity information by using type slot as adhoc marker;
wenzelm [Thu, 11 Oct 2012 19:25:36 +0200] rev 49820
refined aprop_tr' -- retain entity information by using type slot as adhoc marker;
Thu, 11 Oct 2012 16:09:44 +0200 refrain from quantifying outer fixes, to enable nesting of contexts like "context fixes x context assumes A x";
wenzelm [Thu, 11 Oct 2012 16:09:44 +0200] rev 49819
refrain from quantifying outer fixes, to enable nesting of contexts like "context fixes x context assumes A x"; tuned;
Thu, 11 Oct 2012 15:26:33 +0200 tuned;
wenzelm [Thu, 11 Oct 2012 15:26:33 +0200] rev 49818
tuned;
Thu, 11 Oct 2012 15:06:27 +0200 tuned;
wenzelm [Thu, 11 Oct 2012 15:06:27 +0200] rev 49817
tuned;
Thu, 11 Oct 2012 12:38:18 +0200 more position information for hyperlink and placement of message;
wenzelm [Thu, 11 Oct 2012 12:38:18 +0200] rev 49816
more position information for hyperlink and placement of message;
Thu, 11 Oct 2012 12:37:38 +0200 tuned;
wenzelm [Thu, 11 Oct 2012 12:37:38 +0200] rev 49815
tuned;
Thu, 11 Oct 2012 00:13:21 +0200 mira: discontinued special settings for lxbroy10, which are probably made obsolete by newer polyml
krauss [Thu, 11 Oct 2012 00:13:21 +0200] rev 49814
mira: discontinued special settings for lxbroy10, which are probably made obsolete by newer polyml
Wed, 10 Oct 2012 22:53:48 +0200 removed unused legacy material from mira.py
krauss [Wed, 10 Oct 2012 22:53:48 +0200] rev 49813
removed unused legacy material from mira.py
Wed, 10 Oct 2012 17:43:23 +0200 eliminated some remaining uses of typedef with implicit set definition;
wenzelm [Wed, 10 Oct 2012 17:43:23 +0200] rev 49812
eliminated some remaining uses of typedef with implicit set definition;
Wed, 10 Oct 2012 16:41:19 +0200 merged
Andreas Lochbihler [Wed, 10 Oct 2012 16:41:19 +0200] rev 49811
merged
Wed, 10 Oct 2012 16:18:27 +0200 fix code equation for RBT_Impl.fold
Andreas Lochbihler [Wed, 10 Oct 2012 16:18:27 +0200] rev 49810
fix code equation for RBT_Impl.fold
Wed, 10 Oct 2012 15:17:18 +0200 merged
Andreas Lochbihler [Wed, 10 Oct 2012 15:17:18 +0200] rev 49809
merged
Wed, 10 Oct 2012 15:16:44 +0200 tail-recursive implementation for length
Andreas Lochbihler [Wed, 10 Oct 2012 15:16:44 +0200] rev 49808
tail-recursive implementation for length
Wed, 10 Oct 2012 15:05:07 +0200 correct definition for skip_black
Andreas Lochbihler [Wed, 10 Oct 2012 15:05:07 +0200] rev 49807
correct definition for skip_black
Wed, 10 Oct 2012 16:19:52 +0200 merged
wenzelm [Wed, 10 Oct 2012 16:19:52 +0200] rev 49806
merged
Wed, 10 Oct 2012 13:30:50 +0200 merged
hoelzl [Wed, 10 Oct 2012 13:30:50 +0200] rev 49805
merged
Wed, 10 Oct 2012 12:12:37 +0200 infprod generator works also with empty index set
hoelzl [Wed, 10 Oct 2012 12:12:37 +0200] rev 49804
infprod generator works also with empty index set
Wed, 10 Oct 2012 12:12:36 +0200 add finite entropy
hoelzl [Wed, 10 Oct 2012 12:12:36 +0200] rev 49803
add finite entropy
Wed, 10 Oct 2012 12:12:36 +0200 continuous version of mutual_information_eq_entropy_conditional_entropy
hoelzl [Wed, 10 Oct 2012 12:12:36 +0200] rev 49802
continuous version of mutual_information_eq_entropy_conditional_entropy
Wed, 10 Oct 2012 12:12:35 +0200 add induction for real Borel measurable functions
hoelzl [Wed, 10 Oct 2012 12:12:35 +0200] rev 49801
add induction for real Borel measurable functions
Wed, 10 Oct 2012 12:12:34 +0200 induction prove for positive_integral_fst
hoelzl [Wed, 10 Oct 2012 12:12:34 +0200] rev 49800
induction prove for positive_integral_fst
Wed, 10 Oct 2012 12:12:34 +0200 strong nonnegativ (instead of ae nn) for induction rule
hoelzl [Wed, 10 Oct 2012 12:12:34 +0200] rev 49799
strong nonnegativ (instead of ae nn) for induction rule
Wed, 10 Oct 2012 12:12:33 +0200 induction prove for positive_integral_density
hoelzl [Wed, 10 Oct 2012 12:12:33 +0200] rev 49798
induction prove for positive_integral_density
Wed, 10 Oct 2012 12:12:32 +0200 add induction rules for simple functions and for Borel measurable functions
hoelzl [Wed, 10 Oct 2012 12:12:32 +0200] rev 49797
add induction rules for simple functions and for Borel measurable functions
Wed, 10 Oct 2012 12:12:32 +0200 introduce induction rules for simple functions and for Borel measurable functions
hoelzl [Wed, 10 Oct 2012 12:12:32 +0200] rev 49796
introduce induction rules for simple functions and for Borel measurable functions
Wed, 10 Oct 2012 12:12:31 +0200 joint distribution of independent variables
hoelzl [Wed, 10 Oct 2012 12:12:31 +0200] rev 49795
joint distribution of independent variables
Wed, 10 Oct 2012 12:12:30 +0200 indep_vars does not need sigma-sets
hoelzl [Wed, 10 Oct 2012 12:12:30 +0200] rev 49794
indep_vars does not need sigma-sets
Wed, 10 Oct 2012 12:12:29 +0200 simplified definitions
hoelzl [Wed, 10 Oct 2012 12:12:29 +0200] rev 49793
simplified definitions
Wed, 10 Oct 2012 12:12:29 +0200 remove unnecessary assumption from conditional_entropy_eq
hoelzl [Wed, 10 Oct 2012 12:12:29 +0200] rev 49792
remove unnecessary assumption from conditional_entropy_eq
Wed, 10 Oct 2012 12:12:28 +0200 alternative definition of conditional entropy
hoelzl [Wed, 10 Oct 2012 12:12:28 +0200] rev 49791
alternative definition of conditional entropy
Wed, 10 Oct 2012 12:12:27 +0200 remove unneeded assumption from conditional_entropy_generic_eq
hoelzl [Wed, 10 Oct 2012 12:12:27 +0200] rev 49790
remove unneeded assumption from conditional_entropy_generic_eq
Wed, 10 Oct 2012 12:12:27 +0200 add induction rule for intersection-stable sigma-sets
hoelzl [Wed, 10 Oct 2012 12:12:27 +0200] rev 49789
add induction rule for intersection-stable sigma-sets
Wed, 10 Oct 2012 12:12:26 +0200 show and use distributed_swap and distributed_jointI
hoelzl [Wed, 10 Oct 2012 12:12:26 +0200] rev 49788
show and use distributed_swap and distributed_jointI
Wed, 10 Oct 2012 12:12:25 +0200 rule to show that conditional mutual information is non-negative in the continuous case
hoelzl [Wed, 10 Oct 2012 12:12:25 +0200] rev 49787
rule to show that conditional mutual information is non-negative in the continuous case
Wed, 10 Oct 2012 12:12:25 +0200 continuous version of entropy_le
hoelzl [Wed, 10 Oct 2012 12:12:25 +0200] rev 49786
continuous version of entropy_le
Wed, 10 Oct 2012 12:12:24 +0200 simplified entropy_uniform
hoelzl [Wed, 10 Oct 2012 12:12:24 +0200] rev 49785
simplified entropy_uniform
Wed, 10 Oct 2012 12:12:23 +0200 remove incseq assumption from measure_eqI_generator_eq
hoelzl [Wed, 10 Oct 2012 12:12:23 +0200] rev 49784
remove incseq assumption from measure_eqI_generator_eq
Wed, 10 Oct 2012 12:12:23 +0200 generalize from prob_space to finite_measure
hoelzl [Wed, 10 Oct 2012 12:12:23 +0200] rev 49783
generalize from prob_space to finite_measure
Wed, 10 Oct 2012 12:12:22 +0200 add measurable_compose
hoelzl [Wed, 10 Oct 2012 12:12:22 +0200] rev 49782
add measurable_compose
Wed, 10 Oct 2012 12:12:21 +0200 simplified assumptions for kolmogorov_0_1_law
hoelzl [Wed, 10 Oct 2012 12:12:21 +0200] rev 49781
simplified assumptions for kolmogorov_0_1_law
Wed, 10 Oct 2012 12:12:21 +0200 merge should operate on pairs
hoelzl [Wed, 10 Oct 2012 12:12:21 +0200] rev 49780
merge should operate on pairs
Wed, 10 Oct 2012 12:12:20 +0200 remove incseq assumption from sigma_prod_algebra_sigma_eq
hoelzl [Wed, 10 Oct 2012 12:12:20 +0200] rev 49779
remove incseq assumption from sigma_prod_algebra_sigma_eq
Wed, 10 Oct 2012 12:12:19 +0200 sigma_finite_iff_density_finite does not require a positive density function
hoelzl [Wed, 10 Oct 2012 12:12:19 +0200] rev 49778
sigma_finite_iff_density_finite does not require a positive density function
Wed, 10 Oct 2012 12:12:18 +0200 tuned Lebesgue measure proofs
hoelzl [Wed, 10 Oct 2012 12:12:18 +0200] rev 49777
tuned Lebesgue measure proofs
Wed, 10 Oct 2012 12:12:18 +0200 tuned product measurability
hoelzl [Wed, 10 Oct 2012 12:12:18 +0200] rev 49776
tuned product measurability
Wed, 10 Oct 2012 12:12:17 +0200 remove some unneeded positivity assumptions; generalize some assumptions to AE; tuned proofs
hoelzl [Wed, 10 Oct 2012 12:12:17 +0200] rev 49775
remove some unneeded positivity assumptions; generalize some assumptions to AE; tuned proofs
Wed, 10 Oct 2012 12:12:16 +0200 use continuity to show Borel-measurability
hoelzl [Wed, 10 Oct 2012 12:12:16 +0200] rev 49774
use continuity to show Borel-measurability
Wed, 10 Oct 2012 12:12:15 +0200 tuned measurable_If; moved countably_additive equalities to Measure_Space; tuned proofs
hoelzl [Wed, 10 Oct 2012 12:12:15 +0200] rev 49773
tuned measurable_If; moved countably_additive equalities to Measure_Space; tuned proofs
Wed, 10 Oct 2012 12:12:14 +0200 rename terminal_events to tail_event
hoelzl [Wed, 10 Oct 2012 12:12:14 +0200] rev 49772
rename terminal_events to tail_event
Wed, 10 Oct 2012 13:04:15 +0200 merged
Andreas Lochbihler [Wed, 10 Oct 2012 13:04:15 +0200] rev 49771
merged
Wed, 10 Oct 2012 13:03:50 +0200 efficient construction of red black trees from sorted associative lists
Andreas Lochbihler [Wed, 10 Oct 2012 13:03:50 +0200] rev 49770
efficient construction of red black trees from sorted associative lists
Wed, 10 Oct 2012 12:52:24 +0200 more explicit code equations
haftmann [Wed, 10 Oct 2012 12:52:24 +0200] rev 49769
more explicit code equations
Wed, 10 Oct 2012 10:48:55 +0200 adding necessary syntactic functions in set_comprehension_pointfree simproc as a first step to integrate an improved simproc
bulwahn [Wed, 10 Oct 2012 10:48:55 +0200] rev 49768
adding necessary syntactic functions in set_comprehension_pointfree simproc as a first step to integrate an improved simproc
Wed, 10 Oct 2012 10:48:33 +0200 special code setup for step function in IMP is redundant as definition was tuned (cf. c54d901d2946)
bulwahn [Wed, 10 Oct 2012 10:48:33 +0200] rev 49767
special code setup for step function in IMP is redundant as definition was tuned (cf. c54d901d2946)
Wed, 10 Oct 2012 10:48:17 +0200 test case for set_comprehension_pointfree simproc succeeds now
bulwahn [Wed, 10 Oct 2012 10:48:17 +0200] rev 49766
test case for set_comprehension_pointfree simproc succeeds now
Wed, 10 Oct 2012 10:47:52 +0200 unfolding bounded existential quantifiers as first step in the set_comprehension_pointfree simproc
bulwahn [Wed, 10 Oct 2012 10:47:52 +0200] rev 49765
unfolding bounded existential quantifiers as first step in the set_comprehension_pointfree simproc
Wed, 10 Oct 2012 10:47:43 +0200 moving simproc from Finite_Set to more appropriate Product_Type theory
bulwahn [Wed, 10 Oct 2012 10:47:43 +0200] rev 49764
moving simproc from Finite_Set to more appropriate Product_Type theory
Wed, 10 Oct 2012 10:47:21 +0200 generalizing set_comprehension_pointfree simproc to work for arbitrary predicates (and not just the finite predicate)
bulwahn [Wed, 10 Oct 2012 10:47:21 +0200] rev 49763
generalizing set_comprehension_pointfree simproc to work for arbitrary predicates (and not just the finite predicate)
Wed, 10 Oct 2012 10:41:18 +0200 adding some example that motivates some of the current changes in the set_comprehension_pointfree simproc
bulwahn [Wed, 10 Oct 2012 10:41:18 +0200] rev 49762
adding some example that motivates some of the current changes in the set_comprehension_pointfree simproc
Wed, 10 Oct 2012 10:41:16 +0200 set_comprehension_pointfree also handles terms where the equation is not at the first position, which is a necessary generalisation to eventually handle bounded existentials; tuned
bulwahn [Wed, 10 Oct 2012 10:41:16 +0200] rev 49761
set_comprehension_pointfree also handles terms where the equation is not at the first position, which is a necessary generalisation to eventually handle bounded existentials; tuned
Wed, 10 Oct 2012 08:45:27 +0200 more consistent error messages on malformed code equations
haftmann [Wed, 10 Oct 2012 08:45:27 +0200] rev 49760
more consistent error messages on malformed code equations
Tue, 09 Oct 2012 17:33:46 +0200 removed support for set constant definitions in HOLCF {cpo,pcpo,domain}def commands;
huffman [Tue, 09 Oct 2012 17:33:46 +0200] rev 49759
removed support for set constant definitions in HOLCF {cpo,pcpo,domain}def commands; removed '(open)', '(set_name)' and '(open set_name)' options
Tue, 09 Oct 2012 16:58:36 +0200 use Set.filter instead of Finite_Set.filter, which is removed then
kuncar [Tue, 09 Oct 2012 16:58:36 +0200] rev 49758
use Set.filter instead of Finite_Set.filter, which is removed then
Tue, 09 Oct 2012 16:57:58 +0200 rename Set.project to Set.filter - more appropriate name
kuncar [Tue, 09 Oct 2012 16:57:58 +0200] rev 49757
rename Set.project to Set.filter - more appropriate name
Wed, 10 Oct 2012 15:39:01 +0200 added some ad-hoc namespace prefixes to avoid duplicate facts;
wenzelm [Wed, 10 Oct 2012 15:39:01 +0200] rev 49756
added some ad-hoc namespace prefixes to avoid duplicate facts;
Wed, 10 Oct 2012 15:27:10 +0200 avoid duplicate facts;
wenzelm [Wed, 10 Oct 2012 15:27:10 +0200] rev 49755
avoid duplicate facts;
Wed, 10 Oct 2012 15:21:26 +0200 more explicit namespace prefix for 'statespace' -- duplicate facts;
wenzelm [Wed, 10 Oct 2012 15:21:26 +0200] rev 49754
more explicit namespace prefix for 'statespace' -- duplicate facts;
Wed, 10 Oct 2012 15:17:40 +0200 eliminated spurious fact duplicates;
wenzelm [Wed, 10 Oct 2012 15:17:40 +0200] rev 49753
eliminated spurious fact duplicates;
Wed, 10 Oct 2012 15:01:20 +0200 modernized dynamic "rules" -- avoid rebinding of static facts;
wenzelm [Wed, 10 Oct 2012 15:01:20 +0200] rev 49752
modernized dynamic "rules" -- avoid rebinding of static facts;
Tue, 09 Oct 2012 22:24:24 +0200 removed redundant lemma, cf. class zero_neq_one in HOL/Rings.thy;
wenzelm [Tue, 09 Oct 2012 22:24:24 +0200] rev 49751
removed redundant lemma, cf. class zero_neq_one in HOL/Rings.thy;
Tue, 09 Oct 2012 21:33:12 +0200 clarified Element.init vs. Element.activate: refrain from hard-wiring Thm.def_binding_optional to avoid duplicate facts;
wenzelm [Tue, 09 Oct 2012 21:33:12 +0200] rev 49750
clarified Element.init vs. Element.activate: refrain from hard-wiring Thm.def_binding_optional to avoid duplicate facts;
Tue, 09 Oct 2012 20:23:58 +0200 tuned;
wenzelm [Tue, 09 Oct 2012 20:23:58 +0200] rev 49749
tuned;
Tue, 09 Oct 2012 20:05:17 +0200 clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional;
wenzelm [Tue, 09 Oct 2012 20:05:17 +0200] rev 49748
clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional; clarified Generic_Target.define: avoid duplicate def binding via Local_Defs.add_def;
Tue, 09 Oct 2012 19:24:19 +0200 more explicit flags for facts table;
wenzelm [Tue, 09 Oct 2012 19:24:19 +0200] rev 49747
more explicit flags for facts table;
Tue, 09 Oct 2012 15:31:45 +0200 minor tuning;
wenzelm [Tue, 09 Oct 2012 15:31:45 +0200] rev 49746
minor tuning;
Tue, 09 Oct 2012 13:57:51 +0200 more conventional Double constants;
wenzelm [Tue, 09 Oct 2012 13:57:51 +0200] rev 49745
more conventional Double constants;
Tue, 09 Oct 2012 13:50:24 +0200 tuned source structure;
wenzelm [Tue, 09 Oct 2012 13:50:24 +0200] rev 49744
tuned source structure;
Tue, 09 Oct 2012 13:29:43 +0200 tuned;
wenzelm [Tue, 09 Oct 2012 13:29:43 +0200] rev 49743
tuned;
Tue, 09 Oct 2012 13:27:52 +0200 tuned;
wenzelm [Tue, 09 Oct 2012 13:27:52 +0200] rev 49742
tuned;
Tue, 09 Oct 2012 11:51:06 +0200 merged
wenzelm [Tue, 09 Oct 2012 11:51:06 +0200] rev 49741
merged
Tue, 09 Oct 2012 00:40:33 +0200 added type annotations to generated Isar proofs -- code by Steffen Smolka
blanchet [Tue, 09 Oct 2012 00:40:33 +0200] rev 49740
added type annotations to generated Isar proofs -- code by Steffen Smolka
Mon, 08 Oct 2012 12:03:49 +0200 consolidated names of theorems on composition;
haftmann [Mon, 08 Oct 2012 12:03:49 +0200] rev 49739
consolidated names of theorems on composition; generalized former theorem UN_o; comp_assoc orients to the right, as is more common
Mon, 08 Oct 2012 11:37:03 +0200 corrected NEWS
haftmann [Mon, 08 Oct 2012 11:37:03 +0200] rev 49738
corrected NEWS
Mon, 08 Oct 2012 23:29:07 +0200 avoid somewhat heavy rebuilding of SortedMap via map where plain iteration is sufficient;
wenzelm [Mon, 08 Oct 2012 23:29:07 +0200] rev 49737
avoid somewhat heavy rebuilding of SortedMap via map where plain iteration is sufficient; more elementary level_list: avoid stack overflow; prefer elementary graph operations; tuned;
Mon, 08 Oct 2012 21:17:20 +0200 clarified long_names -- conform to usual Isabelle practice of not analysing internal names;
wenzelm [Mon, 08 Oct 2012 21:17:20 +0200] rev 49736
clarified long_names -- conform to usual Isabelle practice of not analysing internal names;
Mon, 08 Oct 2012 20:39:57 +0200 more precise repaint and revalidate -- the latter is important to keep in sync with content update;
wenzelm [Mon, 08 Oct 2012 20:39:57 +0200] rev 49735
more precise repaint and revalidate -- the latter is important to keep in sync with content update;
Mon, 08 Oct 2012 14:49:04 +0200 tuned;
wenzelm [Mon, 08 Oct 2012 14:49:04 +0200] rev 49734
tuned;
Mon, 08 Oct 2012 14:10:38 +0200 prefer synchronous Mutator_Event.Bus on Swing_Thread;
wenzelm [Mon, 08 Oct 2012 14:10:38 +0200] rev 49733
prefer synchronous Mutator_Event.Bus on Swing_Thread;
Mon, 08 Oct 2012 13:20:55 +0200 more direct tooltip content;
wenzelm [Mon, 08 Oct 2012 13:20:55 +0200] rev 49732
more direct tooltip content;
Mon, 08 Oct 2012 12:54:00 +0200 tuned;
wenzelm [Mon, 08 Oct 2012 12:54:00 +0200] rev 49731
tuned;
Mon, 08 Oct 2012 12:40:35 +0200 use Pretty_Tooltip for Graphview_Panel;
wenzelm [Mon, 08 Oct 2012 12:40:35 +0200] rev 49730
use Pretty_Tooltip for Graphview_Panel; tuned signature;
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip