History log of /seL4-l4v-10.1.1/isabelle/src/HOL/Nominal/nominal_atoms.ML
Revision Date Author Comments
# bee57ad5 23-Jun-2016 wenzelm <none@none>

tuned signature;


# 86d79029 30-May-2016 wenzelm <none@none>

allow 'for' fixes for multi_specs;


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

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


# 7f7de75b 18-Jul-2015 wenzelm <none@none>

prefer tactics with explicit context;


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

renamed ML funs


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

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


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

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


# 8cc66666 27-Mar-2015 wenzelm <none@none>

tuned signature;


# f6e927dc 24-Mar-2015 wenzelm <none@none>

clarified case_tac fixes and context;


# b8d56fe6 10-Feb-2015 wenzelm <none@none>

proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
occasionally clarified use of context;


# b68ac3dc 17-Sep-2014 blanchet <none@none>

support (finite values of) codatatypes in Quickcheck


# 8f15946b 11-Sep-2014 blanchet <none@none>

speed up old Nominal by killing type variables


# 2a2a6d06 08-Sep-2014 blanchet <none@none>

ported old Nominal to use new datatypes


# 233dc2cb 08-Sep-2014 blanchet <none@none>

use compatibility layer


# 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


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

tuned structure inclusion


# a3807495 22-Mar-2014 wenzelm <none@none>

more antiquotations;


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


# 0928b2db 18-Apr-2013 wenzelm <none@none>

simplifier uses proper Proof.context instead of historic type simpset;


# 0fe14a59 10-Apr-2013 wenzelm <none@none>

more standard module name Axclass (according to file name);


# 9e4021ad 10-Apr-2013 wenzelm <none@none>

formal proof context for axclass proofs;
avoid global_simpset_of -- refer to simpset of proof context;


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

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


# 43e6bbbc 10-Jan-2012 berghofe <none@none>

Corrected pt_set_inst, added missing cp_set_inst, deleted obsolete
pt_insert_eqvt, pt_set_eqvt, and perm_set_eq


# 8037af38 24-Dec-2011 haftmann <none@none>

treatment of type constructor `set`


# b96f1ad1 13-Dec-2011 wenzelm <none@none>

'datatype' specifications allow explicit sort constraints;
tuned signatures;


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

discontinued obsolete datatype "alt_names";


# 5267fff3 12-Oct-2011 wenzelm <none@none>

modernized structure Induct_Tacs;


# 9281cfaf 03-Sep-2011 haftmann <none@none>

tuned specifications


# 3f5fbd75 03-Sep-2011 haftmann <none@none>

assert Pure equations for theorem references; tuned


# 7ca37425 14-Jan-2011 berghofe <none@none>

Finally removed old primrec package, since Primrec.add_primrec_global
can be used instead.


# d0437948 15-Dec-2010 wenzelm <none@none>

eliminated dead code;


# 308c65f5 20-Sep-2010 wenzelm <none@none>

renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;

--HG--
rename : src/Pure/pure_thy.ML => src/Pure/global_theory.ML


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

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


# 42aff2ea 09-Jun-2010 haftmann <none@none>

tuned quotes, antiquotations and whitespace


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

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


# 71833c27 08-Nov-2009 wenzelm <none@none>

adapted Theory_Data;
tuned;


# 079cde2d 17-Oct-2009 wenzelm <none@none>

eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;


# 75401f7b 15-Oct-2009 wenzelm <none@none>

replaced String.concat by implode;
replaced String.concatWith by space_implode;
replaced (Seq.flat o Seq.map) by Seq.maps;
replaced List.mapPartial by map_filter;
replaced List.concat by flat;
replaced (flat o map) by maps, which produces less garbage;


# d0b33b8e 23-Jun-2009 haftmann <none@none>

tuned interfaces of datatype module


# 16f1fcf4 23-Jun-2009 haftmann <none@none>

add_datatypes does not yield particular rules any longer


# 62a0f4ee 23-Jun-2009 haftmann <none@none>

add_datatype interface yields type names and less rules


# 3351a6d8 21-Jun-2009 haftmann <none@none>

simplified names of common datatype types


# 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


# b6633991 17-Jun-2009 haftmann <none@none>

datatype packages: record datatype_config for configuration flags; less verbose signatures


# 8c61bfe1 06-May-2009 haftmann <none@none>

