History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Nominal/nominal_primrec.ML
Revision Date Author Comments
# 07cdfca0 13-Aug-2019 wenzelm <none@none>

clarified modules;


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# ea4853ba 28-Jan-2018 wenzelm <none@none>

clarified take/drop/chop prefix/suffix;


# 46bb214d 11-Jun-2016 wenzelm <none@none>

clarified syntax;


# 68f9ecca 28-Apr-2016 wenzelm <none@none>

support 'assumes' in specifications, e.g. 'definition', 'inductive';
tuned signatures;


# 369e4785 13-Dec-2015 wenzelm <none@none>

more general types Proof.method / context_tactic;
proper context for Method.insert_tac;
tuned;


# 2ea85337 26-Jul-2015 wenzelm <none@none>

updated to infer_instantiate;


# 3f438084 10-Apr-2015 blanchet <none@none>

renamed ML funs


# 8a1b73d1 08-Apr-2015 wenzelm <none@none>

tuned signature;


# 4aa541f4 06-Apr-2015 wenzelm <none@none>

@{command_spec} is superseded by @{command_keyword};


# 740a17d4 06-Mar-2015 wenzelm <none@none>

Thm.cterm_of and Thm.ctyp_of operate on local context;


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

tuned signature -- prefer qualified names;


# b7bf58e6 03-Mar-2015 traytel <none@none>

eliminated some clones of Proof_Context.cterm_of


# d6623f99 09-Nov-2014 wenzelm <none@none>

proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);


# 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


# b1da7acd 18-Aug-2014 wenzelm <none@none>

simplified type Proof.method;


# 2c8d6176 21-Mar-2014 wenzelm <none@none>

more qualified names;


# 63a76875 14-Dec-2013 wenzelm <none@none>

proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
clarified tool context in some boundary cases;


# 150d8520 16-Mar-2012 wenzelm <none@none>

outer syntax command definitions based on formal command_spec derived from theory header declarations;


# de9fb383 15-Mar-2012 wenzelm <none@none>

prefer formally checked @{keyword} parser;


# 10581850 14-Jan-2012 wenzelm <none@none>

discontinued old-style Term.list_all_free in favour of plain Logic.all;


# 941cf8eb 02-Dec-2011 wenzelm <none@none>

more antiquotations;


# 8b9f08d0 02-Dec-2011 wenzelm <none@none>

do not open ML structures;


# cfe58b3e 19-Nov-2011 wenzelm <none@none>

added ML antiquotation @{attributes};


# 7b43a234 17-Aug-2011 wenzelm <none@none>

modernized signature of Term.absfree/absdummy;
eliminated obsolete Term.list_abs_free;


# 68ed89ae 10-Aug-2011 wenzelm <none@none>

old term operations are legacy;


# 1a5a42ee 09-Jun-2011 wenzelm <none@none>

simplified Name.variant -- discontinued builtin fold_map;


# ec1196d6 09-Jun-2011 wenzelm <none@none>

discontinued Name.variant to emphasize that this is old-style / indirect;


# 6d2612c8 16-Apr-2011 wenzelm <none@none>

modernized structure Proof_Context;


# f1d76d3c 10-Jan-2011 wenzelm <none@none>

standardized split_last/last_elem towards List.last;
eliminated obsolete Library.last_elem;


# 7a6b0131 17-May-2010 wenzelm <none@none>

prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
eliminated old-style structure aliases K = Keyword, P = Parse;


# f3ff5f68 15-May-2010 wenzelm <none@none>

prefer structure Parse_Spec;


# 14c9715d 25-Apr-2010 wenzelm <none@none>

modernized naming conventions of main Isar proof elements;


# d530d839 10-Feb-2010 berghofe <none@none>

Fixed bug in code for guessing the name of the variable representing the freshness context.


# 1a637a6c 30-Nov-2009 haftmann <none@none>

modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML

--HG--
rename : src/HOL/Tools/Datatype/datatype.ML => src/HOL/Tools/Datatype/datatype_data.ML
extra : rebase_source : 552900fbf6783258465fa5000202d52cf1f99a1f


# 8d32b36e 19-Nov-2009 wenzelm <none@none>

adapted Local_Theory.define -- eliminated odd thm kind;


