2011-07-11 |
Cezary Kaliszyk |
Remove copy of FCB and cleanup
|
changeset |
files
|
2011-07-11 |
Cezary Kaliszyk |
Experiment with permuting eqvt_at
|
changeset |
files
|
2011-07-11 |
Christian Urban |
combinators for local theories and lists
|
changeset |
files
|
2011-07-11 |
Christian Urban |
merged
|
changeset |
files
|
2011-07-11 |
Christian Urban |
some more experiments with let and bns
|
changeset |
files
|
2011-07-08 |
Christian Urban |
some code refactoring
|
changeset |
files
|
2011-07-07 |
Christian Urban |
merged
|
changeset |
files
|
2011-07-07 |
Christian Urban |
code refactoring; introduced a record for raw_dt_info
|
changeset |
files
|
2011-07-06 |
Christian Urban |
more on NBE
|
changeset |
files
|
2011-07-06 |
Christian Urban |
more on the NBE function
|
changeset |
files
|
2011-07-05 |
Christian Urban |
a little further with NBE
|
changeset |
files
|
2011-07-05 |
Cezary Kaliszyk |
Setup eqvt_at for first goal
|
changeset |
files
|
2011-07-05 |
Christian Urban |
attempt for NBE
|
changeset |
files
|
2011-07-05 |
Christian Urban |
added some relatively simple examples from paper by Norrish
|
changeset |
files
|
2011-07-05 |
Christian Urban |
changed bind to binds in specifications; bind will cause trouble with Monad_Syntax
|
changeset |
files
|
2011-07-05 |
Christian Urban |
side commment for future use
|
changeset |
files
|
2011-07-05 |
Christian Urban |
made the tests go through again
|
changeset |
files
|
2011-07-05 |
Christian Urban |
added another example which seems difficult to define
|
changeset |
files
|
2011-07-05 |
Christian Urban |
added a tactic "all_trivials" which simplifies all trivial constructor cases and leaves the others untouched.
|
changeset |
files
|
2011-07-05 |
Christian Urban |
merged
|
changeset |
files
|
2011-07-05 |
Christian Urban |
all FCB lemmas
|
changeset |
files
|
2011-07-05 |
Christian Urban |
exported various FCB-lemmas to a separate file
|
changeset |
files
|
2011-07-05 |
Cezary Kaliszyk |
Express trans_db with Option.map and Option.bind. Possibly mbind is a copy of bind?
|
changeset |
files
|
2011-07-05 |
Cezary Kaliszyk |
Define a version of aux only for same binders. Completeness is fine.
|
changeset |
files
|
2011-07-05 |
Cezary Kaliszyk |
Move If / Let with 'True' to the end of Lambda
|
changeset |
files
|
2011-07-04 |
Christian Urban |
merged
|
changeset |
files
|
2011-07-04 |
Christian Urban |
tuned
|
changeset |
files
|
2011-07-04 |
Christian Urban |
added an example that recurses over two arguments; the interesting proof-obligation is not yet done
|
changeset |
files
|
2011-07-04 |
Cezary Kaliszyk |
Let with a different invariant; not true.
|
changeset |
files
|
2011-07-03 |
Cezary Kaliszyk |
Add non-working Lambda_F_T using FCB2
|
changeset |
files
|
2011-07-03 |
Cezary Kaliszyk |
Added non-working CPS3 using FCB2
|
changeset |
files
|
2011-07-03 |
Cezary Kaliszyk |
Change CPS1 to FCB2
|
changeset |
files
|
2011-07-02 |
Cezary Kaliszyk |
Did the proofs of height and subst for Let with list-like binders. Having apply_assns allows proving things by alpha_bn
|
changeset |
files
|
2011-07-01 |
Christian Urban |
side-by-side tests of lets with single assignment; deep-binder case works if the recursion is avoided using an auxiliary function
|
changeset |
files
|
2011-07-01 |
Cezary Kaliszyk |
Exhaust Issue
|
changeset |
files
|
2011-06-30 |
Christian Urban |
clarified a sentence
|
changeset |
files
|
2011-06-30 |
Christian Urban |
more code refactoring
|
changeset |
files
|
2011-06-29 |
Christian Urban |
combined distributed data for alpha in alpha_result (partially done)
|
changeset |
files
|
2011-06-29 |
Christian Urban |
moved Classical and Let temporarily into a section where "sorry" is allowed; this makes all test go through
|
changeset |
files
|
2011-06-29 |
Christian Urban |
added a warning if a theorem is already declared as equivariant
|
changeset |
files
|
2011-06-29 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-29 |
Cezary Kaliszyk |
Prove bn injectivity and experiment more with Let
|
changeset |
files
|
2011-06-28 |
Christian Urban |
some experiments
|
changeset |
files
|
2011-06-28 |
Cezary Kaliszyk |
trying new fcb in let/subst
|
changeset |
files
|
2011-06-28 |
Cezary Kaliszyk |
Leftover only inj and eqvt
|
changeset |
files
|
2011-06-28 |
Cezary Kaliszyk |
eapply fcb ok
|
changeset |
files
|
2011-06-28 |
Cezary Kaliszyk |
Removed Inl and Inr
|
changeset |
files
|
2011-06-28 |
Christian Urban |
relaxed type in fcb
|
changeset |
files
|
2011-06-28 |
Christian Urban |
fcb with explicit bn function
|
changeset |
files
|
2011-06-28 |
Christian Urban |
added let-rec example
|
changeset |
files
|
2011-06-28 |
Cezary Kaliszyk |
Experiments with res
|
changeset |
files
|
2011-06-27 |
Christian Urban |
proved the fcb also for sets (no restriction yet)
|
changeset |
files
|
2011-06-27 |
Christian Urban |
copied all work to Lambda.thy; had to derive a special version of fcb1 for concrete atom
|
changeset |
files
|
2011-06-27 |
Christian Urban |
streamlined the fcb-proof and made fcb1 a special case of fcb
|
changeset |
files
|
2011-06-27 |
Christian Urban |
completed proof in Classical; the fcb lemma works for any list of atoms (despite what was written earlier)
|
changeset |
files
|
2011-06-27 |
Christian Urban |
fcb for multible (list) binders; at the moment all of them have to have the same sort (at-class); this should also work for set binders, but not yet for restriction.
|
changeset |
files
|
2011-06-27 |
Christian Urban |
renamed ds to dset (disagreement set)
|
changeset |
files
|
2011-06-27 |
Christian Urban |
added small lemma about disagreement set
|
changeset |
files
|
2011-06-26 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-26 |
Cezary Kaliszyk |
New-style fcb for multiple binders.
|
changeset |
files
|
2011-06-26 |
Cezary Kaliszyk |
equality of lst_binder and a few helper lemmas
|
changeset |
files
|
2011-06-26 |
Christian Urban |
only one of the fcb precondistions are needed (probably the same with the perm-conditions)
|
changeset |
files
|
2011-06-26 |
Christian Urban |
another change to the fcb2; this is needed in order to get all proofs through in Lambda.thy
|
changeset |
files
|
2011-06-25 |
Christian Urban |
did all cases, except the multiple binder case
|
changeset |
files
|
2011-06-25 |
Christian Urban |
an alternative FCB for Abs_lst1; seems simpler but not as simple as I thought; not sure whether it generalises to multiple binders.
|
changeset |
files
|
2011-06-24 |
Christian Urban |
except for the interated binder case, finished definition in Calssical.thy
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
Make examples work with non-precompiled image
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
Remove Lambda_add.thy
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
The examples in Lambda_add can be defined by nominal_function directly
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
Theory name changes for JEdit
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
More usual names for substitution properties
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
Second Fixed Point Theorem
|
changeset |
files
|
2011-06-24 |
Cezary Kaliszyk |
Speed-up the completeness proof.
|
changeset |
files
|
2011-06-23 |
Christian Urban |
the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
|
changeset |
files
|
2011-06-23 |
Christian Urban |
added file
|
changeset |
files
|
2011-06-23 |
Christian Urban |
expanded the example
|
changeset |
files
|
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
|
changeset |
files
|
2011-06-22 |
Christian Urban |
tuned
|
changeset |
files
|
2011-06-22 |
Christian Urban |
deleted some dead code
|
changeset |
files
|
2011-06-22 |
Christian Urban |
some rudimentary infrastructure for storing data about nominal datatypes
|
changeset |
files
|
2011-06-22 |
Cezary Kaliszyk |
constants with the same names
|
changeset |
files
|
2011-06-21 |
Cezary Kaliszyk |
Quotients/TODO addtion
|
changeset |
files
|
2011-06-21 |
Cezary Kaliszyk |
Minor
|
changeset |
files
|
2011-06-21 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-21 |
Cezary Kaliszyk |
spelling
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
Abs_set_fcb
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
function for let-rec
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
TODO/minor
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
Move lst_fcb to Nominal2_Abs
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
More minor TODOs
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
Update TODO
|
changeset |
files
|
2011-06-20 |
Cezary Kaliszyk |
Let/minor
|
changeset |
files
|
2011-06-19 |
Cezary Kaliszyk |
Update Quotient/TODO and remove some attic code
|
changeset |
files
|
2011-06-19 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-19 |
Cezary Kaliszyk |
little on cps2
|
changeset |
files
|
2011-06-16 |
Christian Urban |
got rid of the boolean flag in the raw_equivariance function
|
changeset |
files
|
2011-06-16 |
Cezary Kaliszyk |
Fix
|
changeset |
files
|
2011-06-16 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-16 |
Cezary Kaliszyk |
CPS3 can be defined with eqvt_rhs.
|
changeset |
files
|
2011-06-16 |
Christian Urban |
moved for the moment CPS translations into the example directory
|
changeset |
files
|
2011-06-16 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-16 |
Christian Urban |
added eqvt_at and invariant for boths sides of the equations
|
changeset |
files
|
2011-06-16 |
Cezary Kaliszyk |
Added the CPS translation experiments. CPS1 comes with all the proofs, CPS2,3 just have the function and need eqvt_rhs to finish the obligations.
|
changeset |
files
|
2011-06-16 |
Christian Urban |
added a test that every function must be of pt-sort
|
changeset |
files
|
2011-06-16 |
Christian Urban |
all tests work again
|
changeset |
files
|
2011-06-15 |
Christian Urban |
added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method
|
changeset |
files
|
2011-06-15 |
Christian Urban |
added an abstract
|
changeset |
files
|
2011-06-15 |
Christian Urban |
added a stub for function paper; "isabelle make fnpaper"
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
one TODO and one Problem?
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
Some TODOs
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-15 |
Cezary Kaliszyk |
TypeSchemes work with 'default'.
|
changeset |
files
|
2011-06-14 |
Christian Urban |
tuned some proofs
|
changeset |
files
|
2011-06-14 |
Christian Urban |
fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough
|
changeset |
files
|
2011-06-14 |
Christian Urban |
tuned
|
changeset |
files
|
2011-06-10 |
Cezary Kaliszyk |
Move working examples before non-working ones
|
changeset |
files
|
2011-06-10 |
Cezary Kaliszyk |
Optimized proofs and removed some garbage.
|
changeset |
files
|
2011-06-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-10 |
Cezary Kaliszyk |
Slightly modify fcb for list1 and put in common place.
|
changeset |
files
|
2011-06-10 |
Cezary Kaliszyk |
Experiments with Let
|
changeset |
files
|
2011-06-09 |
Cezary Kaliszyk |
Eval can be defined with additional freshness
|
changeset |
files
|
2011-06-09 |
Cezary Kaliszyk |
Minor simplification
|
changeset |
files
|
2011-06-09 |
Cezary Kaliszyk |
abs_res_fcb will be enough to finish the multiple-recursive proof, if we have a working 'default'.
|
changeset |
files
|
2011-06-09 |
Cezary Kaliszyk |
More experiments with 'default'
|
changeset |
files
|
2011-06-08 |
Cezary Kaliszyk |
Finished the proof with the invariant
|
changeset |
files
|
2011-06-08 |
Cezary Kaliszyk |
Issue with 'default'
|
changeset |
files
|
2011-06-08 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-08 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-08 |
Christian Urban |
using the option "default" the function package allows one to give an explicit default value
|
changeset |
files
|
2011-06-08 |
Cezary Kaliszyk |
Simpler proof of TypeSchemes/substs
|
changeset |
files
|
2011-06-08 |
Cezary Kaliszyk |
Simplify fcb_res
|
changeset |
files
|
2011-06-08 |
Cezary Kaliszyk |
FCB for res binding and simplified proof of subst for type schemes
|
changeset |
files
|
2011-06-07 |
Cezary Kaliszyk |
Simplify ln-trans proof
|
changeset |
files
|
2011-06-07 |
Cezary Kaliszyk |
cbvs can be easily defined without an invariant
|
changeset |
files
|
2011-06-07 |
Christian Urban |
defined the "count-bound-variables-occurences" function which has an accumulator like trans
|
changeset |
files
|
2011-06-07 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-07 |
Cezary Kaliszyk |
remove garbage (proofs that assumes the invariant outside function)
|
changeset |
files
|
2011-06-07 |
Cezary Kaliszyk |
Proof of trans with invariant
|
changeset |
files
|
2011-06-07 |
Cezary Kaliszyk |
Testing invariant in Lambda_F_T
|
changeset |
files
|
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
|
changeset |
files
|
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
|
changeset |
files
|
2011-06-06 |
Christian Urban |
slightly stronger property in fundef_ex_prop
|
changeset |
files
|
2011-06-05 |
Christian Urban |
added an option for an invariant (at the moment only a stub)
|
changeset |
files
|
2011-06-05 |
Christian Urban |
added a more general lemma fro fundef_ex1
|
changeset |
files
|
2011-06-04 |
Cezary Kaliszyk |
Trying the induction on the graph
|
changeset |
files
|
2011-06-04 |
Cezary Kaliszyk |
Finish and test the locale approach
|
changeset |
files
|
2011-06-03 |
Cezary Kaliszyk |
FiniteSupp precondition in the function is enough to get rid of completeness obligationss
|
changeset |
files
|
2011-06-03 |
Christian Urban |
recursion combinator inside a locale
|
changeset |
files
|
2011-06-03 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-03 |
Cezary Kaliszyk |
F for lambda used to define translation to locally nameless
|
changeset |
files
|
2011-06-02 |
Christian Urban |
typo
|
changeset |
files
|
2011-06-02 |
Christian Urban |
removed dead code
|
changeset |
files
|
2011-06-02 |
Cezary Kaliszyk |
finished the missing obligations
|
changeset |
files
|
2011-06-02 |
Christian Urban |
merged
|
changeset |
files
|
2011-06-02 |
Christian Urban |
a test with a recursion combinator defined on top of nominal_primrec
|
changeset |
files
|
2011-06-02 |
Cezary Kaliszyk |
Use FCB to simplify proof
|
changeset |
files
|
2011-06-02 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-06-02 |
Cezary Kaliszyk |
Remove SMT
|
changeset |
files
|
2011-06-01 |
Christian Urban |
hopefully final fix for ho-functions
|
changeset |
files
|
2011-06-01 |
Christian Urban |
first test to fix the problem with free variables
|
changeset |
files
|
2011-06-01 |
Cezary Kaliszyk |
proved subst for All constructor in type schemes.
|
changeset |
files
|
2011-06-01 |
Cezary Kaliszyk |
DB translation using index; easier to reason about.
|
changeset |
files
|
2011-06-01 |
Cezary Kaliszyk |
Problem: free variables in the goal
|
changeset |
files
|
2011-06-01 |
Cezary Kaliszyk |
fixed previous commit
|
changeset |
files
|
2011-06-01 |
Cezary Kaliszyk |
equivariance of db_trans
|
changeset |
files
|
2011-05-31 |
Christian Urban |
fixed the problem with cps-like functions
|
changeset |
files
|
2011-05-31 |
Cezary Kaliszyk |
DeBruijn translation in a simplifier friendly way
|
changeset |
files
|
2011-05-31 |
Cezary Kaliszyk |
map_term can be defined when equivariance is assumed
|
changeset |
files
|
2011-05-31 |
Cezary Kaliszyk |
map_term is not a function the way it is defined
|
changeset |
files
|
2011-05-31 |
Cezary Kaliszyk |
Defined translation from nominal to de-Bruijn; with a freshness condition for the lambda case.
|
changeset |
files
|
2011-05-31 |
Cezary Kaliszyk |
Simple eqvt proofs with perm_simps for clarity
|
changeset |
files
|
2011-05-30 |
Christian Urban |
tuned last commit
|
changeset |
files
|
2011-05-30 |
Christian Urban |
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
|
changeset |
files
|
2011-05-26 |
Christian Urban |
updated to new Isabelle
|
changeset |
files
|
2011-05-25 |
Christian Urban |
added eq_iff and distinct lemmas of nominal datatypes to the simplifier
|
changeset |
files
|
2011-05-24 |
Christian Urban |
more on slides
|
changeset |
files
|
2011-05-22 |
Christian Urban |
added slides for copenhagen
|
changeset |
files
|
2011-05-14 |
Christian Urban |
added a problem with inductive_cases (reported by Randy)
|
changeset |
files
|
2011-05-13 |
Christian Urban |
misc
|
changeset |
files
|
2011-05-10 |
Christian Urban |
made the subtyping work again
|
changeset |
files
|
2011-05-10 |
Christian Urban |
updated to new Isabelle (> 9 May)
|
changeset |
files
|
2011-05-09 |
Christian Urban |
merged
|
changeset |
files
|
2011-05-03 |
Christian Urban |
added two mutual recursive inductive definitions
|
changeset |
files
|
2011-05-03 |
Christian Urban |
deleted two functions from the API
|
changeset |
files
|
2011-05-03 |
Christian Urban |
proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
|
changeset |
files
|
2011-05-09 |
Christian Urban |
more on pearl-paper
|
changeset |
files
|
2011-05-04 |
Christian Urban |
more on pearl-paper
|
changeset |
files
|
2011-05-02 |
Christian Urban |
updated Quotient paper so that it compiles again
|
changeset |
files
|
2011-04-28 |
Christian Urban |
merged
|
changeset |
files
|
2011-04-28 |
Christian Urban |
added slides for beijing
|
changeset |
files
|
2011-04-21 |
Christian Urban |
more to the pearl paper
|
changeset |
files
|
2011-04-19 |
Christian Urban |
updated to snapshot Isabelle 19 April
|
changeset |
files
|
2011-04-18 |
Christian Urban |
merged
|
changeset |
files
|
2011-04-18 |
Christian Urban |
added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
|
changeset |
files
|
2011-04-15 |
Cezary Kaliszyk |
New way of forward elimination of Abs1_eq and simplifications of the function obligation proofs.
|
changeset |
files
|
2011-04-13 |
Christian Urban |
merged
|
changeset |
files
|
2011-04-13 |
Christian Urban |
introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
|
changeset |
files
|
2011-04-12 |
Christian Urban |
shanghai slides
|
changeset |
files
|
2011-04-11 |
Christian Urban |
pictures for slides
|
changeset |
files
|
2011-04-11 |
Christian Urban |
Shanghai slides
|
changeset |
files
|
2011-04-10 |
Christian Urban |
more paper
|
changeset |
files
|
2011-04-09 |
Christian Urban |
eqvt of supp and fresh is proved using equivariance infrastructure
|
changeset |
files
|
2011-04-09 |
Christian Urban |
more paper
|
changeset |
files
|
2011-04-09 |
Christian Urban |
more on the paper
|
changeset |
files
|
2011-04-08 |
Christian Urban |
tuned paper
|
changeset |
files
|
2011-04-08 |
Christian Urban |
tuned paper
|
changeset |
files
|
2011-04-08 |
Christian Urban |
typo
|
changeset |
files
|
2011-04-08 |
Christian Urban |
more on paper
|
changeset |
files
|
2011-04-07 |
Christian Urban |
eqvt_lambda without eta-expansion
|
changeset |
files
|
2011-04-06 |
Christian Urban |
changed default preprocessor that does not catch variables only occuring on the right
|
changeset |
files
|
2011-03-31 |
Christian Urban |
final version of slides
|
changeset |
files
|
2011-03-30 |
Christian Urban |
more on the slides
|
changeset |
files
|
2011-03-30 |
Christian Urban |
tuned IsaMakefile
|
changeset |
files
|
2011-03-29 |
Christian Urban |
rearranged directories and updated to new Isabelle
|
changeset |
files
|
2011-03-16 |
Christian Urban |
precise path to LaTeXsugar
|
changeset |
files
|
2011-03-16 |
Christian Urban |
a lit bit more on the pearl-jv paper
|
changeset |
files
|
2011-03-16 |
Christian Urban |
ported changes from function package....needs Isabelle 16 March or above
|
changeset |
files
|
2011-03-14 |
Christian Urban |
more on the pearl paper
|
changeset |
files
|
2011-03-14 |
Christian Urban |
equivariance for All and Ex can be proved in terms of their definition
|
changeset |
files
|
2011-03-11 |
Christian Urban |
more on the paper
|
changeset |
files
|
2011-03-08 |
Christian Urban |
merged
|
changeset |
files
|
2011-03-08 |
Christian Urban |
more on the pearl paper
|
changeset |
files
|
2011-03-02 |
Cezary Kaliszyk |
distinct names at toplevel
|
changeset |
files
|
2011-03-02 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-03-02 |
Cezary Kaliszyk |
Pairing function
|
changeset |
files
|
2011-03-02 |
Christian Urban |
updated pearl papers
|
changeset |
files
|
2011-03-01 |
Christian Urban |
a bit more tuning
|
changeset |
files
|
2011-02-28 |
Christian Urban |
included old test cases for perm_simp into ROOT.ML file
|
changeset |
files
|
2011-02-28 |
Christian Urban |
split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
|
changeset |
files
|
2011-02-25 |
Christian Urban |
some slight polishing
|
changeset |
files
|
2011-02-24 |
Christian Urban |
merged
|
changeset |
files
|
2011-02-24 |
Christian Urban |
added a lemma about fresh_star and Abs
|
changeset |
files
|
2011-02-23 |
Cezary Kaliszyk |
Reduce the definition of trans to FCB; test that FCB can be proved with simp rules.
|
changeset |
files
|
2011-02-19 |
Cezary Kaliszyk |
typeschemes/subst
|
changeset |
files
|
2011-02-17 |
Cezary Kaliszyk |
further experiments with typeschemes subst
|
changeset |
files
|
2011-02-17 |
Cezary Kaliszyk |
Finished the proof of a function that invents fresh variable names.
|
changeset |
files
|
2011-02-16 |
Christian Urban |
added eqvt for length
|
changeset |
files
|
2011-02-16 |
Christian Urban |
added eqvt lemmas for filter and distinct
|
changeset |
files
|
2011-02-07 |
Christian Urban |
added eqvt for cartesian products
|
changeset |
files
|
2011-02-07 |
Christian Urban |
cleaned up the experiments so that the tests go through
|
changeset |
files
|
2011-02-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-02-04 |
Cezary Kaliszyk |
Experiments defining a function on Let
|
changeset |
files
|
2011-02-04 |
Christian Urban |
updated TODO
|
changeset |
files
|
2011-02-04 |
Christian Urban |
Lambda.thy which works with Nominal_Isabelle2011
|
changeset |
files
|
2011-02-03 |
Christian Urban |
merged
|
changeset |
files
|
2011-02-03 |
Christian Urban |
removed diagnostic code
|
changeset |
files
|
2011-02-01 |
Cezary Kaliszyk |
Only one of the subgoals is needed
|
changeset |
files
|
2011-01-31 |
Cezary Kaliszyk |
Experiments with substitution on set+
|
changeset |
files
|
2011-01-31 |
Cezary Kaliszyk |
More properties that relate abs_res and abs_set. Also abs_res with less binders.
|
changeset |
files
|
2011-01-30 |
Cezary Kaliszyk |
alpha_res implies alpha_set :)
|
changeset |
files
|
2011-01-30 |
Cezary Kaliszyk |
Showing that the binders difference is fresh for the left side solves the goal for 'set'.
|
changeset |
files
|
2011-01-29 |
Cezary Kaliszyk |
Experiments with functions
|
changeset |
files
|
2011-01-27 |
Christian Urban |
some experiments
|
changeset |
files
|
2011-01-27 |
Christian Urban |
the proofs with eqvt_at
|
changeset |
files
|
2011-01-25 |
Christian Urban |
made eqvt-proof explicit in the function definitions
|
changeset |
files
|
2011-01-24 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-01-24 |
Cezary Kaliszyk |
minor
|
changeset |
files
|
2011-01-24 |
Cezary Kaliszyk |
Down as infixr
|
changeset |
files
|
2011-01-23 |
Christian Urban |
added some slides
|
changeset |
files
|
2011-01-23 |
Christian Urban |
added Tutorial6
|
changeset |
files
|
2011-01-23 |
Christian Urban |
cleaning up
|
changeset |
files
|
2011-01-22 |
Christian Urban |
merged
|
changeset |
files
|
2011-01-22 |
Christian Urban |
cleaned up Tutorial 3 with solutions
|
changeset |
files
|
2011-01-22 |
Cezary Kaliszyk |
Missing val.simps
|
changeset |
files
|
2011-01-22 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2011-01-22 |
Cezary Kaliszyk |
Tutorial 4s
|
changeset |
files
|
2011-01-22 |
Christian Urban |
cleaned up and solution section
|
changeset |
files
|
2011-01-22 |
Christian Urban |
cleaned up tutorial1...added solution file
|
changeset |
files
|
2011-01-22 |
Christian Urban |
better version of Tutorial 1
|
changeset |
files
|
2011-01-21 |
Christian Urban |
better flow of proofs and definitions and proof
|
changeset |
files
|
2011-01-21 |
Christian Urban |
separated type preservation and progress into a separate file
|
changeset |
files
|
2011-01-21 |
Christian Urban |
substitution lemma in separate file
|
changeset |
files
|
2011-01-21 |
Christian Urban |
added unbind example
|
changeset |
files
|
2011-01-20 |
Christian Urban |
a bit tuning
|
changeset |
files
|
2011-01-20 |
Christian Urban |
first split of tutorrial theory
|
changeset |
files
|
2011-01-19 |
Christian Urban |
added a very rough version of the tutorial; all seems to work
|
changeset |
files
|
2011-01-19 |
Christian Urban |
added obtain_fresh lemma; tuned Lambda.thy
|
changeset |
files
|
2011-01-19 |
Christian Urban |
base file for the tutorial (contains definitions for heigt, subst and beta-reduction)
|
changeset |
files
|
2011-01-19 |
Christian Urban |
ported some of the old proofs to serve as testcases
|
changeset |
files
|
2011-01-19 |
Christian Urban |
added eqvt and supp lemma for removeAll (function from List.thy)
|
changeset |
files
|
2011-01-19 |
Christian Urban |
theory name as it should be
|
changeset |
files
|
2011-01-19 |
Christian Urban |
removed diagnostic code
|
changeset |
files
|
2011-01-19 |
Christian Urban |
added Minimal file to test things
|
changeset |
files
|
2011-01-19 |
Christian Urban |
defined height as a function that returns an integer
|
changeset |
files
|
2011-01-18 |
Christian Urban |
deleted diagnostic code
|
changeset |
files
|
2011-01-18 |
Christian Urban |
some tryes about substitution over type-schemes
|
changeset |
files
|
2011-01-18 |
Christian Urban |
defined properly substitution
|
changeset |
files
|
2011-01-18 |
Christian Urban |
derived stronger Abs_eq_iff2 theorems
|
changeset |
files
|
2011-01-18 |
Christian Urban |
made alpha_abs_set_stronger1 stronger
|
changeset |
files
|
2011-01-18 |
Christian Urban |
removed finiteness assumption from set_rename_perm
|
changeset |
files
|
2011-01-18 |
Cezary Kaliszyk |
alpha_abs_set_stronger1
|
changeset |
files
|
2011-01-18 |
Cezary Kaliszyk |
alpha_abs_let_stronger is not true in the same form
|
changeset |
files
|
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
|
changeset |
files
|
2011-01-18 |
Christian Urban |
modified the renaming_perm lemmas
|
changeset |
files
|
2011-01-17 |
Christian Urban |
added a translation function from lambda-terms to deBruijn terms (equivariance fails at the moment)
|
changeset |
files
|
2011-01-17 |
Christian Urban |
added a few examples of functions to Lambda.thy
|
changeset |
files
|
2011-01-17 |
Christian Urban |
exported nominal function code to external file
|
changeset |
files
|
2011-01-17 |
Christian Urban |
removed old testing code from Lambda.thy
|
changeset |
files
|
2011-01-17 |
Christian Urban |
moved high level code from LamTest into the main libraries.
|
changeset |
files
|
2011-01-17 |
Christian Urban |
eliminated tracing code; added flag so that equivariance is only proved for the function graph, not the relation
|
changeset |
files
|
2011-01-15 |
Christian Urban |
subst also works now
|
changeset |
files
|
2011-01-15 |
Christian Urban |
nominal_function works now completely for frees and depth; still a propbelm with subst; no unproved assumptions
|
changeset |
files
|
2011-01-14 |
Christian Urban |
strengthened renaming lemmas
|
changeset |
files
|
2011-01-13 |
Christian Urban |
added eqvt_lemmas for subset and psubset
|
changeset |
files
|
2011-01-10 |
Christian Urban |
a few lemmas about freshness for at and at_base
|
changeset |
files
|
2011-01-10 |
Christian Urban |
added a property about finite support in the presense of eqvt_at
|
changeset |
files
|
2011-01-09 |
Christian Urban |
instantiated fundef_ex1_eqvt_at theorem with the indction hypothesis
|
changeset |
files
|
2011-01-09 |
Christian Urban |
solved subgoals for depth and subst function
|
changeset |
files
|
2011-01-09 |
Christian Urban |
added eqvt_at premises in function definition - however not proved at the moment
|
changeset |
files
|
2011-01-07 |
Christian Urban |
added one further lemma about equivariance of THE_default
|
changeset |
files
|
2011-01-07 |
Christian Urban |
equivariance of THE_default under the uniqueness assumption
|
changeset |
files
|
2011-01-07 |
Christian Urban |
derived equivariance for the function graph and function relation
|
changeset |
files
|
2011-01-06 |
Christian Urban |
a modified function package where, as a test, True has been injected into the compatibility condictions
|
changeset |
files
|
2011-01-06 |
Christian Urban |
removed last traces of debugging code
|
changeset |
files
|
2011-01-06 |
Christian Urban |
removed debugging code abd introduced a guarded tracing function
|
changeset |
files
|
2011-01-06 |
Christian Urban |
moved Weakening up....it does not compile when put at the last position
|
changeset |
files
|
2011-01-06 |
Christian Urban |
tuned
|
changeset |
files
|
2011-01-06 |
Christian Urban |
added weakening to the test cases
|
changeset |
files
|
2011-01-06 |
Christian Urban |
cleaned up weakening proof and added a version with finit sets
|
changeset |
files
|
2011-01-06 |
Christian Urban |
same
|
changeset |
files
|
2011-01-06 |
Christian Urban |
some further lemmas for fsets
|
changeset |
files
|
2011-01-06 |
Christian Urban |
made sure the raw datatypes and raw functions do not get any mixfix syntax
|
changeset |
files
|
2011-01-05 |
Christian Urban |
exported the code into a separate file
|
changeset |
files
|
2011-01-05 |
Christian Urban |
strong rule inductions; as an example the weakening lemma works
|
changeset |
files
|
2011-01-04 |
Christian Urban |
final version of the ESOP paper; used set+ instead of res as requested by one reviewer
|
changeset |
files
|
2011-01-03 |
Christian Urban |
file with most of the strong rule induction development
|
changeset |
files
|
2011-01-03 |
Christian Urban |
simple cases for string rule inductions
|
changeset |
files
|
2010-12-31 |
Christian Urban |
changed res keyword to set+ for restrictions; comment by a referee
|
changeset |
files
|
2010-12-31 |
Christian Urban |
added proper case names for all induct and exhaust theorems
|
changeset |
files
|
2010-12-31 |
Christian Urban |
added small example for strong inductions; functions still need a sorry
|
changeset |
files
|
2010-12-30 |
Christian Urban |
removed local fix for bug in induction_schema; added setup method for strong inductions
|
changeset |
files
|
2010-12-28 |
Christian Urban |
automated all strong induction lemmas
|
changeset |
files
|
2010-12-28 |
Christian Urban |
proper application of induction_schema and strong_exhaust rules; needs local fix in induction_schema.ML
|
changeset |
files
|
2010-12-26 |
Christian Urban |
generated goals for strong induction theorems.
|
changeset |
files
|
2010-12-23 |
Christian Urban |
test with strong inductions
|
changeset |
files
|
2010-12-23 |
Christian Urban |
moved all strong_exhaust code to nominal_dt_quot; tuned examples
|
changeset |
files
|
2010-12-23 |
Christian Urban |
moved generic functions into nominal_library
|
changeset |
files
|
2010-12-22 |
Christian Urban |
slight tuning
|
changeset |
files
|
2010-12-22 |
Christian Urban |
slight tuning
|
changeset |
files
|
2010-12-22 |
Christian Urban |
tuned examples
|
changeset |
files
|
2010-12-22 |
Christian Urban |
added fold_right which produces the correct term for left-infix operators
|
changeset |
files
|
2010-12-22 |
Christian Urban |
updated to Isabelle 22 December
|
changeset |
files
|
2010-12-22 |
Christian Urban |
a bit tuning
|
changeset |
files
|
2010-12-22 |
Christian Urban |
corrected premises of strong exhausts theorems
|
changeset |
files
|
2010-12-22 |
Christian Urban |
properly exported strong exhaust theorem; cleaned up some examples
|
changeset |
files
|
2010-12-21 |
Christian Urban |
all examples for strong exhausts work; recursive binders need to be treated differently; still unclean version with lots of diagnostic code
|
changeset |
files
|
2010-12-19 |
Christian Urban |
one interesting case done
|
changeset |
files
|
2010-12-19 |
Christian Urban |
a stronger statement for at_set_avoiding
|
changeset |
files
|
2010-12-17 |
Christian Urban |
tuned
|
changeset |
files
|
2010-12-17 |
Christian Urban |
tuned
|
changeset |
files
|
2010-12-16 |
Christian Urban |
simple cases for strong inducts done; infrastructure for the difficult ones is there
|
changeset |
files
|
2010-12-16 |
Christian Urban |
added theorem-rewriter conversion
|
changeset |
files
|
2010-12-14 |
Christian Urban |
freshness theorem in strong exhausts; (temporarily includes a cheat_tac to make all tests go through)
|
changeset |
files
|
2010-12-12 |
Christian Urban |
created strong_exhausts terms
|
changeset |
files
|
2010-12-12 |
Christian Urban |
moved setify and listify functions into the library; introduced versions that have a type argument
|
changeset |
files
|
2010-12-10 |
Christian Urban |
updated
|
changeset |
files
|
2010-12-09 |
Christian Urban |
a bit more tuning of the paper
|
changeset |
files
|
2010-12-09 |
Christian Urban |
brought the paper to 20 pages plus one page appendix
|
changeset |
files
|
2010-12-08 |
Christian Urban |
first tests about exhaust
|
changeset |
files
|
2010-12-08 |
Christian Urban |
moved some code into the nominal_library
|
changeset |
files
|
2010-12-08 |
Christian Urban |
moved definition of raw bn-functions into nominal_dt_rawfuns
|
changeset |
files
|
2010-12-08 |
Christian Urban |
kept the nested structure of constructors (belonging to one datatype)
|
changeset |
files
|
2010-12-07 |
Christian Urban |
moved general theorems into the libraries
|
changeset |
files
|
2010-12-07 |
Christian Urban |
automated permute_bn theorems
|
changeset |
files
|
2010-12-07 |
Christian Urban |
updated to changes in Isabelle
|
changeset |
files
|
2010-12-06 |
Christian Urban |
deleted nominal_dt_supp.ML
|
changeset |
files
|
2010-12-06 |
Christian Urban |
moved code from nominal_dt_supp to nominal_dt_quot
|
changeset |
files
|
2010-12-06 |
Christian Urban |
automated alpha_perm_bn theorems
|
changeset |
files
|
2010-12-06 |
Christian Urban |
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
|
changeset |
files
|
2010-12-03 |
Christian Urban |
updated to Isabelle 2nd December
|
changeset |
files
|
2010-11-29 |
Christian Urban |
isarfied some of the high-level proofs
|
changeset |
files
|
2010-11-29 |
Christian Urban |
added abs_rename_res lemma
|
changeset |
files
|
2010-11-29 |
Christian Urban |
completed proofs in Foo2
|
changeset |
files
|
2010-11-28 |
Christian Urban |
completed the strong exhausts rules for Foo2 using general lemmas
|
changeset |
files
|
2010-11-27 |
Christian Urban |
tuned proof to reduce number of warnings
|
changeset |
files
|
2010-11-27 |
Christian Urban |
disabled the Foo examples, because of heavy work
|
changeset |
files
|
2010-11-26 |
Christian Urban |
slightly simplified the Foo2 tests and hint at a general lemma
|
changeset |
files
|
2010-11-26 |
Christian Urban |
completely different method fro deriving the exhaust lemma
|
changeset |
files
|
2010-11-26 |
Christian Urban |
merged
|
changeset |
files
|
2010-11-25 |
Christian Urban |
merged
|
changeset |
files
|
2010-11-24 |
Christian Urban |
added example from the F-ing paper by Rossberg, Russo and Dreyer
|
changeset |
files
|
2010-11-24 |
Christian Urban |
implemented concrete suggestion of 3rd reviewer
|
changeset |
files
|
2010-11-26 |
Cezary Kaliszyk |
missing freshness assumptions
|
changeset |
files
|
2010-11-25 |
Cezary Kaliszyk |
foo2 strong induction
|
changeset |
files
|
2010-11-24 |
Cezary Kaliszyk |
foo2 full exhausts
|
changeset |
files
|
2010-11-24 |
Cezary Kaliszyk |
Foo2 strong_exhaust for first variable.
|
changeset |
files
|
2010-11-22 |
Cezary Kaliszyk |
single rename in let2
|
changeset |
files
|
2010-11-22 |
Cezary Kaliszyk |
current isabelle
|
changeset |
files
|
2010-11-21 |
Christian Urban |
added example Foo2.thy
|
changeset |
files
|
2010-11-15 |
Christian Urban |
tuned example
|
changeset |
files
|
2010-11-15 |
Christian Urban |
proved that bn functions return a finite set
|
changeset |
files
|
2010-11-15 |
Christian Urban |
added a test for the various shallow binders
|
changeset |
files
|
2010-11-15 |
Christian Urban |
fixed bug in fv function where a shallow binder binds lists of names
|
changeset |
files
|
2010-11-14 |
Christian Urban |
merged Nominal-General directory into Nominal; renamed Abs.thy to Nominal2_Abs.thy
|
changeset |
files
|
2010-11-14 |
Christian Urban |
deleted special Nominal2_FSet theory
|
changeset |
files
|
2010-11-14 |
Christian Urban |
moved rest of the lemmas from Nominal2_FSet to the TypeScheme example
|
changeset |
files
|
2010-11-14 |
Christian Urban |
moved most material fron Nominal2_FSet into the Nominal_Base theory
|
changeset |
files
|
2010-11-14 |
Christian Urban |
tuned example
|
changeset |
files
|
2010-11-14 |
Christian Urban |
lifted permute_bn simp rules
|
changeset |
files
|
2010-11-13 |
Christian Urban |
lifted permute_bn constants
|
changeset |
files
|
2010-11-13 |
Christian Urban |
respectfulness for permute_bn functions
|
changeset |
files
|
2010-11-12 |
Christian Urban |
automated permute_bn functions (raw ones first)
|
changeset |
files
|
2010-11-10 |
Christian Urban |
adapted to changes by Florian on the quotient package and removed local fix for function package
|
changeset |
files
|
2010-11-10 |
Christian Urban |
expanded the paper by uncommenting the comments and adding the appendix
|
changeset |
files
|
2010-11-07 |
Christian Urban |
fixed locally the problem with the function package; all tests work again
|
changeset |
files
|
2010-11-06 |
Christian Urban |
added a test about subtyping; disabled two tests, because of problem with function package
|
changeset |
files
|
2010-11-05 |
Christian Urban |
small typo
|
changeset |
files
|
2010-10-29 |
Christian Urban |
squeezed qpaper to 6 pages
|
changeset |
files
|
2010-10-29 |
Cezary Kaliszyk |
Qpaper / Move examples to commented out appendix
|
changeset |
files
|
2010-10-28 |
Cezary Kaliszyk |
Unanonymize qpaper
|
changeset |
files
|
2010-10-28 |
Cezary Kaliszyk |
FSet changes for Qpaper
|
changeset |
files
|
2010-10-28 |
Cezary Kaliszyk |
Remove FSet and use the one from Isabelle
|
changeset |
files
|
2010-10-19 |
Christian Urban |
took out comment about map-types / adapted to recent changes
|
changeset |
files
|
2010-10-19 |
Christian Urban |
use definitions instead of functions
|
changeset |
files
|
2010-10-18 |
Christian Urban |
tuned
|
changeset |
files
|
2010-10-18 |
Christian Urban |
used functions instead of definitions
|
changeset |
files
|
2010-10-18 |
Christian Urban |
added missing style file
|
changeset |
files
|
2010-10-18 |
Cezary Kaliszyk |
Use the generalized compositional quotient theorem
|
changeset |
files
|
2010-10-17 |
Christian Urban |
fixed typo
|
changeset |
files
|
2010-10-17 |
Christian Urban |
all tests work again
|
changeset |
files
|
2010-10-17 |
Christian Urban |
some tuning
|
changeset |
files
|
2010-10-17 |
Christian Urban |
naming scheme is now *_fset (not f*_)
|
changeset |
files
|
2010-10-15 |
Christian Urban |
more cleaning
|
changeset |
files
|
2010-10-15 |
Christian Urban |
further tuning
|
changeset |
files
|
2010-10-15 |
Christian Urban |
renamed fminus_raw to diff_list
|
changeset |
files
|
2010-10-15 |
Christian Urban |
renamed fcard_raw to card_list
|
changeset |
files
|
2010-10-15 |
Christian Urban |
slight update
|
changeset |
files
|
2010-10-15 |
Christian Urban |
Further reorganisation and cleaning
|
changeset |
files
|
2010-10-15 |
Christian Urban |
further cleaning
|
changeset |
files
|
2010-10-15 |
Christian Urban |
typo
|
changeset |
files
|
2010-10-15 |
Cezary Kaliszyk |
FSet: stronger fact in Isabelle.
|
changeset |
files
|
2010-10-15 |
Cezary Kaliszyk |
FSet synchronizing
|
changeset |
files
|
2010-10-15 |
Cezary Kaliszyk |
Synchronizing FSet further.
|
changeset |
files
|
2010-10-15 |
Cezary Kaliszyk |
Partially merging changes from Isabelle
|
changeset |
files
|
2010-10-14 |
Christian Urban |
fixed the typo in the abstract and the problem with append (the type of map_k
|
changeset |
files
|
2010-10-14 |
Christian Urban |
changed format of the pearl paper
|
changeset |
files
|
2010-10-14 |
Christian Urban |
deleted some unused lemmas
|
changeset |
files
|
2010-10-14 |
Christian Urban |
major reorganisation of fset (renamed fset_to_set to fset, changed the definition of list_eq and fcard_raw)
|
changeset |
files
|
2010-10-13 |
Christian Urban |
more on the pearl paper
|
changeset |
files
|
2010-10-12 |
Christian Urban |
added a section about abstractions
|
changeset |
files
|
2010-10-12 |
Christian Urban |
tiny work on the pearl paper
|
changeset |
files
|
2010-10-08 |
Christian Urban |
tuned
|
changeset |
files
|
2010-10-08 |
Christian Urban |
added apendix to paper detailing one proof
|
changeset |
files
|
2010-10-08 |
Christian Urban |
minor
|
changeset |
files
|
2010-10-08 |
Christian Urban |
minor
|
changeset |
files
|
2010-10-08 |
Christian Urban |
down to 20 pages
|
changeset |
files
|
2010-10-07 |
Cezary Kaliszyk |
minor
|
changeset |
files
|
2010-10-06 |
Christian Urban |
down to 21 pages and changed strong induction section
|
changeset |
files
|
2010-10-06 |
Christian Urban |
tuned
|
changeset |
files
|
2010-10-06 |
Christian Urban |
down to 22 pages
|
changeset |
files
|
2010-10-05 |
Christian Urban |
down to 23 pages
|
changeset |
files
|
2010-10-05 |
Christian Urban |
down to 24 pages and a bit
|
changeset |
files
|
2010-10-05 |
Christian Urban |
llncs and more sqeezing
|
changeset |
files
|
2010-10-04 |
Christian Urban |
first part of sqeezing everything into 20 pages (at the moment we have 26)
|
changeset |
files
|
2010-10-04 |
Christian Urban |
changed to llncs
|
changeset |
files
|
2010-10-01 |
Christian Urban |
merged
|
changeset |
files
|
2010-10-01 |
Christian Urban |
minor experiments
|
changeset |
files
|
2010-09-30 |
Christian Urban |
merged
|
changeset |
files
|
2010-09-29 |
Christian Urban |
simplified exhaust proofs
|
changeset |
files
|
2010-10-01 |
Cezary Kaliszyk |
Made the paper to compile with the renamings.
|
changeset |
files
|
2010-09-29 |
Christian Urban |
merged
|
changeset |
files
|
2010-09-29 |
Christian Urban |
worked example Foo1 with induct_schema
|
changeset |
files
|
2010-09-29 |
Christian Urban |
merged
|
changeset |
files
|
2010-09-29 |
Christian Urban |
use also induct_schema for the Let-example (permute_bn is used)
|
changeset |
files
|
2010-09-29 |
Christian Urban |
test with induct_schema for simpler strong_ind proofs
|
changeset |
files
|
2010-09-29 |
Cezary Kaliszyk |
substitution definition with 'next_name'.
|
changeset |
files
|
2010-09-28 |
Christian Urban |
merged
|
changeset |
files
|
2010-09-28 |
Christian Urban |
added Foo1 to explore a contrived example
|
changeset |
files
|
2010-09-27 |
Christian Urban |
added postprocessed fresh-lemmas for constructors
|
changeset |
files
|
2010-09-27 |
Christian Urban |
post-processed eq_iff and supp threormes according to the fv-supp equality
|
changeset |
files
|
2010-09-27 |
Christian Urban |
more consistent naming in Abs.thy
|
changeset |
files
|
2010-09-27 |
Christian Urban |
some experiments
|
changeset |
files
|
2010-09-27 |
Christian Urban |
added simp rules for prod_fv and prod_alpha
|
changeset |
files
|
2010-09-26 |
Christian Urban |
a few more words about Ott
|
changeset |
files
|
2010-09-25 |
Christian Urban |
lifted size_thms and exported them as <name>.size
|
changeset |
files
|
2010-09-25 |
Christian Urban |
cleaned up two examples
|
changeset |
files
|
2010-09-25 |
Christian Urban |
added example about datatypes
|
changeset |
files
|
2010-09-23 |
Christian Urban |
updated to Isabelle 22 Sept
|
changeset |
files
|
2010-09-22 |
Christian Urban |
removed dead code
|
changeset |
files
|
2010-09-22 |
Christian Urban |
fixed
|
changeset |
files
|
2010-09-22 |
Christian Urban |
made supp proofs more robust by not using the standard induction; renamed some example files
|
changeset |
files
|
2010-09-20 |
Christian Urban |
introduced a general procedure for structural inductions; simplified reflexivity proof
|
changeset |
files
|
2010-09-17 |
Christian Urban |
updated to Isabelle Sept 16
|
changeset |
files
|
2010-09-17 |
Christian Urban |
updated to Isabelle Sept 13
|
changeset |
files
|
2010-09-12 |
Christian Urban |
tuned code
|
changeset |
files
|
2010-09-10 |
Christian Urban |
tuned (to conform with indentation policy of Markus)
|
changeset |
files
|
2010-09-10 |
Christian Urban |
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
|
changeset |
files
|
2010-09-04 |
Christian Urban |
generated inducts rule by Project_Rule.projections
|
changeset |
files
|
2010-09-04 |
Christian Urban |
added the definition supp_rel (support w.r.t. a relation)
|
changeset |
files
|
2010-09-04 |
Christian Urban |
merged
|
changeset |
files
|
2010-09-03 |
Christian Urban |
got rid of Nominal2_Supp (is now in Nomina2_Base)
|
changeset |
files
|
2010-09-03 |
Christian Urban |
moved everything out of Nominal_Supp
|
changeset |
files
|
2010-09-03 |
Christian Urban |
renamed alpha_gen -> alpha_set and Abs -> Abs_set etc
|
changeset |
files
|
2010-09-03 |
Christian Urban |
moved a proof to Abs
|
changeset |
files
|
2010-09-03 |
Christian Urban |
got rid of Nominal_Atoms (folded into Nominal2_Base)
|
changeset |
files
|
2010-09-03 |
Christian Urban |
cleaned a bit various thy-files in Nominal-General
|
changeset |
files
|
2010-09-03 |
Christian Urban |
adapted paper to changes
|
changeset |
files
|
2010-09-03 |
Christian Urban |
made the fv-definition aggree more with alpha (needed in the support proofs)
|
changeset |
files
|
2010-09-03 |
Christian Urban |
removed lemma finite_set (already in simpset)
|
changeset |
files
|
2010-09-03 |
Christian Urban |
added supp_set lemma
|
changeset |
files
|
2010-09-02 |
Christian Urban |
some experiments with support
|
changeset |
files
|
2010-09-01 |
Christian Urban |
added eqvt-attribute for permute_abs lemmas
|
changeset |
files
|
2010-08-31 |
Christian Urban |
slides of my talk
|
changeset |
files
|
2010-08-30 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-08-30 |
Cezary Kaliszyk |
update qpaper to new isabelle
|
changeset |
files
|
2010-08-30 |
Cezary Kaliszyk |
No need to unfold mem_def with rsp/prs (requires new isabelle).
|
changeset |
files
|
2010-08-30 |
Cezary Kaliszyk |
Anonymize, change Quotient to Quot and fix indentation
|
changeset |
files
|
2010-08-29 |
Christian Urban |
renamed NewParser to Nominal2
|
changeset |
files
|
2010-08-29 |
Christian Urban |
tuned
|
changeset |
files
|
2010-08-29 |
Christian Urban |
updated todos
|
changeset |
files
|
2010-08-28 |
Christian Urban |
added fs-instance proofs
|
changeset |
files
|
2010-08-28 |
Christian Urban |
added proofs for fsupp properties
|
changeset |
files
|
2010-08-28 |
Christian Urban |
fiexed problem with constructors that have no arguments
|
changeset |
files
|
2010-08-28 |
Christian Urban |
proved supports lemmas
|
changeset |
files
|
2010-08-28 |
Christian Urban |
slight cleaning
|
changeset |
files
|
2010-08-28 |
Christian Urban |
updated to new Isabelle
|
changeset |
files
|
2010-08-27 |
Christian Urban |
cut out most of the lifting section and cleaned up everything
|
changeset |
files
|
2010-08-27 |
Christian Urban |
made all typographic changes
|
changeset |
files
|
2010-08-27 |
Christian Urban |
first pass on section 1
|
changeset |
files
|
2010-08-27 |
Christian Urban |
make copies of the "old" files
|
changeset |
files
|
2010-08-27 |
Cezary Kaliszyk |
Ball Bex can be lifted after unfolding.
|
changeset |
files
|
2010-08-26 |
Christian Urban |
"isabelle make test" makes all major examples....they work up to supp theorems (excluding)
|
changeset |
files
|
2010-08-26 |
Christian Urban |
merged
|
changeset |
files
|
2010-08-26 |
Christian Urban |
corrected bug with fv-function generation (that was the problem with recursive binders)
|
changeset |
files
|
2010-08-26 |
Cezary Kaliszyk |
minor
|
changeset |
files
|
2010-08-25 |
Christian Urban |
cleaned up (almost completely) the examples
|
changeset |
files
|
2010-08-25 |
Christian Urban |
cleaning of unused files and code
|
changeset |
files
|
2010-08-25 |
Christian Urban |
automatic lifting
|
changeset |
files
|
2010-08-25 |
Christian Urban |
everything now lifts as expected
|
changeset |
files
|
2010-08-25 |
Christian Urban |
now every lemma lifts (even with type variables)
|
changeset |
files
|
2010-08-25 |
Christian Urban |
can now deal with type variables in nominal datatype definitions
|
changeset |
files
|
2010-08-22 |
Christian Urban |
updated to new Isabelle
|
changeset |
files
|
2010-08-22 |
Christian Urban |
merged
|
changeset |
files
|
2010-08-22 |
Christian Urban |
updated to new Isabelle
|
changeset |
files
|
2010-08-21 |
Christian Urban |
not needed anymore
|
changeset |
files
|
2010-08-21 |
Christian Urban |
moved lifting code from Lift.thy to nominal_dt_quot.ML
|
changeset |
files
|
2010-08-21 |
Christian Urban |
nominal_datatypes with type variables do not work
|
changeset |
files
|
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
|
changeset |
files
|
2010-08-20 |
Cezary Kaliszyk |
Clarifications to FIXMEs.
|
changeset |
files
|
2010-08-20 |
Cezary Kaliszyk |
Finished adding remarks from the reviewers.
|
changeset |
files
|
2010-08-20 |
Cezary Kaliszyk |
few remaining remarks as fixme's.
|
changeset |
files
|
2010-08-19 |
Christian Urban |
used @{const_name} hopefully everywhere
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
Intuition behind REL
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
add missing mathpartir
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
Add 2 FIXMEs
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
The type does determine respectfulness, the constant without an instantiated type does not.
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
Add the SAC stylesheet and updated root file.
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
TODO
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
further comments from the referees
|
changeset |
files
|
2010-08-19 |
Cezary Kaliszyk |
fixes for referees
|
changeset |
files
|
2010-08-17 |
Christian Urban |
put everything in a "timeit"
|
changeset |
files
|
2010-08-17 |
Christian Urban |
improved runtime slightly, by constructing an explicit size measure for the function definitions
|
changeset |
files
|
2010-08-17 |
Christian Urban |
more tuning of the code
|
changeset |
files
|
2010-08-17 |
Christian Urban |
deleted unused code
|
changeset |
files
|
2010-08-17 |
Christian Urban |
improved code
|
changeset |
files
|
2010-08-16 |
Christian Urban |
can also lift the various eqvt lemmas for bn, fv, fv_bn and size
|
changeset |
files
|
2010-08-16 |
Christian Urban |
also able to lift the bn_defs
|
changeset |
files
|
2010-08-16 |
Christian Urban |
added rsp-lemmas for alpha_bns
|
changeset |
files
|
2010-08-16 |
Christian Urban |
cezary made the eq_iff lemmas to lift (still needs some infrastructure in quotient)
|
changeset |
files
|
2010-08-16 |
Christian Urban |
pinpointed the problem
|
changeset |
files
|
2010-08-16 |
Christian Urban |
modified the code for class instantiations (with help from Florian)
|
changeset |
files
|
2010-08-15 |
Christian Urban |
defined qperms and qsizes
|
changeset |
files
|
2010-08-15 |
Christian Urban |
simplified code
|
changeset |
files
|
2010-08-14 |
Christian Urban |
improved code
|
changeset |
files
|
2010-08-14 |
Christian Urban |
more experiments with lifting
|
changeset |
files
|
2010-08-12 |
Christian Urban |
updated to Isabelle 12th Aug
|
changeset |
files
|
2010-08-11 |
Christian Urban |
rsp for constructors
|
changeset |
files
|
2010-08-11 |
Christian Urban |
updated to Isabelle 11 Aug
|
changeset |
files
|
2010-08-11 |
Christian Urban |
added a function that transforms the helper-rsp lemmas into real rsp lemmas
|
changeset |
files
|
2010-08-08 |
Christian Urban |
proved rsp-helper lemmas of size functions
|
changeset |
files
|
2010-07-31 |
Christian Urban |
tuning
|
changeset |
files
|
2010-07-31 |
Christian Urban |
further simplification with alpha_prove
|
changeset |
files
|
2010-07-31 |
Christian Urban |
introduced a general alpha_prove method
|
changeset |
files
|
2010-07-29 |
Christian Urban |
equivariance for size
|
changeset |
files
|
2010-07-29 |
Christian Urban |
helper lemmas for rsp-lemmas
|
changeset |
files
|
2010-07-27 |
Christian Urban |
tests
|
changeset |
files
|
2010-07-27 |
Christian Urban |
cleaned up a bit Abs.thy
|
changeset |
files
|
2010-07-27 |
Christian Urban |
fixed order of fold_union to make alpha and fv agree
|
changeset |
files
|
2010-07-26 |
Christian Urban |
small cleaning
|
changeset |
files
|
2010-07-25 |
Christian Urban |
added paper by james; some minor cleaning
|
changeset |
files
|
2010-07-23 |
Christian Urban |
samll changes
|
changeset |
files
|
2010-07-23 |
Christian Urban |
made compatible
|
changeset |
files
|
2010-07-23 |
Christian Urban |
added
|
changeset |
files
|
2010-07-22 |
Christian Urban |
updated to new Isabelle; made FSet more "quiet"
|
changeset |
files
|
2010-07-20 |
Christian Urban |
merged
|
changeset |
files
|
2010-07-19 |
Christian Urban |
minor
|
changeset |
files
|
2010-07-19 |
Christian Urban |
minor polishing
|
changeset |
files
|
2010-07-19 |
Christian Urban |
quote for a new paper
|
changeset |
files
|
2010-07-19 |
Christian Urban |
corrected lambda-preservation theorem
|
changeset |
files
|
2010-07-19 |
Christian Urban |
minor
|
changeset |
files
|
2010-07-18 |
Christian Urban |
minor things on the paper
|
changeset |
files
|
2010-07-18 |
Christian Urban |
merged
|
changeset |
files
|
2010-07-18 |
Christian Urban |
minor things
|
changeset |
files
|
2010-07-18 |
Christian Urban |
some test with quotient
|
changeset |
files
|
2010-07-17 |
Christian Urban |
some minor changes
|
changeset |
files
|
2010-07-17 |
Christian Urban |
changes suggested by Peter Homeier
|
changeset |
files
|
2010-07-17 |
Christian Urban |
tests
|
changeset |
files
|
2010-07-16 |
Christian Urban |
submitted version
|
changeset |
files
|
2010-07-16 |
Christian Urban |
more paper
|
changeset |
files
|
2010-07-16 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-16 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-15 |
Christian Urban |
a bit more to the paper
|
changeset |
files
|
2010-07-14 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-13 |
Christian Urban |
more on slides
|
changeset |
files
|
2010-07-13 |
Christian Urban |
slides
|
changeset |
files
|
2010-07-12 |
Christian Urban |
more on slides
|
changeset |
files
|
2010-07-11 |
Christian Urban |
slides
|
changeset |
files
|
2010-07-10 |
Christian Urban |
slides
|
changeset |
files
|
2010-07-10 |
Christian Urban |
more on slides
|
changeset |
files
|
2010-07-10 |
Christian Urban |
more on slides
|
changeset |
files
|
2010-07-10 |
Christian Urban |
added material for slides
|
changeset |
files
|
2010-07-09 |
Christian Urban |
fixed
|
changeset |
files
|
2010-07-09 |
Christian Urban |
before examples
|
changeset |
files
|
2010-07-09 |
Christian Urban |
finished alpha-section
|
changeset |
files
|
2010-07-07 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-07 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-02 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-02 |
Christian Urban |
finished fv-section
|
changeset |
files
|
2010-07-01 |
Christian Urban |
more on the paper
|
changeset |
files
|
2010-07-01 |
Christian Urban |
spell check
|
changeset |
files
|
2010-06-30 |
Christian Urban |
more work on the paper
|
changeset |
files
|
2010-06-29 |
Christian Urban |
removed an "eqvt"-warning
|
changeset |
files
|
2010-06-28 |
Christian Urban |
more quotient-definitions
|
changeset |
files
|
2010-06-28 |
Christian Urban |
slight cleaning
|
changeset |
files
|
2010-06-27 |
Christian Urban |
fixed according to changes in quotient
|
changeset |
files
|
2010-06-24 |
Christian Urban |
added definition of the quotient types
|
changeset |
files
|
2010-06-24 |
Christian Urban |
fixed according to changes in quotient
|
changeset |
files
|
2010-06-23 |
Christian Urban |
added comment about partial equivalence relations
|
changeset |
files
|
2010-06-23 |
Christian Urban |
even further polishing of the qpaper
|
changeset |
files
|
2010-06-23 |
Christian Urban |
polished paper again (and took out some claims about Homeier's package)
|
changeset |
files
|
2010-06-23 |
Christian Urban |
some slight polishing on the paper
|
changeset |
files
|
2010-06-23 |
Christian Urban |
merged cezary's changes
|
changeset |
files
|
2010-06-23 |
Christian Urban |
whitespace
|
changeset |
files
|
2010-06-23 |
Cezary Kaliszyk |
Un-do the second change to SingleLet.
|
changeset |
files
|
2010-06-23 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-06-23 |
Cezary Kaliszyk |
Changes for PER and list_all2 committed to Isabelle
|
changeset |
files
|
2010-06-18 |
Cezary Kaliszyk |
changes for partial-equivalence quotient package
|
changeset |
files
|
2010-06-23 |
Christian Urban |
deleted compose-lemmas in Abs (not needed anymore)
|
changeset |
files
|
2010-06-23 |
Christian Urban |
deleted equivp_hack
|
changeset |
files
|
2010-06-22 |
Christian Urban |
proved eqvip theorems for alphas
|
changeset |
files
|
2010-06-22 |
Christian Urban |
cleaned up the FSet (noise was introduced by error)
|
changeset |
files
|
2010-06-22 |
Christian Urban |
prove that alpha implies alpha_bn (needed for rsp proofs)
|
changeset |
files
|
2010-06-21 |
Christian Urban |
further post-submission tuning
|
changeset |
files
|
2010-06-21 |
Christian Urban |
merged with main line
|
changeset |
files
|
2010-06-21 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-11 |
Christian Urban |
also symmetry
|
changeset |
files
|
2010-06-10 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-10 |
Christian Urban |
premerge
|
changeset |
files
|
2010-06-09 |
Christian Urban |
transitivity proofs done
|
changeset |
files
|
2010-06-07 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-07 |
Christian Urban |
work on transitivity proof
|
changeset |
files
|
2010-06-03 |
Christian Urban |
added uminus_eqvt
|
changeset |
files
|
2010-06-03 |
Christian Urban |
fixed problem with eqvt proofs
|
changeset |
files
|
2010-06-02 |
Christian Urban |
fixed problem with bn_info
|
changeset |
files
|
2010-06-01 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-01 |
Christian Urban |
equivariance done
|
changeset |
files
|
2010-06-01 |
Christian Urban |
smaller code for raw-eqvt proofs
|
changeset |
files
|
2010-05-31 |
Christian Urban |
all raw definitions are defined using function
|
changeset |
files
|
2010-05-27 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-27 |
Christian Urban |
intermediate state
|
changeset |
files
|
2010-05-26 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-26 |
Christian Urban |
added FSet to the correct paper
|
changeset |
files
|
2010-05-24 |
Christian Urban |
added slides
|
changeset |
files
|
2010-05-24 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-24 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-24 |
Christian Urban |
alpha works now
|
changeset |
files
|
2010-05-23 |
Christian Urban |
started to work on alpha
|
changeset |
files
|
2010-05-22 |
Christian Urban |
properly exported bn_descr
|
changeset |
files
|
2010-05-21 |
Christian Urban |
hving a working fv-definition without the export
|
changeset |
files
|
2010-05-21 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-20 |
Christian Urban |
proper parser for "exclude:"
|
changeset |
files
|
2010-05-20 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-20 |
Christian Urban |
moved some mk_union and mk_diff into the library
|
changeset |
files
|
2010-05-20 |
Christian Urban |
new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
|
changeset |
files
|
2010-06-21 |
Christian Urban |
some post-submission polishing
|
changeset |
files
|
2010-06-20 |
Christian Urban |
added a few points that need to be looked at the next version of the qpaper
|
changeset |
files
|
2010-06-20 |
Christian Urban |
eliminated a quot_thm flag
|
changeset |
files
|
2010-06-20 |
Christian Urban |
fixed example
|
changeset |
files
|
2010-06-20 |
Christian Urban |
small addition to the acknowledgement
|
changeset |
files
|
2010-06-17 |
Cezary Kaliszyk |
qpaper / address FIXMEs.
|
changeset |
files
|
2010-06-17 |
Cezary Kaliszyk |
forgot to save
|
changeset |
files
|
2010-06-17 |
Cezary Kaliszyk |
Fix regularization. Two "FIXME" left in introduction. Minor spellings.
|
changeset |
files
|
2010-06-16 |
Christian Urban |
polished everything and submitted
|
changeset |
files
|
2010-06-16 |
Christian Urban |
conclusion done
|
changeset |
files
|
2010-06-16 |
Cezary Kaliszyk |
Answer questions in comments
|
changeset |
files
|
2010-06-16 |
Christian Urban |
tuned
|
changeset |
files
|
2010-06-16 |
Christian Urban |
finished section 4, but put some things I do not understand on comment
|
changeset |
files
|
2010-06-16 |
Christian Urban |
4 almost finished
|
changeset |
files
|
2010-06-15 |
Christian Urban |
cleaned up definitions
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
qpaper/Rewrite section5
|
changeset |
files
|
2010-06-15 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-15 |
Christian Urban |
tuned everytinh up to section 4
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
Definition of Respects.
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
conclusion
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
Qpaper / Clarify the typing system and composition of quotients issue.
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
Remove only reference to 'equivp'.
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
qpaper/ackno
|
changeset |
files
|
2010-06-15 |
Christian Urban |
tuned
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
qpaper / hol4
|
changeset |
files
|
2010-06-15 |
Cezary Kaliszyk |
qpaper/related work
|
changeset |
files
|
2010-06-15 |
Christian Urban |
finished preliminary section
|
changeset |
files
|
2010-06-14 |
Christian Urban |
typo
|
changeset |
files
|
2010-06-14 |
Christian Urban |
some slight tuning of the preliminary section
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-06-14 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-14 |
Christian Urban |
tuned
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
Qpaper / beginnig of sec5
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper/unfold the ball_reg_right statement
|
changeset |
files
|
2010-06-14 |
Christian Urban |
merged
|
changeset |
files
|
2010-06-14 |
Christian Urban |
some tuning and start work on section 4
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper / INJ
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper / REG
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper / minor
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper/various
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper/more on example
|
changeset |
files
|
2010-06-14 |
Cezary Kaliszyk |
qpaper/examples
|
changeset |
files
|
2010-06-14 |
Christian Urban |
completed proof and started section about respectfulness and preservation
|
changeset |
files
|
2010-06-13 |
Christian Urban |
more on the qpaper
|
changeset |
files
|
2010-06-13 |
Christian Urban |
tuned
|
changeset |
files
|
2010-06-13 |
Christian Urban |
more on the constant lifting section
|
changeset |
files
|
2010-06-13 |
Christian Urban |
something about the quotient ype definitions
|
changeset |
files
|
2010-06-13 |
Christian Urban |
added some examples
|
changeset |
files
|
2010-06-13 |
Christian Urban |
improved definition of ABS and REP
|
changeset |
files
|
2010-06-13 |
Cezary Kaliszyk |
qpaper.
|
changeset |
files
|
2010-06-13 |
Cezary Kaliszyk |
some spelling
|
changeset |
files
|
2010-06-13 |
Cezary Kaliszyk |
minor
|
changeset |
files
|
2010-06-13 |
Cezary Kaliszyk |
qpaper / tuning in preservation and general display
|
changeset |
files
|
2010-06-13 |
Christian Urban |
polishing of ABS/REP
|
changeset |
files
|
2010-06-12 |
Christian Urban |
some slight tuning of the intro
|
changeset |
files
|
2010-06-12 |
Cezary Kaliszyk |
Fix integer relation.
|
changeset |
files
|
2010-06-12 |
Christian Urban |
completed the intro (except minor things)
|
changeset |
files
|
2010-06-11 |
Christian Urban |
more intro
|
changeset |
files
|
2010-06-11 |
Christian Urban |
more on the qpaper
|
changeset |
files
|
2010-06-11 |
Christian Urban |
even more on the qpaper (intro almost done)
|
changeset |
files
|
2010-06-11 |
Christian Urban |
more to the introduction of the qpaper
|
changeset |
files
|
2010-06-10 |
Christian Urban |
adapted to the official sigplan style file (this gives us more space)
|
changeset |
files
|
2010-06-10 |
Christian Urban |
added to the popl-paper a pointer to work by Altenkirch
|
changeset |
files
|
2010-06-10 |
Christian Urban |
more on the qpaper
|
changeset |
files
|
2010-06-07 |
Christian Urban |
new title for POPL paper
|
changeset |
files
|
2010-06-07 |
Christian Urban |
more work on intro and abstract (done for today)
|
changeset |
files
|
2010-06-07 |
Christian Urban |
a bit more in the introduction and abstract
|
changeset |
files
|
2010-06-07 |
Christian Urban |
improved abstract, some tuning
|
changeset |
files
|
2010-06-06 |
Cezary Kaliszyk |
Qpaper / minor on cleaning
|
changeset |
files
|
2010-06-05 |
Cezary Kaliszyk |
qpaper / injection proof.
|
changeset |
files
|
2010-06-05 |
Cezary Kaliszyk |
qpaper / example interaction
|
changeset |
files
|
2010-06-05 |
Cezary Kaliszyk |
Qpaper/regularization proof.
|
changeset |
files
|
2010-06-05 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-06-02 |
Cezary Kaliszyk |
Qpaper/more.
|
changeset |
files
|
2010-06-02 |
Cezary Kaliszyk |
Qpaper/Minor
|
changeset |
files
|
2010-06-01 |
Christian Urban |
added larry's quote
|
changeset |
files
|
2010-06-01 |
Christian Urban |
added larry's paper
|
changeset |
files
|
2010-06-01 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-28 |
Christian Urban |
first version of the abstract
|
changeset |
files
|
2010-05-27 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-27 |
Christian Urban |
fixed bug where perm_simp 'forgets' how to prove equivariance for the empty set
|
changeset |
files
|
2010-05-27 |
Cezary Kaliszyk |
qpaper / lemmas used in proofs
|
changeset |
files
|
2010-05-27 |
Cezary Kaliszyk |
qpaper / injection statement
|
changeset |
files
|
2010-05-27 |
Cezary Kaliszyk |
qpaper / regularize
|
changeset |
files
|
2010-05-27 |
Cezary Kaliszyk |
qpaper / a bit about prs
|
changeset |
files
|
2010-05-27 |
Cezary Kaliszyk |
Functionalized the ABS/REP definition.
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper / lifting introduction
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
merged
|
changeset |
files
|
2010-05-26 |
Christian Urban |
fixed compile error
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper / composition of quotients.
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper..
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper.
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
Name some respectfullness
|
changeset |
files
|
2010-05-26 |
Christian Urban |
added FSet to the correct paper
|
changeset |
files
|
2010-05-26 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-26 |
Christian Urban |
added FSet
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-05-26 |
Cezary Kaliszyk |
qpaper
|
changeset |
files
|
2010-05-25 |
Cezary Kaliszyk |
Substitution Lemma for TypeSchemes.
|
changeset |
files
|
2010-05-25 |
Cezary Kaliszyk |
Simplified the proof
|
changeset |
files
|
2010-05-25 |
Cezary Kaliszyk |
A lemma about substitution in TypeSchemes.
|
changeset |
files
|
2010-05-25 |
Cezary Kaliszyk |
reversing the direction of fresh_star
|
changeset |
files
|
2010-05-25 |
Cezary Kaliszyk |
overlapping deep binders proof
|
changeset |
files
|
2010-05-25 |
Christian Urban |
edits from the reviewers
|
changeset |
files
|
2010-05-24 |
Christian Urban |
tuned paper
|
changeset |
files
|
2010-05-23 |
Christian Urban |
changed qpaper to lncs-style
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Match_Lam defined on Quotient Level.
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
More on Function-defined subst.
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Isabelle renamings
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Renamings.
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Renamings
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
merge (non-trival)
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Previously uncommited direct subst definition changes.
|
changeset |
files
|
2010-05-21 |
Cezary Kaliszyk |
Function experiments
|
changeset |
files
|
2010-05-19 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-19 |
Christian Urban |
added comments about pottiers work
|
changeset |
files
|
2010-05-19 |
Cezary Kaliszyk |
more subst experiments
|
changeset |
files
|
2010-05-19 |
Cezary Kaliszyk |
More subst experminets
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
more on subst
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
Single variable substitution
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
subst fix
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
subst experiments
|
changeset |
files
|
2010-05-18 |
Christian Urban |
soem minor tuning
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
Fix broken add
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
add missing .bib
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-18 |
Cezary Kaliszyk |
starting bibliography
|
changeset |
files
|
2010-05-17 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-17 |
Christian Urban |
updated to new Isabelle (More_Conv -> Conv)
|
changeset |
files
|
2010-05-17 |
Christian Urban |
made this example to work again
|
changeset |
files
|
2010-05-17 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-17 |
Cezary Kaliszyk |
alpha_alphabn for bindings in a type under bn.
|
changeset |
files
|
2010-05-17 |
Christian Urban |
minor tuning
|
changeset |
files
|
2010-05-17 |
Cezary Kaliszyk |
Ex4 does work, and I don't see the difference between the alphas.
|
changeset |
files
|
2010-05-17 |
Christian Urban |
slight tuning
|
changeset |
files
|
2010-05-17 |
Christian Urban |
somewhat simplified the main parsing function; failed to move a Note-statement to define_raw_perms
|
changeset |
files
|
2010-05-16 |
Christian Urban |
moved the exporting part into the parser (this is still a hack); re-added CoreHaskell again to the examples - there seems to be a problem with the variable name pat
|
changeset |
files
|
2010-05-16 |
Christian Urban |
tuned paper
|
changeset |
files
|
2010-05-15 |
Christian Urban |
tuned paper
|
changeset |
files
|
2010-05-14 |
Christian Urban |
tuned a bit the paper
|
changeset |
files
|
2010-05-14 |
Christian Urban |
started a new file for the parser to make some experiments
|
changeset |
files
|
2010-05-14 |
Christian Urban |
moved old parser and fv into attic
|
changeset |
files
|
2010-05-14 |
Christian Urban |
polished example
|
changeset |
files
|
2010-05-14 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-14 |
Christian Urban |
tuned a bit the paper
|
changeset |
files
|
2010-05-14 |
Cezary Kaliszyk |
Proper fv/alpha for multiple compound binders
|
changeset |
files
|
2010-05-14 |
Cezary Kaliszyk |
SingleLetFoo with everything.
|
changeset |
files
|
2010-05-14 |
Cezary Kaliszyk |
Fv for multiple binding functions
|
changeset |
files
|
2010-05-13 |
Christian Urban |
added a more instructive example - has some problems with fv though
|
changeset |
files
|
2010-05-13 |
Christian Urban |
added flip_eqvt and swap_eqvt to the equivariance lists
|
changeset |
files
|
2010-05-13 |
Christian Urban |
tuned the paper
|
changeset |
files
|
2010-05-13 |
Christian Urban |
properly declared outer keyword
|
changeset |
files
|
2010-05-13 |
Christian Urban |
added an example which goes outside our current speciifcation
|
changeset |
files
|
2010-05-13 |
Christian Urban |
made out of STEPS a configuration value so that it can be set individually in each file
|
changeset |
files
|
2010-05-13 |
Christian Urban |
tuned eqvt-proofs about prod_rel and prod_fv
|
changeset |
files
|
2010-05-13 |
Christian Urban |
removed internal functions from the signature (they are not needed anymore)
|
changeset |
files
|
2010-05-13 |
Christian Urban |
added term4 back to the examples
|
changeset |
files
|
2010-05-13 |
Cezary Kaliszyk |
Make Term4 use 'equivariance'.
|
changeset |
files
|
2010-05-12 |
Christian Urban |
fixed the examples for the new eqvt-procedure....temporarily disabled Manual/Term4.thy
|
changeset |
files
|
2010-05-12 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-12 |
Christian Urban |
moved the data-transformation into the parser
|
changeset |
files
|
2010-05-12 |
Christian Urban |
added a test whether some of the constants already equivariant (then the procedure has to fail).
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
include set_simps and append_simps in fv_rsp
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
Move alpha_eqvt to unused.
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
Use equivariance instead of alpha_eqvt
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
fvbv_rsp include prod_rel.simps
|
changeset |
files
|
2010-05-12 |
Christian Urban |
better ML-interface (returning only a list of theorems and a context)
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-12 |
Cezary Kaliszyk |
Use raw_induct instead of induct
|
changeset |
files
|
2010-05-12 |
Christian Urban |
ingnored parameters in equivariance; added a proper interface to be called from ML
|
changeset |
files
|
2010-05-12 |
Christian Urban |
properly exported defined bn-functions
|
changeset |
files
|
2010-05-11 |
Cezary Kaliszyk |
Include raw permutation definitions in eqvt
|
changeset |
files
|
2010-05-11 |
Cezary Kaliszyk |
Declare alpha_gen_eqvt as eqvt and change the proofs that used 'eqvts[symmetric]'
|
changeset |
files
|
2010-05-11 |
Christian Urban |
a bit for the introduction of the q-paper
|
changeset |
files
|
2010-05-11 |
Christian Urban |
added some of the quotient literature; a bit more to the qpaper
|
changeset |
files
|
2010-05-10 |
Christian Urban |
fixed a problem with non-existant alphas2
|
changeset |
files
|
2010-05-10 |
Christian Urban |
added comment about bind_set
|
changeset |
files
|
2010-05-10 |
Christian Urban |
fixing bind_set problem
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Term8 comment
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Restore set bindings in CoreHaskell
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Recursive examples with relation composition
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
prod_rel and prod_fv eqvt and mono
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
ExLetRec
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Parser changes for compound relations
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Use mk_compound_fv' and mk_compound_rel'
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Membership in a pair of lists.
|
changeset |
files
|
2010-05-10 |
Cezary Kaliszyk |
Synchronize FSet with repository
|
changeset |
files
|
2010-05-09 |
Christian Urban |
tuned file names for examples
|
changeset |
files
|
2010-05-09 |
Christian Urban |
cleaned up a bit the examples; added equivariance to all examples
|
changeset |
files
|
2010-05-09 |
Christian Urban |
fixed the problem with alpha containing splits
|
changeset |
files
|
2010-05-09 |
Christian Urban |
added eqvt-lemma for split; changed semantics of perm_simp: excluded stands for constants about which no complaint is written out...eqvt_apply is now always applied
|
changeset |
files
|
2010-05-07 |
Cezary Kaliszyk |
Manually added some newer keywords from the distribution
|
changeset |
files
|
2010-05-07 |
Cezary Kaliszyk |
Regularize experiments
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
alpha_eqvt_tac with prod_rel and prod_fv simps
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
mem => member
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
Fixes for new Isabelle
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
compound versions with prod_rel and prod_fun, not made default yet.
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
prod_rel and prod_fv simps
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
mem => member
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
prod_rel.simps and Fixed for new isabelle
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
Fixes for new isabelle
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
prod_fv and its respectfullness and preservation.
|
changeset |
files
|
2010-05-06 |
Cezary Kaliszyk |
Experiments with equivariance.
|
changeset |
files
|
2010-05-05 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-05 |
Christian Urban |
a bit mor on the pearl journal paper
|
changeset |
files
|
2010-05-05 |
Christian Urban |
solved the problem with equivariance by first eta-normalising the goal
|
changeset |
files
|
2010-05-05 |
Cezary Kaliszyk |
Some cleaning in Term4
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
"isabelle make" compiles all examples with newparser/newfv/newalpha only.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move Term4 to NewParser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Fix Term4 for permutation signature change
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move LF to NewParser. Just works.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
ExLetMult
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Ex1Rec.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
ExPS3 in NewParser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move ExPS8 to new parser.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Fix for new isabelle
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Minor
|
changeset |
files
|
2010-05-04 |
Christian Urban |
increased step counter so that all steps go through
|
changeset |
files
|
2010-05-04 |
Christian Urban |
fixed my error with define_raw_fv
|
changeset |
files
|
2010-05-04 |
Christian Urban |
tuned and added some comments to the code; added also an exception for early exit of the nominal2_cmd function
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Separate Term8, as it may work soon.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
moved CoreHaskell to NewParser.
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
ExPS7 in NewParser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move ExLeroy to New Parser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move 2 more to NewParser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move TypeSchemes to NewParser
|
changeset |
files
|
2010-05-04 |
Cezary Kaliszyk |
Move ExLet to NewParser.
|
changeset |
files
|
2010-05-04 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-04 |
Christian Urban |
roll back of the last commit (there was a difference)
|
changeset |
files
|
2010-05-04 |
Christian Urban |
tuned
|
changeset |
files
|
2010-05-04 |
Christian Urban |
to my best knowledge the number of datatypes is equal to the length of the dt_descr; so we can save one argument in define_raw_perm
|
changeset |
files
|
2010-05-04 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-04 |
Christian Urban |
some preliminary changes to the pearl-jv paper
|
changeset |
files
|
2010-05-03 |
Christian Urban |
some preliminary notes of the abstract (qpaper); still need to see the motivating example
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Added cheats to classical
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Ex2 moved to new parser.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
alpha_eqvt_tac fixed to work when the existential is not at the top level.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
SingleLet and Ex3 work with NewParser.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Comment
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Another example where only alpha_eqvt fails.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Register only non-looping rules in eq_iff
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Equivariance fails for single let?
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
NewParser
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Introduce eq_iff_simp to match the one from Parser.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
remove tracing
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Cheat support equations in new parser
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Remove dependency on NewFv
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Fix Parser
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Add explicit cheats in NewParser and comment out the examples for outside use.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Fix Datatype_Aux calls in NewParser.
|
changeset |
files
|
2010-05-03 |
Cezary Kaliszyk |
Move old fv_alpha_export to Fv.
|
changeset |
files
|
2010-05-02 |
Christian Urban |
moved old parser and old fv back into their original places; isabelle make works again
|
changeset |
files
|
2010-05-02 |
Christian Urban |
slight tuning
|
changeset |
files
|
2010-05-02 |
Christian Urban |
simplified the supp-of-finite-sets proof
|
changeset |
files
|
2010-05-02 |
Christian Urban |
tried to add some comments in the huge(!) nominal2_cmd function
|
changeset |
files
|
2010-05-02 |
Christian Urban |
replaced make_pair with library function HOLogic.mk_prod
|
changeset |
files
|
2010-05-02 |
Christian Urban |
removed duplicate eqvt attribute
|
changeset |
files
|
2010-05-02 |
Christian Urban |
attempted to remove dependency on (old) Fv and (old) Parser; lifting still uses Fv.thy; the examples do not work at the moment (with equivp proofs failing)
|
changeset |
files
|
2010-05-01 |
Christian Urban |
merged
|
changeset |
files
|
2010-05-01 |
Christian Urban |
tuned
|
changeset |
files
|
2010-04-30 |
Christian Urban |
replaced hide by the new hide_const
|
changeset |
files
|