History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Code_Evaluation.thy
Revision Date Author Comments
# 3a4a7136 24-Apr-2018 haftmann <none@none>

proper datatype for 8-bit characters


# a7d124d3 05-Jun-2017 haftmann <none@none>

streamlined code setup for fake terms

--HG--
extra : rebase_source : ef86accead7e67a7aee552c92c5306c6bbf34d86


# d6b5ab04 05-Sep-2016 wenzelm <none@none>

clarified modules;

--HG--
rename : src/HOL/Tools/value.ML => src/HOL/Tools/value_command.ML


# ae5c5b60 26-May-2016 haftmann <none@none>

delegate inclusion of required dictionaries to user-space instead of half-working magic


# 53a62d5e 12-Apr-2016 wenzelm <none@none>

Type_Infer.object_logic controls improvement of type inference result;


# 8175ce0f 12-Mar-2016 haftmann <none@none>

model characters directly as range 0..255
* * *
operate on syntax terms rather than asts


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

isabelle update_cartouches -c -t;


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

eliminated \<Colon>;


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

isabelle update_cartouches;


# 103d949b 05-Feb-2015 haftmann <none@none>

slightly more standard code setup for String.literal, with explicit special case in predicate compiler


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


# 0c940374 22-Aug-2014 Andreas Lochbihler <none@none>

add code equation for term_of on integer


# 0655670a 25-Aug-2014 Andreas Lochbihler <none@none>

correct code equation for term_of on integer


# 8a1b76f7 09-May-2014 haftmann <none@none>

dropped term_of obfuscation -- not really required;
tuned theory structure


# a8dfe60c 09-May-2014 haftmann <none@none>

hardcoded nbe and sml into value command


# 3af0b49a 09-May-2014 haftmann <none@none>

modernized setups


# 956343f7 09-May-2014 haftmann <none@none>

degeneralized value command into HOL

--HG--
rename : src/Tools/value.ML => src/HOL/Tools/value.ML


# 81d6c2a2 21-Mar-2014 wenzelm <none@none>

more qualified names;


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

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


# 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


# de8113c2 01-Jun-2013 haftmann <none@none>

make reification part of HOL

--HG--
rename : src/HOL/Tools/reflection.ML => src/HOL/Tools/reification.ML
extra : rebase_source : 16e93aafd01e25dc85b597f0e457983c2b9cfe1b


# ffcd6989 25-May-2013 wenzelm <none@none>

syntax translations always depend on context;


# 963a5558 15-Feb-2013 haftmann <none@none>

systematic conversions between nat and nibble/char;
more uniform approaches to execute operations on nibble/char

--HG--
extra : rebase_source : 982810ecce9e31070e2293715ed744c3b68ae21d


# cbe9d601 15-Feb-2013 haftmann <none@none>

less customary term_of conversions;
spurious side effect on method reflection

--HG--
extra : rebase_source : e98673d202c69d48235f67e609bfe8d39d2ec105


# 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


# fa22b8b3 13-Feb-2013 haftmann <none@none>

abandoned theory Plain

--HG--
extra : rebase_source : 6f5a395a55e8879386d1f79ab252c6fc2aca7dc5


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

tuned import order


# e3227796 22-Aug-2012 wenzelm <none@none>

prefer ML_file over old uses;


# 8bb6233a 25-Mar-2012 huffman <none@none>

merged fork with new numeral representation (see NEWS)


# 484c9d58 24-Feb-2012 haftmann <none@none>

moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy

--HG--
extra : rebase_source : ed15629634477aff0a8efea30547f496c70907ad


# 37822d49 23-Feb-2012 haftmann <none@none>

moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy


# ad000439 26-May-2011 bulwahn <none@none>

extending terms of Code_Evaluation by Free to allow partial terms


# 467fcb61 02-Dec-2010 haftmann <none@none>

corrected representation for code_numeral numerals


# 7ca617b6 02-Dec-2010 haftmann <none@none>

separate term_of function for integers -- more canonical representation of negative integers


# 7e340696 22-Nov-2010 bulwahn <none@none>

adding dummy definition for Code_Evaluation.Abs and hiding constants App less strict


# 04d3a461 20-Sep-2010 haftmann <none@none>

dynamic_eval_conv static_eval_conv: certification of previously unreliably reconstructed evaluated term


# 4c4b77cf 20-Sep-2010 haftmann <none@none>

Factored out ML into separate file


# c1588037 16-Sep-2010 haftmann <none@none>

adjusted to changes in Code_Runtime


# 20932752 15-Sep-2010 haftmann <none@none>

Code_Runtime.value, corresponding to ML_Context.value


# 67db8f56 15-Sep-2010 haftmann <none@none>

code_eval renamed to code_runtime

--HG--
rename : src/Tools/Code/code_eval.ML => src/Tools/Code/code_runtime.ML


# df7a0e34 15-Sep-2010 haftmann <none@none>

replaced ML_Context.evaluate by ML_Context.value -- using context data instead of bare metal references; tuned structures


# 3c66cf8a 10-Sep-2010 bulwahn <none@none>

fiddling with the correct setup for String.literal


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

renamed class/constant eq to equal; tuned some instantiations


# 512ca872 11-Aug-2010 haftmann <none@none>

moved instantiation target formally to class_target.ML


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


# bbc8cf56 20-Mar-2010 wenzelm <none@none>

renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;


# 74f51502 24-Feb-2010 haftmann <none@none>

evaluation for abstypes


# 9bbce8ca 22-Feb-2010 haftmann <none@none>

proper distinction of code datatypes and abstypes


# f62da38e 07-Dec-2009 haftmann <none@none>

split off evaluation mechanisms in separte module Code_Eval

--HG--
rename : src/Tools/Code/code_ml.ML => src/Tools/Code/code_eval.ML


# 4b04568f 12-Nov-2009 haftmann <none@none>

repaired broken code_const for term_of [String.literal]


# 8ce10e6a 10-Nov-2009 wenzelm <none@none>

modernized structure Theory_Target;


# d0ca4829 06-Nov-2009 bulwahn <none@none>

adding tracing function for evaluated code; annotated compilation in the predicate compiler


# 1e5beb93 29-Sep-2009 wenzelm <none@none>

explicit indication of Unsynchronized.ref;


# 750e49b5 23-Sep-2009 haftmann <none@none>

Code_Eval(uation)

--HG--
rename : src/HOL/Code_Eval.thy => src/HOL/Code_Evaluation.thy