explicit type_name antiquotations


# 5bc6a8d3 19-Mar-2009 wenzelm <none@none>

proper spacing before ML antiquotations -- note that @ may be part of symbolic ML identifiers;


# 2586c8fb 07-Mar-2009 wenzelm <none@none>

more uniform handling of binding in packages;


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

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


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

Merge.


# ba721cb0 25-Feb-2009 berghofe <none@none>

Added equivariance lemmas for fresh_star.


# ebe1304b 21-Jan-2009 haftmann <none@none>

binding replaces bstring


# af73b126 16-Dec-2008 Christian Urban <urbanc@in.tum.de>

changed the names of insert_eqvt and set_eqvt so that it is clear that they have preconditions


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

cleaned up binding module and related code


# b1945bd8 10-Nov-2008 berghofe <none@none>

Some more functions for accessing information about atoms.


# c590bd51 26-Sep-2008 berghofe <none@none>

Added some more theorems to NominalData.


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

explicit type Name.binding for higher-specification elements;


# 5f90a8a4 26-Aug-2008 urbanc <none@none>

added equivariance lemmas for ex1 and the


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

PureThy: dropped note_thmss_qualified, dropped _i suffix


# 0bd7449d 30-Jun-2008 urbanc <none@none>

added facts to lemma swap_simps and tuned lemma calc_atms


# 2128b92a 14-Jun-2008 wenzelm <none@none>

InductTacs.case_tac: removed obsolete declare, which is now part of Goal.prove;


# c46af099 10-Jun-2008 wenzelm <none@none>

InductTacs.case_tac with proper context and proper declaration of local variable;


# 9dc3ded6 10-Jun-2008 haftmann <none@none>

polished interface of datatype package


# 21d87522 09-Jun-2008 wenzelm <none@none>

adapted case_tac/induct_tac;


# 05adf2fe 07-May-2008 berghofe <none@none>

- Deleted arity proofs for set
- Produce specific instances of theorems insert_eqvt, set_eqvt and perm_set_eq


# 57174c6e 02-May-2008 urbanc <none@none>

added more infrastructure for fresh_star


# 460d6b91 29-Mar-2008 wenzelm <none@none>

eliminated non-linear access to thy1 and thy12c;


# 34b7a9b4 25-Mar-2008 wenzelm <none@none>

removed redundant axiomatizations of XXX_infinite (fact already proven);


# a6513468 19-Mar-2008 wenzelm <none@none>

simplified get_thm(s): back to plain name argument;


# 18d73cff 19-Mar-2008 wenzelm <none@none>

auxiliary dynamic_thm(s) for fact lookup;


# b6f674de 17-Feb-2008 urbanc <none@none>

added eqvt-flag to subseteq-lemma


# c5f3ac4f 15-Jan-2008 haftmann <none@none>

joined theories IntDef, Numeral, IntArith to theory Int


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

added new primrec package


# d338564b 05-Dec-2007 haftmann <none@none>

map_product and fold_product


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


# 308c901d 23-Sep-2007 urbanc <none@none>

changed the representation of atoms to datatypes over nats


# 34311ae0 13-Sep-2007 berghofe <none@none>

Added equivariance lemmas for induct_forall.


# 4959a6a9 05-Sep-2007 urbanc <none@none>

modified proofs so that they are not using claset()


# 16312c38 10-Aug-2007 haftmann <none@none>

ClassPackage renamed to Class


# 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


# 95ee7518 21-Jul-2007 wenzelm <none@none>

tactics: avoid dynamic reference to accidental theory context (via ML_Context.the_context etc.);


# c1259d09 31-May-2007 urbanc <none@none>

introduced symmetric variants of the lemmas for alpha-equivalence


# b04c881c 19-May-2007 haftmann <none@none>

constant op @ now named append


# b62fe892 06-May-2007 wenzelm <none@none>

simplified DataFun interfaces;


# 3ded8aed 25-Apr-2007 narboux <none@none>

add the lemma supp_eqvt and put the right attribute


# 38dae9a5 24-Apr-2007 narboux <none@none>

fixes last commit


# 716b4814 24-Apr-2007 narboux <none@none>

add two lemmas dealing with freshness on permutations.


# 7c964051 23-Apr-2007 urbanc <none@none>

simplified the proof of pt_set_eqvt (as suggested by Randy Pollack)


