wenzelm [Fri, 03 Dec 2010 17:59:13 +0100] rev 40939
setup subtyping/coercions once in HOL.thy, but enable it only later via configuration option;
traytel [Thu, 02 Dec 2010 21:48:36 +0100] rev 40938
use "fold_map" instead of "fold (fn .. => .. (ts @ [t], ..)) .."
wenzelm [Fri, 03 Dec 2010 17:31:27 +0100] rev 40937
updated generated file;
wenzelm [Fri, 03 Dec 2010 17:29:27 +0100] rev 40936
removed confusing comments (cf. 500171e7aa59);
wenzelm [Fri, 03 Dec 2010 17:18:41 +0100] rev 40935
merged
haftmann [Fri, 03 Dec 2010 14:00:55 +0100] rev 40934
removed outdated lint script
blanchet [Fri, 03 Dec 2010 10:43:09 +0100] rev 40933
merged
blanchet [Fri, 03 Dec 2010 10:28:39 +0100] rev 40932
compile
blanchet [Fri, 03 Dec 2010 09:55:45 +0100] rev 40931
run synchronous Auto Tools in parallel
krauss [Fri, 03 Dec 2010 10:17:55 +0100] rev 40930
really fixed comment (cf. 7abeb749ae99)
huffman [Fri, 03 Dec 2010 10:03:13 +0100] rev 40929
theorem names generated by the (rep_)datatype command now have mandatory qualifiers
krauss [Fri, 03 Dec 2010 10:03:10 +0100] rev 40928
eliminated unqualified accesses of datatype facts -- it seems like they all of them were unintended
bulwahn [Fri, 03 Dec 2010 09:58:32 +0100] rev 40927
NEWS
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40926
only instantiate type variable if there exists some in quickcheck
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40925
fixing comment in library
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40924
adapting predicate_compile_quickcheck
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40923
adding a nice definition of Id_on for quickcheck and nitpick
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40922
adding code equation for finiteness of finite types
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40921
improving sledgehammer_tactic and adding relevance filtering to the tactic
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40920
adapting mutabelle
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40919
adapting SML_Quickcheck to recent changes
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40918
explaining quickcheck testers in the documentation
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40917
adapting quickcheck examples
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40916
improving presentation of quickcheck reports
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40915
declaring quickcheck testers as default after their setup
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40914
activating construction of exhaustive testing combinators
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40913
renamed generator into exhaustive
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40912
checking if parameter is name of a tester which allows e.g. quickcheck[random]
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40911
moving iteration of tests to the testers in quickcheck
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40910
removed dead test_term_small function in quickcheck
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40909
renamed parameter from generator to tester; quickcheck only applies one tester on invocation
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40908
adding configuration quickcheck_tester
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40907
adding smart quantifiers to exhaustive testing
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40906
adapting mutabelle
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40905
only handle TimeOut exception if used interactively
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40904
removed interrupt handling that violates Isabelle/ML exception model
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40903
corrected indentation
bulwahn [Fri, 03 Dec 2010 08:40:47 +0100] rev 40902
tuned
bulwahn [Fri, 03 Dec 2010 08:40:46 +0100] rev 40901
smallvalue_generator are defined quick via oracle or sound via function package
bulwahn [Fri, 03 Dec 2010 08:40:46 +0100] rev 40900
adding shorter output syntax for the finite types of quickcheck
bulwahn [Fri, 03 Dec 2010 08:40:46 +0100] rev 40899
improving readability of Smallcheck theory; adding constant orelse to improve performance of the function package
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
nipkow [Thu, 02 Dec 2010 08:34:23 +0100] rev 40866
coercions
nipkow [Wed, 01 Dec 2010 20:59:40 +0100] rev 40865
merged
nipkow [Wed, 01 Dec 2010 20:59:29 +0100] rev 40864
moved activation of coercion inference into RealDef and declared function real a coercion.
Made use of it in theory Ln.
hoelzl [Wed, 01 Dec 2010 19:42:09 +0100] rev 40863
Corrected IsaMakefile
hoelzl [Wed, 01 Dec 2010 19:36:05 +0100] rev 40862
merged
hoelzl [Wed, 01 Dec 2010 19:33:49 +0100] rev 40861
Updated NEWS
hoelzl [Wed, 01 Dec 2010 19:27:53 +0100] rev 40860
More correct make dependencies for HOL-Multivariate_Analysis and HOL-Probability.
hoelzl [Wed, 01 Dec 2010 19:20:30 +0100] rev 40859
Support product spaces on sigma finite measures.
Introduce the almost everywhere quantifier.
Introduce 'morphism' theorems for most constants.
Prove uniqueness of measures on cut stable generators.
Prove uniqueness of the Radon-Nikodym derivative.
Removed misleading suffix from borel_space and lebesgue_space.
Use product spaces to introduce Fubini on the Lebesgue integral.
Combine Euclidean_Lebesgue and Lebesgue_Measure.
Generalize theorems about mutual information and entropy to arbitrary probability spaces.
Remove simproc mult_log as it does not work with interpretations.
Introduce completion of measure spaces.
Change type of sigma.
Introduce dynkin systems.
haftmann [Wed, 01 Dec 2010 18:00:40 +0100] rev 40858
merged
haftmann [Wed, 01 Dec 2010 15:46:27 +0100] rev 40857
use type constructor as name for variable
haftmann [Wed, 01 Dec 2010 11:46:20 +0100] rev 40856
optional explicit prefix for type mapper theorems
haftmann [Wed, 01 Dec 2010 11:33:17 +0100] rev 40855
file for package tool type_mapper carries the same name as its Isar command
huffman [Wed, 01 Dec 2010 06:50:54 -0800] rev 40854
merged
huffman [Wed, 01 Dec 2010 06:48:40 -0800] rev 40853
domain package generates non-authentic syntax rules for parsing only
wenzelm [Thu, 02 Dec 2010 10:46:03 +0100] rev 40852
builtin time bounds (again);
wenzelm [Thu, 02 Dec 2010 10:44:33 +0100] rev 40851
tuned;
wenzelm [Wed, 01 Dec 2010 21:23:21 +0100] rev 40850
more abstract handling of Time properties;
wenzelm [Wed, 01 Dec 2010 21:07:50 +0100] rev 40849
store tooltip-dismiss-delay as Double(seconds);
wenzelm [Wed, 01 Dec 2010 20:34:40 +0100] rev 40848
more abstract/uniform handling of time, preferring seconds as Double;
wenzelm [Wed, 01 Dec 2010 15:38:05 +0100] rev 40847
merged
haftmann [Wed, 01 Dec 2010 11:45:37 +0100] rev 40846
NEWS
wenzelm [Wed, 01 Dec 2010 15:35:40 +0100] rev 40845
just one HOLogic.mk_comp;
wenzelm [Wed, 01 Dec 2010 15:03:44 +0100] rev 40844
more direct use of binder_types/body_type;