bulwahn [Fri, 03 Dec 2010 08:40:46 +0100] rev 40898
changed order of lemmas to overwrite the general code equation with the nbe-specific one
hoelzl [Fri, 03 Dec 2010 00:36:01 +0100] rev 40897
adapt proofs to changed set_plus_image (cf. ee8d0548c148);
wenzelm [Fri, 03 Dec 2010 17:16:53 +0100] rev 40896
bash wrapper: terminate only in exceptional case, keep background processes running (e.g. 'thy_deps' or 'display_drafts');
wenzelm [Fri, 03 Dec 2010 16:39:07 +0100] rev 40895
updated latex dependencies (cf. 7d88ebdce380);
wenzelm [Fri, 03 Dec 2010 11:21:17 +0100] rev 40894
tuned README;
wenzelm [Thu, 02 Dec 2010 23:09:54 +0100] rev 40893
isabellesym.sty: eliminated dependency on latin1, to allow documents using utf8 instead;
wenzelm [Thu, 02 Dec 2010 21:23:56 +0100] rev 40892
proper theory name (cf. e84f82418e09);
wenzelm [Thu, 02 Dec 2010 21:04:20 +0100] rev 40891
merged;
huffman [Thu, 02 Dec 2010 11:18:44 -0800] rev 40890
merged
huffman [Wed, 01 Dec 2010 20:52:16 -0800] rev 40889
tuned cpodef code
huffman [Wed, 01 Dec 2010 20:29:39 -0800] rev 40888
reformulate lemma preorder.ex_ideal, and use it for typedefs
hoelzl [Thu, 02 Dec 2010 16:45:28 +0100] rev 40887
Prove rel_interior_convex_hull_union (by Grechuck Bogdan).
haftmann [Thu, 02 Dec 2010 16:39:15 +0100] rev 40886
merged
haftmann [Thu, 02 Dec 2010 16:39:07 +0100] rev 40885
adapted expected value to more idiomatic numeral representation
haftmann [Thu, 02 Dec 2010 14:34:38 +0100] rev 40884
corrected representation for code_numeral numerals
haftmann [Thu, 02 Dec 2010 13:53:36 +0100] rev 40883
separate term_of function for integers -- more canonical representation of negative integers
hoelzl [Thu, 02 Dec 2010 16:17:01 +0100] rev 40882
merged
hoelzl [Thu, 02 Dec 2010 16:16:18 +0100] rev 40881
Use coercions in Approximation (by Dmitriy Traytel).
wenzelm [Thu, 02 Dec 2010 17:20:34 +0100] rev 40880
more antiquotations;
removed some slightly outdated text;
wenzelm [Thu, 02 Dec 2010 16:52:52 +0100] rev 40879
configuration option "show_abbrevs" supersedes print mode "no_abbrevs", with inverted meaning;
wenzelm [Thu, 02 Dec 2010 16:04:22 +0100] rev 40878
renamed trace_simp to simp_trace, and debug_simp to simp_debug;
wenzelm [Thu, 02 Dec 2010 15:37:32 +0100] rev 40877
merged
hoelzl [Thu, 02 Dec 2010 15:32:48 +0100] rev 40876
merged
hoelzl [Thu, 02 Dec 2010 15:09:02 +0100] rev 40875
generalized simple_functionD
hoelzl [Thu, 02 Dec 2010 14:57:50 +0100] rev 40874
Moved theorems to appropriate place.
hoelzl [Thu, 02 Dec 2010 14:57:21 +0100] rev 40873
Shorter definition for positive_integral.
hoelzl [Thu, 02 Dec 2010 14:34:58 +0100] rev 40872
Move SUP_commute, SUP_less_iff to HOL image;
Cleanup generic complete_lattice lemmas in Positive_Infinite_Real;
Cleanup lemma positive_integral_alt;
hoelzl [Wed, 01 Dec 2010 21:03:02 +0100] rev 40871
Generalized simple_functionD and less_SUP_iff.
Moved theorems to appropriate places.
hoelzl [Wed, 01 Dec 2010 20:12:53 +0100] rev 40870
Tuned setup for borel_measurable with min, max and psuminf.
hoelzl [Wed, 01 Dec 2010 20:09:41 +0100] rev 40869
Replace algebra_eqI by algebra.equality;
Move sets_sigma_subset to Sigma_Algebra;
blanchet [Thu, 02 Dec 2010 14:56:16 +0100] rev 40868
give the Isabelle proof the benefice of the doubt when the Isabelle theorem has fewer literals than the Metis one -- this makes a difference on lemma "Let (x::'a, y::'a) (inv_image (r::'b * 'b => bool) (f::'a => 'b)) = ((f x, f y) : r)" apply (metis in_inv_image mem_def)
wenzelm [Thu, 02 Dec 2010 15:03:21 +0100] rev 40867
merged