History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Probability/ex/Dining_Cryptographers.thy
Revision Date Author Comments
# e977f1fa 31-Jan-2019 haftmann <none@none>

proper congruence rule for image operator

--HG--
extra : rebase_source : 71f59936260619419f4d3f7f86d1b930bc771065


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 23d0d04e 11-Sep-2018 paulson <lp15@cam.ac.uk>

A few new results, elimination of duplicates and more use of "pairwise"


# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


# a7ccdf43 10-Jan-2018 nipkow <none@none>

ran isabelle update_op on all sources


# 17bc899d 18-Aug-2017 wenzelm <none@none>

session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;


# a2bc0021 25-Apr-2016 wenzelm <none@none>

eliminated old 'def';
tuned comments;


# 8f4f8db9 15-Apr-2016 hoelzl <none@none>

fix HOL-Probability-ex


# 8e83c9d2 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 5012105f 13-Sep-2015 wenzelm <none@none>

tuned proofs -- less legacy;


# 6f0c89b5 26-Jun-2015 wenzelm <none@none>

tuned whitespace;


# 9fd71573 10-Jun-2014 Thomas Sewell <thomas.sewell@nicta.com.au>

Hypsubst preserves equality hypotheses

Fixes included for various theories affected by this change.

--HG--
extra : rebase_source : b0150e06a14c2821e03208834282be6eca87aae0


# ab027a86 19-May-2014 hoelzl <none@none>

fixed document generation for HOL-Probability


# 7237bdd9 02-Sep-2013 wenzelm <none@none>

tuned proofs -- clarified flow of facts wrt. calculation;


# 11c87ed0 22-Apr-2012 hoelzl <none@none>

reworked Probability theory

--HG--
extra : rebase_source : 04bef352ab6c7feafcf64ecca49fecffac43bb41


# 95291102 13-Mar-2012 wenzelm <none@none>

prefer abs_def over def_raw;


# 33cd0191 28-Feb-2012 wenzelm <none@none>

avoid undeclared variables in let bindings;
tuned proofs;


# f083f9a4 07-Dec-2011 hoelzl <none@none>

remove unnecessary sublocale instantiations in HOL-Probability (for clarity and speedup); remove Infinite_Product_Measure.product_prob_space which was a duplicate of Probability_Measure.product_prob_space


# 74f532bc 01-Dec-2011 hoelzl <none@none>

use list theorems in Dining Cryptographers and Koepf Duermuth Countermeasure


# ad9e459c 11-Sep-2011 nipkow <none@none>

new fastforce replacing fastsimp - less confusing name


# 7f546ab9 19-Jul-2011 hoelzl <none@none>

Rename extreal => ereal

--HG--
rename : src/HOL/Library/Extended_Reals.thy => src/HOL/Library/Extended_Real.thy


# 6c82f941 14-Mar-2011 hoelzl <none@none>

reworked Probability theory: measures are not type restricted to positive extended reals


# 93b9a16c 01-Feb-2011 hoelzl <none@none>

the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
changed syntax for simple_function, simple_integral, positive_integral, integral and RN_deriv.
introduced binder variants for simple_integral, positive_integral and integral.


# 8dce21d4 03-Dec-2010 hoelzl <none@none>

it is known as the extended reals, not the infinite reals

--HG--
rename : src/HOL/Probability/Positive_Infinite_Real.thy => src/HOL/Probability/Positive_Extended_Real.thy


# 481ae947 01-Dec-2010 hoelzl <none@none>

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.

--HG--
rename : src/HOL/Probability/Borel.thy => src/HOL/Probability/Borel_Space.thy


# dd95aa54 02-Sep-2010 hoelzl <none@none>

Updated proofs in Dining Cryptographers theory


# 2eca6769 23-Aug-2010 hoelzl <none@none>

Rewrite the Probability theory.

Introduced pinfreal as real numbers with infinity.
Use pinfreal as value for measures.
Introduces Lebesgue Measure based on the integral in Multivariate Analysis.
Proved Radon Nikodym for arbitrary sigma finite measure spaces.

--HG--
rename : src/HOL/Probability/Lebesgue.thy => src/HOL/Probability/Lebesgue_Integration.thy


# bb4b3c35 03-May-2010 hoelzl <none@none>

Cleanup information theory


# 9a8190f3 07-Apr-2010 hoelzl <none@none>

Added Information theory and Example: dining cryptographers