# 929fd668 20-Apr-2007 haftmann <none@none>

moved axclass module closer to core system


# 1d87c447 15-Apr-2007 urbanc <none@none>

improved the equivariance lemmas for the quantifiers; had to export the lemma eqvt_force_add and eqvt_force_del in the thmdecls


# 00dd9ae3 06-Apr-2007 urbanc <none@none>

deleted remaining instances of swap_simp_a and swap_simp_b (obsolete now)


# f753eee0 07-Apr-2007 urbanc <none@none>

tuned slightly the previous commit


# a3f83b1e 07-Apr-2007 narboux <none@none>

perm_simp can now simplify using the rules (a,b) o a = b and (a,b) o b = a


# 181b33d2 31-Mar-2007 urbanc <none@none>

added pt_bij' to the collection perm_swap and also added abs_perm to the collection of equivariance lemmas


# 1b163bf4 27-Mar-2007 urbanc <none@none>

made the type sets instance of the "cp" type-class


# 678be968 27-Mar-2007 urbanc <none@none>

added extended the lemma for equivariance of freshness


# 228c94bd 06-Mar-2007 urbanc <none@none>

major update of the nominal package; there is now an infrastructure
for equivariance lemmas which eases definitions of nominal functions


# b94628b2 07-Feb-2007 berghofe <none@none>

Adapted to changes in Finite_Set theory.


# 9f120b31 05-Dec-2006 wenzelm <none@none>

removed legacy ML bindings;


# 20a0be49 15-Nov-2006 urbanc <none@none>

replaced exists_fresh lemma with a version formulated with obtains;
old lemma is available as exists_fresh' (still needed in apply-scripts)


# a6517db6 10-Nov-2006 urbanc <none@none>

deleted all uses of sign_of as it's now the identity function


# a8b0cdf4 14-Aug-2006 berghofe <none@none>

Removed non-trivial definitions from calc_atm theorem list.


# 765b616e 21-Jul-2006 haftmann <none@none>

adaption to argument change in primrec_package


# 0f3ed452 11-Jul-2006 webertj <none@none>

replaced mk_listT by HOLogic.listT; trivial whitespace/comment changes


# 76b45c8b 07-Jul-2006 wenzelm <none@none>

Goal.prove_global;


# e127a823 04-Jul-2006 urbanc <none@none>

added simplification rules to the fresh_guess tactic


# 1cdc91e4 04-Jul-2006 urbanc <none@none>

made calc_atm stronger by including some relative
obvious simplification rules


# 2f44ec19 02-Jul-2006 urbanc <none@none>

added more infrastructure for the recursion combinator


# 2eee07e8 15-May-2006 urbanc <none@none>

added the lemmas pt_fresh_aux and pt_fresh_aux_ineq
(they are used in the proof of the strong
induction principle)

added code to nominal_atoms to collect these
lemmas in "fresh_aux" instantiated for each
atom type

deleted the fresh_fun_eqvt from nominal_atoms,
since fresh_fun is not used anymore in the recursion
combinator


# f5316be0 12-May-2006 wenzelm <none@none>

unchecked definitions;


# 0d0ed495 05-May-2006 urbanc <none@none>

added the lemma abs_fun_eq' to the nominal theory,
and also added code to nominal_atoms for generating
the theorem-list alpha'


# 731aeb57 02-May-2006 urbanc <none@none>

added lemma fresh_right, which is useful
in the proof of the recursion combinator


# 51a04c05 30-Apr-2006 wenzelm <none@none>

AxClass.define_class_i;


# a7810547 28-Apr-2006 berghofe <none@none>

Renamed "nominal" theory to "Nominal".


# dfb499c0 27-Apr-2006 berghofe <none@none>

Adapted to new interface of add_axclass_i.


# 60a21256 26-Apr-2006 urbanc <none@none>

isar-keywords.el
- I am not sure what has changed here

nominal.thy
- includes a number of new lemmas (including freshness
and perm_aux things)

nominal_atoms.ML
- no particular changes here

nominal_permeq.ML
- a new version of the decision procedure using
for permutation composition the constant perm_aux

examples
- various adjustments


# 401ae5de 15-Mar-2006 berghofe <none@none>

add_inst_arity_i renamed to prove_arity.


# 4aedc8ac 01-Mar-2006 urbanc <none@none>

added fresh_fun_eqvt theorem to the theorem collection


