History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Enum.thy
Revision Date Author Comments
# 69def9ca 26-Mar-2018 Manuel Eberl <eberlm@in.tum.de>

Removed some uses of deprecated _tac methods. (Patch from Viorel Preoteasa)

--HG--
extra : amend_source : fa78190ac2ee02ba33d22a4ee58362bc893ff097


# 965df47d 12-Mar-2018 Manuel Eberl <eberlm@in.tum.de>

Changes to complete distributive lattices due to Viorel Preoteasa


# f5796e6d 14-Feb-2018 wenzelm <none@none>

more symbols;


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

ran isabelle update_op on all sources


# c7cc1919 26-Nov-2017 wenzelm <none@none>

more symbols;


# f93a9d94 09-Oct-2017 haftmann <none@none>

clarified uniqueness criterion for euclidean rings

--HG--
extra : rebase_source : 3f8d28b5e69282e9e5f36f72ad0d4d2e551ca7ab


# fd2471a9 08-Oct-2017 haftmann <none@none>

euclidean rings need no normalization

--HG--
extra : rebase_source : 7f2e3f676b513d6c59f526f099be30240183bf05


# 2ef94418 08-Oct-2017 haftmann <none@none>

abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel

--HG--
extra : rebase_source : c6612d6016d811043143eafb7a671631287494a1


# e0d246a1 29-May-2017 eberlm <eberlm@in.tum.de>

reorganised material on sublists

--HG--
rename : src/HOL/Library/Sublist_Order.thy => src/HOL/Library/Subseq_Order.thy
extra : amend_source : e295fcfca4d0d9db4c5591741cb62b62bb340c87


# 40424ca4 17-Dec-2016 haftmann <none@none>

more fine-grained type class hierarchy for div and mod

--HG--
extra : rebase_source : fffbeef99e834ca17596f478178e94bed8a014bc


# 049952fc 18-Oct-2016 haftmann <none@none>

suitable logical type class for abs, sgn

--HG--
extra : rebase_source : 27e95dd7f038f114d0cad11ec69599a166229041


# 3c2b07e1 25-Sep-2016 haftmann <none@none>

syntactic type class for operation mod named after mod;
simplified assumptions of type class semiring_div

--HG--
extra : rebase_source : 3714be7474835787b2a513b731c9864d1ac9d2c4


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

more canonical names


# 6688eecc 17-Feb-2016 haftmann <none@none>

prefer abbreviations for compound operators INFIMUM and SUPREMUM


# 0df376fc 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


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

tuned proofs -- less legacy;


# 85ed9565 01-Sep-2015 wenzelm <none@none>

eliminated \<Colon>;


# 1901affb 18-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


# 603f8dfb 12-Jun-2015 haftmann <none@none>

uniform _ div _ as infix syntax for ring division

--HG--
extra : rebase_source : c4a1892078772c7ce9af33ad66e2abfefe7adea9


# f2ba2c03 01-Jun-2015 haftmann <none@none>

separate class for division operator, with particular syntax added in more specific classes


# ac517014 31-Mar-2015 haftmann <none@none>

given up separate type classes demanding `inverse 0 = 0`


# 34035ccd 04-Mar-2015 wenzelm <none@none>

tuned signature -- prefer qualified names;


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# 830e17f5 19-Oct-2014 haftmann <none@none>

augmented and tuned facts on even/odd and division


# bb4c3636 13-Oct-2014 wenzelm <none@none>

Local_Interpretation is superseded by Plugin with formal Plugin_Name management, avoiding undeclared strings;


# 5d835e75 10-Oct-2014 haftmann <none@none>

specialized specification: avoid trivial instances


# 1e04f9e5 16-Sep-2014 blanchet <none@none>

added 'extraction' plugins -- this might help 'HOL-Proofs'


# 3c8247b0 14-Sep-2014 blanchet <none@none>

disable datatype 'plugins' for internal types


# 5fc26177 11-Sep-2014 blanchet <none@none>

updated news


# 1ba740de 02-Sep-2014 blanchet <none@none>

use 'datatype_new' in 'Main'


# d22c2cb6 31-Aug-2014 haftmann <none@none>

separated listsum material


# fc5591a9 13-Aug-2014 Andreas Lochbihler <none@none>

add algebraic type class instances for Enum.finite* types


# 562c3021 08-Aug-2014 Andreas Lochbihler <none@none>

add complete_lattice instances for Enum.finite_* types such that quickcheck deals with lattice class operations


# bf47da1c 12-Jun-2014 nipkow <none@none>

added [simp]


# 2fc85925 20-Jan-2014 blanchet <none@none>

moved 'bacc' back to 'Enum' (cf. 744934b818c7) -- reduces baggage loaded by 'Hilbert_Choice'


# e93b90ff 31-Dec-2013 haftmann <none@none>

fundamental treatment of undefined vs. universally partial replaces code_abort


