2012-03-17 |
Christian Urban |
updated to new Isabelle (declared keywords)
|
file |
diff |
annotate
|
2011-12-21 |
Cezary Kaliszyk |
Port CR_Takahashi from Nominal1, no more "sorry" in BetaCR.
|
file |
diff |
annotate
|
2011-12-17 |
Christian Urban |
cleaned examples for stable branch
Nominal2-Isabelle2011-1
|
file |
diff |
annotate
|
2011-12-15 |
Christian Urban |
updated to lates changes in the datatype package
|
file |
diff |
annotate
|
2011-11-08 |
Cezary Kaliszyk |
Add equivariance for alpha_lam_raw and abs_lam.
|
file |
diff |
annotate
|
2011-11-07 |
Christian Urban |
all examples work again after quotient package has been "de-localised"
|
file |
diff |
annotate
|
2011-08-19 |
Cezary Kaliszyk |
Comment out examples with 'True' that do not work because function still does not work
|
file |
diff |
annotate
|
2011-07-22 |
Christian Urban |
completed the eqvt-proofs for functions; they are stored under the name function_name.eqvt and added to the eqvt-list
|
file |
diff |
annotate
|
2011-07-19 |
Christian Urban |
preliminary version of automatically generation the eqvt-lemmas for functions defined with nominal_primrec
|
file |
diff |
annotate
|
2011-07-19 |
Christian Urban |
generated the partial eqvt-theorem for functions
|
file |
diff |
annotate
|
2011-07-18 |
Christian Urban |
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
|
file |
diff |
annotate
|
2011-07-18 |
Christian Urban |
moved eqvt for Option.map
|
file |
diff |
annotate
|
2011-07-05 |
Christian Urban |
added some relatively simple examples from paper by Norrish
|
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 |
made the tests go through again
|
file |
diff |
annotate
|
2011-07-05 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2011-07-05 |
Christian Urban |
exported various FCB-lemmas to a separate file
|
file |
diff |
annotate
|
2011-07-05 |
Cezary Kaliszyk |
Express trans_db with Option.map and Option.bind. Possibly mbind is a copy of bind?
|
file |
diff |
annotate
|
2011-07-05 |
Cezary Kaliszyk |
Define a version of aux only for same binders. Completeness is fine.
|
file |
diff |
annotate
|
2011-07-05 |
Cezary Kaliszyk |
Move If / Let with 'True' to the end of Lambda
|
file |
diff |
annotate
|
2011-07-04 |
Christian Urban |
added an example that recurses over two arguments; the interesting proof-obligation is not yet done
|
file |
diff |
annotate
|
2011-06-27 |
Christian Urban |
copied all work to Lambda.thy; had to derive a special version of fcb1 for concrete atom
|
file |
diff |
annotate
|
2011-06-26 |
Christian Urban |
another change to the fcb2; this is needed in order to get all proofs through in Lambda.thy
|
file |
diff |
annotate
|
2011-06-23 |
Christian Urban |
the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
|
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-16 |
Christian Urban |
added a test that every function must be of pt-sort
|
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-15 |
Cezary Kaliszyk |
Some TODOs
|
file |
diff |
annotate
|
2011-06-10 |
Cezary Kaliszyk |
Move working examples before non-working ones
|
file |
diff |
annotate
|
2011-06-10 |
Cezary Kaliszyk |
Optimized proofs and removed some garbage.
|
file |
diff |
annotate
|
2011-06-10 |
Cezary Kaliszyk |
Slightly modify fcb for list1 and put in common place.
|
file |
diff |
annotate
|
2011-06-09 |
Cezary Kaliszyk |
Eval can be defined with additional freshness
|
file |
diff |
annotate
|
2011-06-09 |
Cezary Kaliszyk |
Minor simplification
|
file |
diff |
annotate
|
2011-06-08 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2011-06-08 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2011-06-07 |
Cezary Kaliszyk |
Simplify ln-trans proof
|
file |
diff |
annotate
|
2011-06-07 |
Cezary Kaliszyk |
cbvs can be easily defined without an invariant
|
file |
diff |
annotate
|
2011-06-07 |
Christian Urban |
defined the "count-bound-variables-occurences" function which has an accumulator like trans
|
file |
diff |
annotate
|
2011-06-07 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2011-06-07 |
Cezary Kaliszyk |
remove garbage (proofs that assumes the invariant outside function)
|
file |
diff |
annotate
|
2011-06-07 |
Cezary Kaliszyk |
Proof of trans with invariant
|
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-06-04 |
Cezary Kaliszyk |
Finish and test the locale approach
|
file |
diff |
annotate
|
2011-06-03 |
Christian Urban |
recursion combinator inside a locale
|
file |
diff |
annotate
|
2011-06-02 |
Cezary Kaliszyk |
finished the missing obligations
|
file |
diff |
annotate
|
2011-06-02 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2011-06-02 |
Christian Urban |
a test with a recursion combinator defined on top of nominal_primrec
|
file |
diff |
annotate
|
2011-06-02 |
Cezary Kaliszyk |
Use FCB to simplify proof
|
file |
diff |
annotate
|
2011-06-01 |
Christian Urban |
hopefully final fix for ho-functions
|
file |
diff |
annotate
|
2011-06-01 |
Christian Urban |
first test to fix the problem with free variables
|
file |
diff |
annotate
|
2011-06-01 |
Cezary Kaliszyk |
DB translation using index; easier to reason about.
|
file |
diff |
annotate
|
2011-06-01 |
Cezary Kaliszyk |
Problem: free variables in the goal
|
file |
diff |
annotate
|
2011-06-01 |
Cezary Kaliszyk |
fixed previous commit
|
file |
diff |
annotate
|
2011-06-01 |
Cezary Kaliszyk |
equivariance of db_trans
|
file |
diff |
annotate
|
2011-05-31 |
Christian Urban |
fixed the problem with cps-like functions
|
file |
diff |
annotate
|
2011-05-31 |
Cezary Kaliszyk |
DeBruijn translation in a simplifier friendly way
|
file |
diff |
annotate
|
2011-05-31 |
Cezary Kaliszyk |
map_term can be defined when equivariance is assumed
|
file |
diff |
annotate
|
2011-05-31 |
Cezary Kaliszyk |
map_term is not a function the way it is defined
|
file |
diff |
annotate
|
2011-05-31 |
Cezary Kaliszyk |
Defined translation from nominal to de-Bruijn; with a freshness condition for the lambda case.
|
file |
diff |
annotate
|
2011-05-31 |
Cezary Kaliszyk |
Simple eqvt proofs with perm_simps for clarity
|
file |
diff |
annotate
|
2011-05-30 |
Christian Urban |
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
|
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-14 |
Christian Urban |
added a problem with inductive_cases (reported by Randy)
|
file |
diff |
annotate
|
2011-05-03 |
Christian Urban |
added two mutual recursive inductive definitions
|
file |
diff |
annotate
|
2011-05-03 |
Christian Urban |
proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
|
file |
diff |
annotate
|
2011-04-18 |
Christian Urban |
merged
|
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-04-15 |
Cezary Kaliszyk |
New way of forward elimination of Abs1_eq and simplifications of the function obligation proofs.
|
file |
diff |
annotate
|
2011-04-13 |
Christian Urban |
introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
|
file |
diff |
annotate
|
2011-02-23 |
Cezary Kaliszyk |
Reduce the definition of trans to FCB; test that FCB can be proved with simp rules.
|
file |
diff |
annotate
|
2011-02-01 |
Cezary Kaliszyk |
Only one of the subgoals is needed
|
file |
diff |
annotate
|
2011-01-25 |
Christian Urban |
made eqvt-proof explicit in the function definitions
|
file |
diff |
annotate
|
2011-01-19 |
Christian Urban |
added obtain_fresh lemma; tuned Lambda.thy
|
file |
diff |
annotate
|
2011-01-19 |
Christian Urban |
ported some of the old proofs to serve as testcases
|
file |
diff |
annotate
|
2011-01-19 |
Christian Urban |
defined height as a function that returns an integer
|
file |
diff |
annotate
|
2011-01-18 |
Christian Urban |
defined properly substitution
|
file |
diff |
annotate
|
2011-01-18 |
Christian Urban |
the function translating lambda terms to locally nameless lambda terms; still needs a stronger abs_eq_iff lemma...at the moment only proved for restrictions
|
file |
diff |
annotate
|
2011-01-17 |
Christian Urban |
added a translation function from lambda-terms to deBruijn terms (equivariance fails at the moment)
|
file |
diff |
annotate
|
2011-01-17 |
Christian Urban |
added a few examples of functions to Lambda.thy
|
file |
diff |
annotate
|
2011-01-17 |
Christian Urban |
removed old testing code from Lambda.thy
|
file |
diff |
annotate
|
2011-01-09 |
Christian Urban |
solved subgoals for depth and subst function
|
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 |
tuned
|
file |
diff |
annotate
|
2010-12-31 |
Christian Urban |
changed res keyword to set+ for restrictions; comment by a referee
|
file |
diff |
annotate
|
2010-12-28 |
Christian Urban |
automated all strong induction lemmas
|
file |
diff |
annotate
|
2010-12-22 |
Christian Urban |
properly exported strong exhaust theorem; cleaned up some examples
|
file |
diff |
annotate
|
2010-11-10 |
Christian Urban |
adapted to changes by Florian on the quotient package and removed local fix for function package
|
file |
diff |
annotate
|
2010-09-29 |
Christian Urban |
simplified exhaust proofs
|
file |
diff |
annotate
|
2010-09-29 |
Christian Urban |
test with induct_schema for simpler strong_ind proofs
|
file |
diff |
annotate
|
2010-08-29 |
Christian Urban |
renamed NewParser to Nominal2
|
file |
diff |
annotate
|
2010-08-27 |
Christian Urban |
make copies of the "old" files
|
file |
diff |
annotate
|
2010-08-26 |
Christian Urban |
"isabelle make test" makes all major examples....they work up to supp theorems (excluding)
|
file |
diff |
annotate
|
2010-08-25 |
Christian Urban |
cleaned up (almost completely) the examples
|
file |
diff |
annotate
|
2010-08-25 |
Christian Urban |
automatic lifting
|
file |
diff |
annotate
|
2010-08-25 |
Christian Urban |
now every lemma lifts (even with type variables)
|
file |
diff |
annotate
|
2010-08-25 |
Christian Urban |
can now deal with type variables in nominal datatype definitions
|
file |
diff |
annotate
|
2010-08-21 |
Christian Urban |
nominal_datatypes with type variables do not work
|
file |
diff |
annotate
|
2010-08-21 |
Christian Urban |
changed parser so that the binding mode is indicated as "bind (list)", "bind (set)" or "bind (res)"; if only "bind" is given, then bind (list) is assumed as default
|
file |
diff |
annotate
|
2010-06-07 |
Christian Urban |
work on transitivity proof
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
Match_Lam defined on Quotient Level.
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
More on Function-defined subst.
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
Renamings.
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
merge (non-trival)
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
Previously uncommited direct subst definition changes.
|
file |
diff |
annotate
|
2010-05-21 |
Cezary Kaliszyk |
Function experiments
|
file |
diff |
annotate
|
2010-05-19 |
Cezary Kaliszyk |
more subst experiments
|
file |
diff |
annotate
|
2010-05-19 |
Cezary Kaliszyk |
More subst experminets
|
file |
diff |
annotate
|
2010-05-18 |
Cezary Kaliszyk |
more on subst
|
file |
diff |
annotate
|
2010-05-18 |
Cezary Kaliszyk |
Single variable substitution
|
file |
diff |
annotate
|
2010-05-18 |
Cezary Kaliszyk |
subst fix
|
file |
diff |
annotate
|
2010-05-18 |
Cezary Kaliszyk |
subst experiments
|
file |
diff |
annotate
|
2010-05-12 |
Christian Urban |
fixed the examples for the new eqvt-procedure....temporarily disabled Manual/Term4.thy
|
file |
diff |
annotate
|
2010-05-11 |
Cezary Kaliszyk |
Include raw permutation definitions in eqvt
|
file |
diff |
annotate
|
2010-05-11 |
Cezary Kaliszyk |
Declare alpha_gen_eqvt as eqvt and change the proofs that used 'eqvts[symmetric]'
|
file |
diff |
annotate
|
2010-05-09 |
Christian Urban |
cleaned up a bit the examples; added equivariance to all examples
|
file |
diff |
annotate
|
2010-05-04 |
Cezary Kaliszyk |
Move 2 more to NewParser
|
file |
diff |
annotate
|
2010-04-26 |
Christian Urban |
some changes to the paper
|
file |
diff |
annotate
|
2010-04-26 |
Christian Urban |
eliminated command so that all compiles
|
file |
diff |
annotate
|
2010-04-26 |
Christian Urban |
changed theorem_i to theorem....requires new Isabelle
|
file |
diff |
annotate
|
2010-04-25 |
Christian Urban |
tuned and cleaned
|
file |
diff |
annotate
|
2010-04-16 |
Christian Urban |
automatic proofs for equivariance of alphas
|
file |
diff |
annotate
|
2010-04-16 |
Cezary Kaliszyk |
Finished proof in Lambda.thy
|
file |
diff |
annotate
|
2010-04-16 |
Christian Urban |
attempt to manual prove eqvt for alpha
|
file |
diff |
annotate
|
2010-04-16 |
Christian Urban |
some tuning of eqvt-infrastructure
|
file |
diff |
annotate
|
2010-04-14 |
Christian Urban |
deleted offending [eqvt]-attribute in Abs; Lambda works again, but there is now a problem in CoreHaskell
|
file |
diff |
annotate
|
2010-04-14 |
Christian Urban |
tuned and removed dead code
|
file |
diff |
annotate
|
2010-04-14 |
Christian Urban |
added a library for basic nominal functions; separated nominal_eqvt file
|
file |
diff |
annotate
|
2010-04-14 |
Christian Urban |
first working version of the automatic equivariance procedure
|
file |
diff |
annotate
|
2010-04-14 |
Christian Urban |
preliminary tests
|
file |
diff |
annotate
|
2010-04-13 |
Christian Urban |
made everything to compile
|
file |
diff |
annotate
|
2010-04-12 |
Christian Urban |
some small tunings (incompleted work in Lambda.thy)
|
file |
diff |
annotate
|
2010-04-12 |
Christian Urban |
early ott paper
|
file |
diff |
annotate
|
2010-04-12 |
Christian Urban |
implemented in thmdecls the case where eqvt-lemmas are of the form _ ==> _
|
file |
diff |
annotate
|
2010-04-11 |
Christian Urban |
fixed bug in thmdecls with destructing Trueprop; some initial infrastructure for eqvt-theorems of the form _ ==> _
|
file |
diff |
annotate
|
2010-04-11 |
Christian Urban |
a few tests
|
file |
diff |
annotate
|
2010-04-09 |
Christian Urban |
changed the eqvt-tac to move only outermost permutations inside; added tracing infrastructure for the eqvt-tac
|
file |
diff |
annotate
|
2010-04-09 |
Christian Urban |
renamed ExLam to Lambda and completed the proof of the strong ind principle; tuned paper
|
file |
diff |
annotate
| base
|