History log of /seL4-l4v-master/isabelle/src/HOL/Library/FuncSet.thy
Revision Date Author Comments
# ec78305b 09-Dec-2019 paulson <lp15@cam.ac.uk>

a few new and tidier proofs (mostly about finite sets)


# 695abc8b 05-Apr-2019 paulson <lp15@cam.ac.uk>

fixes for Free_Abelian_Groups


# b0924e81 21-Mar-2019 paulson <lp15@cam.ac.uk>

new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map


# fbeacd92 22-Jan-2019 paulson <lp15@cam.ac.uk>

some renamings and a bit of new material


# a4bab154 04-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 5abaa1a1 17-Oct-2018 paulson <lp15@cam.ac.uk>

new theory Abstract_Topology with lots of stuff from HOL Light's metric.sml


# 56beb7b9 16-Sep-2018 paulson <lp15@cam.ac.uk>

more lemmas


# cbba6851 28-Jul-2018 paulson <lp15@cam.ac.uk>

de-applying and simplification


# 6437a27a 15-May-2018 wenzelm <none@none>

tuned headers;


# f4f1a444 15-May-2018 immler <none@none>

move FuncSet back to HOL-Library (amending 493b818e8e10)

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


# b985f1a3 05-Nov-2017 wenzelm <none@none>

more uniform header syntax, in contrast to the former etc/abbrevs file-format (see 73939a9b70a3);


# 4ed5daad 04-Nov-2017 wenzelm <none@none>

prefer main entry points of HOL;


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

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


# f1b92889 17-Jan-2017 wenzelm <none@none>

removed some old ASCII syntax;


# 9f786ce6 17-Jan-2017 wenzelm <none@none>

more symbols via abbrevs;


# 1daf8189 13-May-2016 wenzelm <none@none>

eliminated use of empty "assms";


# 5cca9e8d 26-Apr-2016 wenzelm <none@none>

some uses of 'obtain' with structure statement;


# 35f7dccd 23-Feb-2016 nipkow <none@none>

more canonical names


# 0bfb73b6 28-Dec-2015 wenzelm <none@none>

former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";


# 26ece69c 05-Nov-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 6c667f5f 10-Oct-2015 wenzelm <none@none>

prefer symbols;


# 607ae3e3 09-Oct-2015 wenzelm <none@none>

discontinued specific HTML syntax;


# 23d5df30 07-Oct-2015 hoelzl <none@none>

cleanup projective limit of probability distributions; proved Ionescu-Tulcea; used it to prove infinite prob. distribution

--HG--
extra : rebase_source : cffce7b3e322f3c274d9117a0dfdd311d4ba66a1


# 6c7ab2bf 22-Jan-2015 hoelzl <none@none>

import general thms from Density_Compiler

--HG--
extra : rebase_source : 48a3b47f755d8099564008b93076eae81453a674


# 34a3534a 02-Nov-2014 wenzelm <none@none>

modernized header;


# 9ecdf15f 25-Oct-2014 wenzelm <none@none>

tuned whitespace;
more symbols;


# e46f9abe 07-Oct-2014 hoelzl <none@none>

add Giry monad

--HG--
extra : rebase_source : 3ceb1c0fa2e24cb05e37856566255a7b56f80af7


# 4e59d26a 28-Apr-2014 wenzelm <none@none>

tuned;


# fa734f47 12-Nov-2013 hoelzl <none@none>

add restrict_space measure


# d7cd41cb 03-Sep-2013 wenzelm <none@none>

tuned proofs -- less guessing;


# 06329277 13-Aug-2013 wenzelm <none@none>

standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;


# 2e3f9613 18-Nov-2012 hoelzl <none@none>

merge extensional dependent function space from FuncSet with the one in Finite_Product_Measure

--HG--
extra : rebase_source : e65af8d29763871aedf04aed10bdeb869effca0b


# 22db1436 16-Nov-2012 hoelzl <none@none>

move theorems to be more generally useable

