History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Extraction.thy
Revision Date Author Comments
# 377854d9 09-Apr-2016 wenzelm <none@none>

clarified context;
avoid Unsynchronized.ref;


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

isabelle update_cartouches;


# 4a1c7495 03-May-2015 nipkow <none@none>

swap False to the right in assumptions to be eliminated at the right end


# 35a9a12f 28-Apr-2015 nipkow <none@none>

undid 6d7b7a037e8d


# d4040e09 25-Apr-2015 nipkow <none@none>

new ==> simp rule


# fcac172f 14-Apr-2015 nipkow <none@none>

prepared for more meta-simp rules (by Stefan Berghofer)


# 7b5a8c0d 06-Apr-2015 wenzelm <none@none>

local setup of induction tools, with restricted access to auxiliary consts;
proper antiquotations for formerly inaccessible consts;


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


# bb6f97cc 15-Sep-2014 blanchet <none@none>

'code' is needed for extraction datatype


# 6b777fb4 15-Sep-2014 blanchet <none@none>

generate 'code' attribute only if 'code' plugin is enabled


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

disable datatype 'plugins' for internal types


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

updated news


# 5352b9d3 02-Sep-2014 blanchet <none@none>

use 'datatype_new'


# fb2f6a3a 01-Sep-2014 blanchet <none@none>

renamed modules defining old datatypes, as a step towards having 'datatype_new' take 'datatype's place

--HG--
rename : src/HOL/Datatype.thy => src/HOL/Old_Datatype.thy
rename : src/HOL/Tools/Function/size.ML => src/HOL/Tools/Function/old_size.ML
rename : src/HOL/Tools/Datatype/datatype.ML => src/HOL/Tools/Old_Datatype/old_datatype.ML
rename : src/HOL/Tools/Datatype/datatype_aux.ML => src/HOL/Tools/Old_Datatype/old_datatype_aux.ML
rename : src/HOL/Tools/Datatype/datatype_codegen.ML => src/HOL/Tools/Old_Datatype/old_datatype_codegen.ML
rename : src/HOL/Tools/Datatype/datatype_data.ML => src/HOL/Tools/Old_Datatype/old_datatype_data.ML
rename : src/HOL/Tools/Datatype/datatype_prop.ML => src/HOL/Tools/Old_Datatype/old_datatype_prop.ML
rename : src/HOL/Tools/Datatype/datatype_realizer.ML => src/HOL/Tools/Old_Datatype/old_datatype_realizer.ML
rename : src/HOL/Tools/Datatype/primrec.ML => src/HOL/Tools/Old_Datatype/old_primrec.ML
rename : src/HOL/Tools/Datatype/rep_datatype.ML => src/HOL/Tools/Old_Datatype/old_rep_datatype.ML


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

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


# 0d093612 12-Feb-2014 blanchet <none@none>

transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
* * *
compile
* * *
tuned imports to prevent merge issues in 'Main'


# 869d0a21 30-Jun-2013 wenzelm <none@none>

just one alternative proof syntax, which also works for Proof_Syntax.pretty_proof/Proof_Syntax.read_proof roundtrip;


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

prefer ML_file over old uses;


# 87ce34be 01-Jun-2010 berghofe <none@none>

Adapted to new format of proof terms containing explicit proofs of class membership.


# d16cef73 10-Jan-2010 berghofe <none@none>

Expand proofs of induct_atomize'/rulify'.


# 3809ce74 17-Nov-2009 wenzelm <none@none>

eliminated dead code;


# 1bfc6f86 15-Nov-2009 wenzelm <none@none>

add_expand_thm: explicit indication of is_def instead of fragile heuristic, tuned signature;
explicit extraction_expand vs. extraction_expand_def attribute;


# b391ac6a 04-Mar-2009 nipkow <none@none>

Made Option a separate theory and renamed option_map to Option.map


# 3993a1f9 15-Feb-2009 berghofe <none@none>

Adapted to encoding of sets as predicates.


# 1129d662 15-Nov-2008 wenzelm <none@none>

rewrite_proof: simplified simprocs (no name required);


# ebb725ca 24-Aug-2008 haftmann <none@none>

default replaces arbitrary


# 2dc6d60e 13-Nov-2007 berghofe <none@none>

Added TrueE to extraction_expand.


# 61bc019f 09-Aug-2007 haftmann <none@none>

re-eliminated Option.thy


# 0708bd13 07-Aug-2007 haftmann <none@none>

split off theory Option for benefit of code generator


# 0cd67398 07-Feb-2007 berghofe <none@none>

Added meta_spec to extraction_expand.


# a2bbab74 10-Oct-2006 haftmann <none@none>

added eq_True eq_False True_implies_equals to extraction_expand


# 75fddbe8 19-Jan-2006 wenzelm <none@none>

setup: theory -> theory;


# d68c2afa 23-Dec-2005 wenzelm <none@none>

removed obsolete induct_atomize_old;


# d01a7f2d 21-Dec-2005 wenzelm <none@none>

updated auxiliary facts for induct method;


# e7b1feab 31-Aug-2005 wenzelm <none@none>

refer to theory instead of low-level tsig;


# a7060872 17-Jun-2005 haftmann <none@none>

migrated theory headers to new format


# 693b136f 31-May-2005 wenzelm <none@none>

tuned;


# 3dffd254 13-Feb-2005 skalberg <none@none>

Deleted Library.option type.


# 4aed9d2d 10-Dec-2004 berghofe <none@none>

Realizer for exE now uses let instead of case.


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

import -> imports


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

New theory header syntax.


# 33b1b845 21-Jun-2004 kleing <none@none>

Merged in license change from Isabelle2004


# 2da5d67d 27-Aug-2003 skalberg <none@none>

Prepared for extended identifiers (\<alpha>, etc.)


# db596a37 01-May-2003 berghofe <none@none>

induct_impliesI is now unfolded.


# 7a2f4958 22-Apr-2003 berghofe <none@none>

Tuned realizer for exE rule, to avoid blowup of extracted program.


# d3e78ee5 27-Nov-2002 berghofe <none@none>

Changed format of realizers / correctness proofs.


# 46dc8feb 30-Sep-2002 berghofe <none@none>

Added elim_vars to preprocessor.


# dfebea80 07-Aug-2002 berghofe <none@none>

Removed (now unneeded) declaration of realizers for induction on natural numbers.


# 0959a7ad 05-Aug-2002 berghofe <none@none>

Removed reference to theory NatDef.


# 49c31672 21-Jul-2002 berghofe <none@none>

Added theory for setting up program extraction.