# cb55365b 26-Feb-2006 urbanc <none@none>

improved the decision-procedure for permutations;
now uses a simproc

FIXME:
the simproc still needs to be adapted for arbitrary
atom types


# d37252ae 24-Feb-2006 berghofe <none@none>

Reverted to old interface of AxClass.add_inst_arity(_i)


# e449e7a5 24-Feb-2006 berghofe <none@none>

Adapted to Florian's recent changes to the AxClass package.


# 12d95b32 23-Jan-2006 krauss <none@none>

Updated to Isabelle 2006-01-23


# 1afef969 22-Jan-2006 urbanc <none@none>

made the change for setup-functions not returning functions
anymore


# bed20105 19-Jan-2006 berghofe <none@none>

Use generic Simplifier.simp_add attribute instead
of Simplifier.simp_add_global.


# e484aa61 10-Jan-2006 urbanc <none@none>

rolled back the last addition since these lemmas were already
in the simpset.


# cc2a5c7b 10-Jan-2006 urbanc <none@none>

added the thms-collection "pt_id" (collection of all pt_<ak>1 lemmas)


# dd1ce565 09-Jan-2006 urbanc <none@none>

added some lemmas to the collection "abs_fresh"

the lemmas are of the form

finite (supp x) ==> (b # [a].x) = (b=a \/ b # x)

previously only lemmas of the form

(b # [a].x) = (b=a \/ b # x)

with the type-constraint that x is finitely supported
were included.


# c745b7f7 07-Jan-2006 urbanc <none@none>

added private datatype nprod (copy of prod) to be
used in the induction rule


# 342cb043 04-Jan-2006 urbanc <none@none>

changed the name of the type "nOption" to "noption".


# d77a556e 19-Dec-2005 urbanc <none@none>

made the changes according to Florian's re-arranging of
tuples (everything up to 19th December).


# bd604388 19-Dec-2005 urbanc <none@none>

added proofs to show that every atom-kind combination
is in the respective finite-support class (now have to
adjust the files according to Florian's changes)


# 6035e5a6 18-Dec-2005 urbanc <none@none>

added thms to perm_compose (so far only composition
theorems were included where the type of the permutation
was equal)


# bdaa2fc0 18-Dec-2005 urbanc <none@none>

tuned one comment


# dffbf33c 18-Dec-2005 urbanc <none@none>

more cleaning up - this time of the cp-instance
proofs


# 99b6c77f 18-Dec-2005 urbanc <none@none>

improved the finite-support proof

added finite support proof for options (I am
surprised that one does not need more fs-proofs;
at the moment only lists, products, units and
atoms are shown to be finitely supported (of
course also every nominal datatype is finitely
supported))

deleted pt_bool_inst - not necessary because discrete
types are treated separately in nominal_atoms


# dd51ff31 18-Dec-2005 urbanc <none@none>

improved the code for showing that a type is
in the pt-axclass (I try to slowly overcome
my incompetence with such ML-code).


# 87469c4c 16-Dec-2005 urbanc <none@none>

added container-lemma fresh_eqvt


(definition: container-lemma contains all instantiations
of a lemma from the general theory)


# c955f9b7 13-Dec-2005 urbanc <none@none>

added a fresh_left lemma that contains all instantiation
for the various atom-types.


# cd2c5db1 09-Dec-2005 urbanc <none@none>

changed the types in accordance with Florian's changes


# 6d9377eb 08-Dec-2005 berghofe <none@none>

Adapted to new type of PureThy.add_defs_i.


# c9a8eb02 05-Dec-2005 urbanc <none@none>

added code to say that discrete types (nat, bool, char)
are instances of cp_*_*.


# 810fc8d7 30-Nov-2005 urbanc <none@none>

added facilities to prove the pt and fs instances
for discrete types


# 5acd82a5 28-Nov-2005 urbanc <none@none>

made some of the theorem look-ups static (by using
thm instead of PureThy.get_thm)


# efa878ce 26-Nov-2005 urbanc <none@none>

finished cleaning up the parts that collect
lemmas (with instantiations) under some
general names


# bcab41c6 07-Nov-2005 urbanc <none@none>

used the function Library.product for the cprod from Stefan


# 9ed55566 02-Nov-2005 berghofe <none@none>

Moved atom stuff to new file nominal_atoms.ML