# 56bf35c4 17-Nov-2009 wenzelm <none@none>

eliminated slightly odd name space grouping -- now managed by Isar toplevel;


# d28e2372 13-Nov-2009 wenzelm <none@none>

modernized structure Local_Theory;


# 21cb7d7d 13-Nov-2009 wenzelm <none@none>

eliminated slightly odd kind argument of LocalTheory.note(s);
added LocalTheory.notes_kind as fall-back for unusual cases;


# 28c1be77 13-Nov-2009 wenzelm <none@none>

eliminated obsolete "generated" kind -- collapsed to unspecific "" (definitely unused according to Lukas Bulwahn);


# d0106d17 29-Oct-2009 wenzelm <none@none>

standardized filter/filter_out;


# 78aa08c8 25-Oct-2009 wenzelm <none@none>

name space groups are identified by serial, not serial_string;


# f56881ab 21-Oct-2009 blanchet <none@none>

renamed "nitpick_const_xxx" attributes to "nitpick_xxx" and "nitpick_ind_intros" to "nitpick_intros"


# d103ca85 21-Oct-2009 haftmann <none@none>

removed old-style \ and \\ infixes


# 8de45ab6 21-Oct-2009 haftmann <none@none>

dropped redundant gen_ prefix


# 68478f6d 20-Oct-2009 haftmann <none@none>

replaced old_style infixes eq_set, subset, union, inter and variants by generic versions


# f1cc0e6d 25-Jul-2009 wenzelm <none@none>

fixed Method.Basic;


# 5371dea8 25-Jul-2009 wenzelm <none@none>

Method.Basic: no position;


# f4ea2464 03-Jul-2009 haftmann <none@none>

nominal.ML is nominal_datatype.ML


# 7b41de27 02-Jul-2009 wenzelm <none@none>

renamed NamedThmsFun to Named_Thms;
simplified/unified names of instances of Named_Thms;


# 91b337ca 19-Jun-2009 haftmann <none@none>

discontinued ancient tradition to suffix certain ML module names with "_package"

--HG--
rename : src/HOL/Import/import_package.ML => src/HOL/Import/import.ML
rename : src/HOL/Nominal/nominal_package.ML => src/HOL/Nominal/nominal.ML
rename : src/HOL/Tools/specification_package.ML => src/HOL/Tools/choice_specification.ML
rename : src/HOL/Tools/datatype_package/datatype_package.ML => src/HOL/Tools/datatype_package/datatype.ML
rename : src/HOL/Tools/function_package/fundef_package.ML => src/HOL/Tools/function_package/fundef.ML
rename : src/HOL/Tools/inductive_package.ML => src/HOL/Tools/inductive.ML
rename : src/HOL/Tools/inductive_set_package.ML => src/HOL/Tools/inductive_set.ML
rename : src/HOL/Tools/old_primrec_package.ML => src/HOL/Tools/old_primrec.ML
rename : src/HOL/Tools/primrec_package.ML => src/HOL/Tools/primrec.ML
rename : src/HOL/Tools/recdef_package.ML => src/HOL/Tools/recdef.ML
rename : src/HOL/Tools/record_package.ML => src/HOL/Tools/record.ML
rename : src/HOL/Tools/typecopy_package.ML => src/HOL/Tools/typecopy.ML
rename : src/HOL/Tools/typedef_package.ML => src/HOL/Tools/typedef.ML


# e9ec6b63 18-May-2009 haftmann <none@none>

introduced Thm.generatedK


# 155bffcd 16-May-2009 bulwahn <none@none>

added new kind generated_theorem for theorems which are generated by packages to distinguish between theorems from users and packages


# 77d6b267 13-Mar-2009 wenzelm <none@none>

unified type Proof.method and pervasive METHOD combinators;


# ab4799d5 12-Mar-2009 wenzelm <none@none>

simplified preparation and outer parsing of specification;
export extern cmd interfaces as well;


# b1ef46dc 08-Mar-2009 wenzelm <none@none>

moved basic algebra of long names from structure NameSpace to Long_Name;


# e3913b9b 04-Mar-2009 wenzelm <none@none>

renamed NameSpace.base to NameSpace.base_name;
renamed NameSpace.map_base to NameSpace.map_base_name;
eliminated alias Sign.base_name = NameSpace.base_name;


