History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Sum_Type.thy
Revision Date Author Comments
# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


# 8806de60 01-Aug-2016 wenzelm <none@none>

misc tuning and modernization;


# b78a0c93 05-Jul-2016 wenzelm <none@none>

misc tuning and modernization;


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


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

modernized header uniformly as section;


# cb40fd66 11-Sep-2014 blanchet <none@none>

renamed 'rep_datatype' to 'old_rep_datatype' (HOL)


# cc5256c1 04-Sep-2014 blanchet <none@none>

added 'plugins' option to control which hooks are enabled


# 433b1b70 06-Mar-2014 blanchet <none@none>

renamed 'map_sum' to 'sum_map'


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

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


# 04523a1c 19-Feb-2014 blanchet <none@none>

moved 'primrec' up (for real this time) and removed temporary 'old_primrec'


# 3154df20 17-Feb-2014 blanchet <none@none>

renamed old 'primrec' to 'old_primrec' (until the new 'primrec' can be moved above 'Nat' in the theory dependencies)


# 8e6ecc59 13-Feb-2014 blanchet <none@none>

aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax


# 1ae6608b 13-Feb-2014 blanchet <none@none>

renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)


# 2f0985b8 13-Feb-2014 blanchet <none@none>

renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)

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


# 80ec2685 12-Feb-2014 blanchet <none@none>

tuning


# 63970edd 12-Feb-2014 blanchet <none@none>

renamed '{prod,sum,bool,unit}_case' to 'case_...'


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

avoid duplicate 'case' definitions by first looking up 'Ctr_Sugar'


# 4fc86ba9 12-Feb-2014 blanchet <none@none>

se 'wrap_free_constructors' to register 'sum' , 'prod', 'unit', 'bool' with their discriminators/selectors
* * *
cleaner simp/iff sets


# 0363b36f 13-Aug-2013 kuncar <none@none>

move useful lemmas to Main


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

moved quite generic material from theory Enum to more appropriate places

--HG--
extra : rebase_source : aada8b3ff46b715201e6ecbb53f390c25461ebd9


# c82bd4c5 12-Oct-2012 wenzelm <none@none>

discontinued obsolete typedef (open) syntax;


# d8e74f87 30-Nov-2011 wenzelm <none@none>

prefer typedef without extra definition and alternative name;
tuned proofs;


# 54c58a18 18-Oct-2011 huffman <none@none>

hide typedef-generated constants Product_Type.prod and Sum_Type.sum


# 36c8d8b8 11-Jan-2011 haftmann <none@none>

"enriched_type" replaces less specific "type_lifting"

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


# e8a2e703 21-Dec-2010 haftmann <none@none>

tuned type_lifting declarations


# 14dbdf06 06-Dec-2010 haftmann <none@none>

replace `type_mapper` by the more adequate `type_lifting`

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


# 5d2b85fb 18-Nov-2010 haftmann <none@none>

mapper for sum type


# 35b2ff45 29-Oct-2010 nipkow <none@none>

hide Sum_Type.Plus


# 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


# 53a0b22e 01-Jul-2010 haftmann <none@none>

"prod" and "sum" replace "*" and "+" respectively


# 66151938 08-Jun-2010 haftmann <none@none>

tuned quotes, antiquotations and whitespace


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


# 5b069144 04-Dec-2009 haftmann <none@none>

tuned whitespace


# eba49d63 27-Nov-2009 haftmann <none@none>

modernized; dropped ancient constant Part

--HG--
extra : rebase_source : 0faf72a7a9ce8bddd68df34e5b385b26d032c146


# 5f5dc738 25-Nov-2009 haftmann <none@none>

centralized sum type matter in Sum_Type.thy

--HG--
extra : rebase_source : e3b0c15d9ae3766c59620daf0f992723a16b9206


# 6ca1bd25 08-May-2009 nipkow <none@none>

lemmas by Andreas Lochbihler


# 445ef536 27-Dec-2008 krauss <none@none>

removed duplicate sum_case used only by function package;
moved projections;
hide (open)


# b58a4a1b 09-Dec-2008 huffman <none@none>

move lemmas from Numeral_Type.thy to other theories


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

arbitrary is undefined


# df0867de 10-Jun-2008 haftmann <none@none>

rep_datatype command now takes list of constructors as input arguments


# 55f28d65 05-Dec-2007 haftmann <none@none>

simplified infrastructure for code generator operational equality


# 21289a33 06-May-2007 haftmann <none@none>

tuned


# dd0755ae 10-Apr-2007 krauss <none@none>

Moving "FunDef" up in the HOL development graph, since it is independent from "Recdef" and "Datatype" now.


# e0f5e1ab 09-Mar-2007 haftmann <none@none>

*** empty log message ***


# 05c1b8f6 22-Nov-2006 haftmann <none@none>

dropped eq const


# 2002f725 16-Oct-2006 haftmann <none@none>

moved HOL code generator setup to Code_Generator


# facb566c 19-Sep-2006 haftmann <none@none>

added operational equality


# d8bb4109 14-Aug-2006 haftmann <none@none>

simplified code generator setup


# df2fe26f 10-Feb-2006 haftmann <none@none>

improved code generator devarification


# fff82f5e 16-Aug-2005 paulson <none@none>

classical rules must have names for ATP integration


# e4eb1332 06-Aug-2005 nipkow <none@none>

new lemma


# 96006019 09-Dec-2004 paulson <none@none>

converted Sum_Type to new-style theory: Inl, Inr are NO LONGER global


# 383d093b 27-Sep-2001 wenzelm <none@none>

eliminated theories "equalities" and "mono" (made part of "Typedef",
which supercedes "subset");


# ee7fa931 09-Jan-2001 nipkow <none@none>

`` -> and ``` -> ``


# 322ec07c 12-Oct-2000 nipkow <none@none>

*** empty log message ***