# ade011bf 10-Nov-2013 haftmann <none@none>

qualifed popular user space names


# 6d11884a 18-Oct-2013 blanchet <none@none>

killed more "no_atp"s


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

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


# a7b3de52 23-Jun-2013 haftmann <none@none>

migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier

--HG--
extra : rebase_source : ff8027ac9606264aa4b2d4f8da037c426a3db98b


# 543a4919 16-Dec-2012 bulwahn <none@none>

providing a custom code equation for vimage to overwrite the vimage definition that would be rewritten by set_comprehension_pointfree simproc in the code preprocessor to an non-terminating code equation


# e455b9c3 22-Oct-2012 haftmann <none@none>

incorporated constant chars into instantiation proof for enum;
tuned proofs for properties on enum of chars;
swapped theory dependency of Enum.thy and String.thy


# 808f7fa1 20-Oct-2012 haftmann <none@none>

tailored enum specification towards simple instantiation;
tuned enum instantiations

--HG--
extra : rebase_source : 0b8e3e6fb67c5a5bf29b205ea3072f7927d6dc6b


# 8a46b7d4 20-Oct-2012 haftmann <none@none>

refined internal structure of Enum.thy

--HG--
extra : rebase_source : e1ee78f9065555b71380d5352e73c013e17e11ff


# bbf74aa0 20-Oct-2012 haftmann <none@none>

moved quite generic material from theory Enum to more appropriate places

--HG--
extra : rebase_source : aada8b3ff46b715201e6ecbb53f390c25461ebd9


# f7d71d1b 25-Jun-2012 bulwahn <none@none>

some special code equations for Id with class constraint enum after adding the set comprehension simproc to the code preprocessing


# 63205ab8 30-Mar-2012 wenzelm <none@none>

tuned proofs, less guesswork;


# d54dcfbd 30-Mar-2012 huffman <none@none>

rephrase lemma card_Pow using '2' instead of 'Suc (Suc 0)'


# 278cb2aa 30-Jan-2012 bulwahn <none@none>

adding code equations for max_extp and mlex


# a13eda07 30-Jan-2012 bulwahn <none@none>

adding code equation for rtranclp in Enum


# 40954648 30-Jan-2012 bulwahn <none@none>

adding code equation for max_ext


# ec806846 30-Jan-2012 bulwahn <none@none>

adding code equation for tranclp


# 7dc4f509 27-Jan-2012 bulwahn <none@none>

an executable version of accessible part (only for finite types yet)


# c94eba99 25-Jan-2012 bulwahn <none@none>

evaluation of THE with a non-singleton set raises a Match exception during the evaluation to yield a potential counterexample in quickcheck.


# 5713eadf 25-Jan-2012 bulwahn <none@none>

adding code equation for Collect on finite types


# 2d7f16fb 24-Dec-2011 haftmann <none@none>

enum type class instance for `set`; dropped misfitting code lemma for trancl


# ee736ef6 14-Oct-2011 haftmann <none@none>

moved sublists to More_List.thy


# 5d6d046e 13-Oct-2011 haftmann <none@none>

avoid very specific code equation for card; corrected spelling

--HG--
extra : rebase_source : 7a43ff22845a7caa93989e5f5ab5908190833404


# c5612a1a 13-Oct-2011 haftmann <none@none>

bouned transitive closure

--HG--
extra : rebase_source : 3d0df473619b9c72b32a96ed4951a34dd2ad6c82


# 698b6152 03-Oct-2011 bulwahn <none@none>

tune text for document generation


# 1d55bef4 03-Oct-2011 bulwahn <none@none>

adding code equations for cardinality and (reflexive) transitive closure on finite types


# 2e718ed8 13-Dec-2010 bulwahn <none@none>

adding an executable THE operator on finite types


# 79dccb7a 08-Dec-2010 bulwahn <none@none>

adding a smarter enumeration scheme for finite functions


# bfc5f6a0 08-Dec-2010 bulwahn <none@none>

adding more efficient implementations for quantifiers in Enum


# 41cd8dbf 03-Dec-2010 bulwahn <none@none>

adding shorter output syntax for the finite types of quickcheck


# 3d1f19df 03-Dec-2010 bulwahn <none@none>

changed order of lemmas to overwrite the general code equation with the nbe-specific one


# b4b599e6 24-Nov-2010 bulwahn <none@none>

removing Enum.in_enum from the claset


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

hiding enum


# 05f9b405 22-Nov-2010 bulwahn <none@none>

hiding the constants


# 2b6a6297 22-Nov-2010 bulwahn <none@none>

adding code equations for EX1 on finite types


# 61d17e7b 22-Nov-2010 bulwahn <none@none>

adding code equation for function equality; adding some instantiations for the finite types


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

adding Enum to HOL-Main image and removing it from HOL-Library


# 0e4c5bd7 22-Nov-2010 bulwahn <none@none>

moving Enum theory from HOL/Library to HOL

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