# bbeb86b5 04-Mar-2009 blanchet <none@none>

Fix parentheses.


# 43e0e947 04-Mar-2009 blanchet <none@none>

Added "nitpick_const_simp" attribute to Nominal primrec.


# 121e82fb 04-Mar-2009 blanchet <none@none>

Merge.


# 4ad18568 03-Mar-2009 wenzelm <none@none>

renamed Binding.name_pos to Binding.make, renamed Binding.base_name to Binding.name_of, renamed Binding.map_base to Binding.map_name, added mandatory flag to Binding.qualify;
minor tuning;


# 5823ee39 21-Jan-2009 haftmann <none@none>

binding is alias for Binding.T


# 7b9e1a05 31-Dec-2008 wenzelm <none@none>

qualified Term.rename_wrt_term;


# b88342b6 30-Dec-2008 wenzelm <none@none>

moved old add_term_vars, add_term_frees etc. to structure OldTerm;


# 1ff366c9 13-Dec-2008 berghofe <none@none>

Modified nominal_primrec to make it work with local theories, unified syntax
with the one used by fun(ction) and new version of primrec command.


# e331b867 05-Dec-2008 haftmann <none@none>

Name.name_of -> Binding.base_name


# e01ddee4 04-Dec-2008 haftmann <none@none>

cleaned up binding module and related code


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

arbitrary is undefined


# f31abf48 02-Sep-2008 wenzelm <none@none>

explicit type Name.binding for higher-specification elements;


# 4da32258 29-Jul-2008 haftmann <none@none>

PureThy: dropped note_thmss_qualified, dropped _i suffix


# 70a4fc69 18-May-2008 wenzelm <none@none>

moved global pretty/string_of functions from Sign to Syntax;


# aeb882b9 29-Mar-2008 wenzelm <none@none>

eliminated quiete_mode ref (unused);


# 2784bfca 06-Dec-2007 haftmann <none@none>

added new primrec package


# 7748ae93 08-Oct-2007 wenzelm <none@none>

turned keywords invariant/freshness_context into reserved indentifiers;


# 8f12f2a9 06-Oct-2007 wenzelm <none@none>

simplified interfaces for outer syntax;


# 9344c4a9 25-Sep-2007 wenzelm <none@none>

proper Sign operations instead of Theory aliases;


# 61b7a7b9 25-Sep-2007 wenzelm <none@none>

Syntax.parse/check/read;


# 02db772e 30-Aug-2007 wenzelm <none@none>

replaced ProofContext.infer_types by general Syntax.check_terms;


# 1fb89380 11-Jul-2007 berghofe <none@none>

Moved unify_consts to PrimrecPackage.


# b57ed59c 19-Jun-2007 wenzelm <none@none>

balanced conjunctions;


# 5cbc418b 12-Jun-2007 wenzelm <none@none>

Method.Basic: include position;


# 697b02bb 18-May-2007 berghofe <none@none>

Fixed bug in subst causing primrec functions returning functions
to be rejected.


# fc3f51b8 18-Apr-2007 wenzelm <none@none>

simplified ProofContext.infer_types(_pats);


# 10cbbe6c 15-Apr-2007 wenzelm <none@none>

removed obsolete TypeInfer.logicT -- use dummyT;


# 22788088 15-Apr-2007 wenzelm <none@none>

proper ProofContext.infer_types;


# 778678db 10-Mar-2007 berghofe <none@none>

- Replaced fold by fold_rev to make sure that list of predicate
variables pvars (for invariants) is in the correct order
- Adapted to new format of datatype descriptor


# 57c9a7cc 16-Feb-2007 berghofe <none@none>

Replaced "raise RecError" by "primrec_err" in function
gen_primrec_i to prevent error message from being suppressed.


# 1de9c7ae 19-Jan-2007 wenzelm <none@none>

moved parts of OuterParse to SpecParse;


# 8218bc98 11-Dec-2006 berghofe <none@none>

nominal_primrec now prints initial proof state.


# c6555363 01-Dec-2006 nipkow <none@none>

Added missing "standard"


# 33ab6c52 26-Nov-2006 berghofe <none@none>

Implemented new "nominal_primrec" command for defining
functions on nominal datatypes.