2012-06-18 |
Christian Urban |
used ML-antiquotation command_spec for new commands
|
file |
diff |
annotate
|
2012-05-31 |
Christian Urban |
added to the simplifier nominal_datatype.fresh lemmas
|
file |
diff |
annotate
|
2012-04-20 |
Cezary Kaliszyk |
Find remaining rsp theorems and provide them with the quotient definitions
|
file |
diff |
annotate
|
2012-04-20 |
Cezary Kaliszyk |
Declare rsp for permute, permute_bn, alpha_bn together with their definitions instead of TrueI
|
file |
diff |
annotate
|
2012-04-20 |
Cezary Kaliszyk |
Pass proper rsp theorems for constructors and for size
|
file |
diff |
annotate
|
2012-04-10 |
Christian Urban |
updated to latest changes (10 April) to quotient package (lift_raw_const only takes dummy theorem TrueI....in the future this will not work anymore)
|
file |
diff |
annotate
|
2012-03-20 |
Christian Urban |
updated to new Isabelle (20 March)
|
file |
diff |
annotate
|
2012-03-17 |
Christian Urban |
updated to new Isabelle (declared keywords)
|
file |
diff |
annotate
|
2011-12-22 |
Christian Urban |
the default sort for type-variables in nominal specifications is fs; it is automatically addded
|
file |
diff |
annotate
|
2011-12-18 |
Christian Urban |
partially localised the parsing process using functions fron Datatype
|
file |
diff |
annotate
|
2011-12-17 |
Christian Urban |
Started Nominal2-Isabelle2011-1 branch and backported changeset 32abaea424bd
Nominal2-Isabelle2011-1
|
file |
diff |
annotate
|
2011-12-15 |
Christian Urban |
updated to lates changes in the datatype package
|
file |
diff |
annotate
|
2011-12-14 |
Christian Urban |
generated the correct thm-list for showing that qfv are equal to support
|
file |
diff |
annotate
|
2011-12-13 |
Christian Urban |
updated to Isabelle 13 Dec
|
file |
diff |
annotate
|
2011-12-06 |
Christian Urban |
updated to Isabelle 6 Dec (thanks to Odrej Kuncar)
|
file |
diff |
annotate
|
2011-11-03 |
Christian Urban |
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
|
file |
diff |
annotate
|
2011-07-18 |
Christian Urban |
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
|
file |
diff |
annotate
|
2011-07-13 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
2011-07-11 |
Christian Urban |
combinators for local theories and lists
|
file |
diff |
annotate
|
2011-07-08 |
Christian Urban |
some code refactoring
|
file |
diff |
annotate
|
2011-07-07 |
Christian Urban |
code refactoring; introduced a record for raw_dt_info
|
file |
diff |
annotate
|
2011-07-05 |
Christian Urban |
changed bind to binds in specifications; bind will cause trouble with Monad_Syntax
|
file |
diff |
annotate
|
2011-07-05 |
Christian Urban |
exported various FCB-lemmas to a separate file
|
file |
diff |
annotate
|
2011-06-30 |
Christian Urban |
more code refactoring
|
file |
diff |
annotate
|
2011-06-29 |
Christian Urban |
combined distributed data for alpha in alpha_result (partially done)
|
file |
diff |
annotate
|
2011-06-28 |
Christian Urban |
some experiments
|
file |
diff |
annotate
|
2011-06-23 |
Christian Urban |
fixed nasty bug with type variables in nominal_datatypes; this included to be careful with the output of the inductive and function package
|
file |
diff |
annotate
|
2011-06-22 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2011-06-22 |
Christian Urban |
deleted some dead code
|
file |
diff |
annotate
|
2011-06-22 |
Christian Urban |
some rudimentary infrastructure for storing data about nominal datatypes
|
file |
diff |
annotate
|
2011-06-16 |
Christian Urban |
got rid of the boolean flag in the raw_equivariance function
|
file |
diff |
annotate
|
2011-06-15 |
Christian Urban |
added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method
|
file |
diff |
annotate
|
2011-06-07 |
Christian Urban |
cleaned ups a bit the examples with the invariant framework; exported nominal_function_config datatype into separate structure and file
|
file |
diff |
annotate
|
2011-06-07 |
Christian Urban |
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
|
file |
diff |
annotate
|
2011-06-05 |
Christian Urban |
added an option for an invariant (at the moment only a stub)
|
file |
diff |
annotate
|
2011-05-25 |
Christian Urban |
added eq_iff and distinct lemmas of nominal datatypes to the simplifier
|
file |
diff |
annotate
|
2011-05-10 |
Christian Urban |
updated to new Isabelle (> 9 May)
|
file |
diff |
annotate
|
2011-04-19 |
Christian Urban |
updated to snapshot Isabelle 19 April
|
file |
diff |
annotate
|
2011-04-18 |
Christian Urban |
added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
|
file |
diff |
annotate
|
2011-02-28 |
Christian Urban |
split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
|
file |
diff |
annotate
|
2011-01-19 |
Christian Urban |
added Minimal file to test things
|
file |
diff |
annotate
|
2011-01-17 |
Christian Urban |
exported nominal function code to external file
|
file |
diff |
annotate
|
2011-01-07 |
Christian Urban |
derived equivariance for the function graph and function relation
|
file |
diff |
annotate
|
2011-01-06 |
Christian Urban |
a modified function package where, as a test, True has been injected into the compatibility condictions
|
file |
diff |
annotate
|
2011-01-06 |
Christian Urban |
removed debugging code abd introduced a guarded tracing function
|
file |
diff |
annotate
|
2011-01-06 |
Christian Urban |
cleaned up weakening proof and added a version with finit sets
|
file |
diff |
annotate
|
2011-01-06 |
Christian Urban |
made sure the raw datatypes and raw functions do not get any mixfix syntax
|
file |
diff |
annotate
|
2011-01-05 |
Christian Urban |
exported the code into a separate file
|
file |
diff |
annotate
|
2010-12-31 |
Christian Urban |
changed res keyword to set+ for restrictions; comment by a referee
|
file |
diff |
annotate
|
2010-12-31 |
Christian Urban |
added proper case names for all induct and exhaust theorems
|
file |
diff |
annotate
|
2010-12-30 |
Christian Urban |
removed local fix for bug in induction_schema; added setup method for strong inductions
|
file |
diff |
annotate
|
2010-12-28 |
Christian Urban |
automated all strong induction lemmas
|
file |
diff |
annotate
|
2010-12-28 |
Christian Urban |
proper application of induction_schema and strong_exhaust rules; needs local fix in induction_schema.ML
|
file |
diff |
annotate
|
2010-12-26 |
Christian Urban |
generated goals for strong induction theorems.
|
file |
diff |
annotate
|
2010-12-23 |
Christian Urban |
moved all strong_exhaust code to nominal_dt_quot; tuned examples
|
file |
diff |
annotate
|
2010-12-23 |
Christian Urban |
moved generic functions into nominal_library
|
file |
diff |
annotate
|
2010-12-22 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
2010-12-22 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
2010-12-22 |
Christian Urban |
added fold_right which produces the correct term for left-infix operators
|
file |
diff |
annotate
|
2010-12-22 |
Christian Urban |
a bit tuning
|
file |
diff |
annotate
|