--HG--
extra : rebase_source : c1c0d1f5576f4d469d1b4618663774e2f297a214


# a184d6d1 25-Apr-2012 hoelzl <none@none>

moved lemmas to appropriate places


# 8f0477c5 22-Aug-2011 wenzelm <none@none>

reduced warnings;


# b9a84d47 22-Nov-2010 bulwahn <none@none>

adding extensional function spaces to the FuncSet library theory


# 8202096c 20-Sep-2010 nipkow <none@none>

new lemmas


# 5b59da77 13-Sep-2010 nipkow <none@none>

renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI


# bb8268b1 07-Sep-2010 nipkow <none@none>

expand_fun_eq -> ext_iff
expand_set_eq -> set_ext_iff
Naming in line now with multisets


# 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


# a9fd0b04 28-Oct-2009 paulson <none@none>

New theory Probability, which contains a development of measure theory


# 179dc521 22-Oct-2009 nipkow <none@none>

inv_onto -> inv_into


# def242e4 17-Oct-2009 nipkow <none@none>

Inv -> inv_onto, inv abbr. inv_onto UNIV.


# d2641aec 23-Jun-2009 haftmann <none@none>

lemma funcset_id by Jeremy Avigad


# dd547ffe 22-Jun-2009 nipkow <none@none>

fixed name


# af2a4903 22-Jun-2009 nipkow <none@none>

tuned FuncSet


# 04f32252 20-Jun-2009 nipkow <none@none>

tuned


# 99760ce7 19-Jun-2009 nipkow <none@none>

Made Pi_I [simp]


# 589cec35 23-Mar-2009 haftmann <none@none>

Main is (Complex_Main) base entry point in library theories


# 16362266 07-Oct-2008 haftmann <none@none>

arbitrary is undefined


# 0fe266ef 07-Jul-2008 haftmann <none@none>

absolute imports of HOL/*.thy theories


# ef956639 26-Jun-2008 haftmann <none@none>

established Plain theory and image


# f1e8b313 12-Jun-2008 wenzelm <none@none>

removed obsolete skolem declarations -- done by Theory.at_end;


# 59a80dc0 21-Feb-2008 nipkow <none@none>

moved bij_betw from Library/FuncSet to Fun, redistributed some lemmas


# cd65d9bc 16-Nov-2006 wenzelm <none@none>

more robust syntax for definition/abbreviation/notation;


# cbb1a051 07-Nov-2006 wenzelm <none@none>

renamed 'const_syntax' to 'notation';


# 910750ca 28-Sep-2006 wenzelm <none@none>

fixed translations: CONST;


# 4bb80b71 08-Aug-2006 paulson <none@none>

skolem declarations for built-in theorems


# 43295b76 27-May-2006 wenzelm <none@none>

tuned;


# 61bd82ad 16-May-2006 wenzelm <none@none>

tuned concrete syntax -- abbreviation/const_syntax;


# 78ccf652 02-May-2006 wenzelm <none@none>

replaced syntax/translations by abbreviation;


# 40ba3cdf 07-Oct-2005 wenzelm <none@none>

print_translation: does not handle _idtdummy;


# 0fe1d442 18-Aug-2004 nipkow <none@none>

import -> imports


# e61c8d7d 16-Aug-2004 nipkow <none@none>

New theory header syntax.


# 83fd9266 01-Jun-2004 paulson <none@none>

more on bij_betw


# 44293067 19-May-2004 paulson <none@none>

new bij_betw operator


# b4dd8211 14-May-2004 paulson <none@none>

new lemmas


# 840009b7 06-May-2004 wenzelm <none@none>

tuned document;


# cd257618 14-Apr-2004 kleing <none@none>

use more symbols in HTML output


# 55720395 27-Sep-2002 paulson <none@none>

Proof tidying


# d4306e3a 27-Sep-2002 paulson <none@none>

Tidied. New Pi-theorem.


# ae060076 26-Sep-2002 paulson <none@none>

new theory for Pi-sets, restrict, etc.