History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Lazy_Sequence.thy
Revision Date Author Comments
# 1901affb 18-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


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

modernized header uniformly as section;


# 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'


# b3e5b66d 04-May-2014 blanchet <none@none>

renamed 'xxx_size' to 'size_xxx' for old datatype package


# 0811cf40 23-Apr-2014 blanchet <none@none>

move size hooks together, with new one preceding old one and sharing same theory data


# dd44ffb4 20-Feb-2014 blanchet <none@none>

adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'


# 447c00c8 13-Feb-2014 blanchet <none@none>

merged 'Option.map' and 'Option.map_option'


# 34a0be19 12-Feb-2014 blanchet <none@none>

adapted theories to 'xxx_case' to 'case_xxx'
* * *
'char_case' -> 'case_char' and same for 'rec'
* * *
compile
* * *
renamed 'xxx_case' to 'case_xxx'


# a6c1110f 12-Feb-2014 blanchet <none@none>

adapted theories to '{case,rec}_{list,option}' names


# 5a8927d0 15-Feb-2013 haftmann <none@none>

two target language numeral types: integer and natural, as replacement for code_numeral;
former theory HOL/Library/Code_Numeral_Types replaces HOL/Code_Numeral;
refined stack of theories implementing int and/or nat by target language numerals;
reduced number of target language numeral types to exactly one

--HG--
extra : rebase_source : ffa0242ad108fe680ff144a716257c0784285d17


# 8e65386b 14-Feb-2013 haftmann <none@none>

reform of predicate compiler / quickcheck theories:
implement yieldn operations uniformly on the ML level -- predicate compiler uses negative integers as parameter to yieldn, whereas code_numeral represents natural numbers!
avoid odd New_ prefix by joining related theories;
avoid overcompact name DSequence;
separated predicate inside random monad into separate theory;
consolidated name of theory Quickcheck

--HG--
rename : src/HOL/DSequence.thy => src/HOL/Limited_Sequence.thy
rename : src/HOL/Quickcheck.thy => src/HOL/Quickcheck_Random.thy
extra : rebase_source : b6adaac1637d6d1cc809d2f937ae890fcc21969c


# 891cc9a4 12-Nov-2012 haftmann <none@none>

tuned import order


# 7cf37f77 20-Oct-2011 bulwahn <none@none>

modernizing predicate_compile_quickcheck


# 0d0a8a60 30-Mar-2011 bulwahn <none@none>

renewing specifications in HOL: replacing types by type_synonym


# 29ea4817 21-Oct-2010 hoelzl <none@none>

Changed section title to please LaTeX.


# cc1f8dab 21-Oct-2010 bulwahn <none@none>

added generator_dseq compilation for a sound depth-limited compilation with small value generators


# 972f5d58 27-Aug-2010 haftmann <none@none>

renamed class/constant eq to equal; tuned some instantiations


# 3c1b8ad5 12-May-2010 huffman <none@none>

use 'subsection' instead of 'section', to maintain 1 chapter per file in generated document


# aabd3797 29-Apr-2010 haftmann <none@none>

dropped unnecessary ML code


# cd0a069b 28-Apr-2010 haftmann <none@none>

export somehow odd mapa explicitly


# 199efb39 28-Apr-2010 haftmann <none@none>

avoid code_datatype antiquotation


# 82fe7ca2 16-Apr-2010 wenzelm <none@none>

replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;


# 508e5844 31-Mar-2010 bulwahn <none@none>

adding iterate_upto interface in compilations and iterate_upto functions in Isabelle theories for arithmetic setup of the predicate compiler


# 69c0ba8b 29-Mar-2010 bulwahn <none@none>

adding Lazy_Sequences with explicit depth-bound


# 2cba73c7 29-Mar-2010 bulwahn <none@none>

removed yieldn in Lazy_Sequence and put in the ML structure; corrects behaviour of values command


# 6d339a77 29-Mar-2010 bulwahn <none@none>

adding values command for new monad; added new random monad compilation to predicate_compile_quickcheck


# bd8108d5 22-Jan-2010 bulwahn <none@none>

correctly hiding facts of Lazy_Sequence


# 2456c710 20-Jan-2010 bulwahn <none@none>

refactoring the predicate compiler; adding theories for Sequences; adding retrieval to Spec_Rules; adding timing to Quickcheck