Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1920
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
some code refactoring
2011-07-08, by Christian Urban
merged
2011-07-07, by Christian Urban
code refactoring; introduced a record for raw_dt_info
2011-07-07, by Christian Urban
more on NBE
2011-07-06, by Christian Urban
more on the NBE function
2011-07-06, by Christian Urban
a little further with NBE
2011-07-06, by Christian Urban
Setup eqvt_at for first goal
2011-07-06, by Cezary Kaliszyk
attempt for NBE
2011-07-06, by Christian Urban
added some relatively simple examples from paper by Norrish
2011-07-05, by Christian Urban
changed bind to binds in specifications; bind will cause trouble with Monad_Syntax
2011-07-05, by Christian Urban
side commment for future use
2011-07-05, by Christian Urban
made the tests go through again
2011-07-05, by Christian Urban
added another example which seems difficult to define
2011-07-05, by Christian Urban
added a tactic "all_trivials" which simplifies all trivial constructor cases and leaves the others untouched.
2011-07-05, by Christian Urban
merged
2011-07-05, by Christian Urban
all FCB lemmas
2011-07-05, by Christian Urban
exported various FCB-lemmas to a separate file
2011-07-05, by Christian Urban
Express trans_db with Option.map and Option.bind. Possibly mbind is a copy of bind?
2011-07-05, by Cezary Kaliszyk
Define a version of aux only for same binders. Completeness is fine.
2011-07-05, by Cezary Kaliszyk
Move If / Let with 'True' to the end of Lambda
2011-07-05, by Cezary Kaliszyk
merged
2011-07-04, by Christian Urban
tuned
2011-07-04, by Christian Urban
added an example that recurses over two arguments; the interesting proof-obligation is not yet done
2011-07-04, by Christian Urban
Let with a different invariant; not true.
2011-07-04, by Cezary Kaliszyk
Add non-working Lambda_F_T using FCB2
2011-07-03, by Cezary Kaliszyk
Added non-working CPS3 using FCB2
2011-07-03, by Cezary Kaliszyk
Change CPS1 to FCB2
2011-07-03, by Cezary Kaliszyk
Did the proofs of height and subst for Let with list-like binders. Having apply_assns allows proving things by alpha_bn
2011-07-02, by Cezary Kaliszyk
side-by-side tests of lets with single assignment; deep-binder case works if the recursion is avoided using an auxiliary function
2011-07-02, by Christian Urban
Exhaust Issue
2011-07-01, by Cezary Kaliszyk
clarified a sentence
2011-06-30, by Christian Urban
more code refactoring
2011-06-30, by Christian Urban
combined distributed data for alpha in alpha_result (partially done)
2011-06-29, by Christian Urban
moved Classical and Let temporarily into a section where "sorry" is allowed; this makes all test go through
2011-06-29, by Christian Urban
added a warning if a theorem is already declared as equivariant
2011-06-29, by Christian Urban
merged
2011-06-29, by Christian Urban
Prove bn injectivity and experiment more with Let
2011-06-29, by Cezary Kaliszyk
some experiments
2011-06-29, by Christian Urban
trying new fcb in let/subst
2011-06-28, by Cezary Kaliszyk
Leftover only inj and eqvt
2011-06-28, by Cezary Kaliszyk
eapply fcb ok
2011-06-28, by Cezary Kaliszyk
Removed Inl and Inr
2011-06-28, by Cezary Kaliszyk
relaxed type in fcb
2011-06-28, by Christian Urban
fcb with explicit bn function
2011-06-28, by Christian Urban
added let-rec example
2011-06-28, by Christian Urban
Experiments with res
2011-06-28, by Cezary Kaliszyk
proved the fcb also for sets (no restriction yet)
2011-06-28, by Christian Urban
copied all work to Lambda.thy; had to derive a special version of fcb1 for concrete atom
2011-06-28, by Christian Urban
streamlined the fcb-proof and made fcb1 a special case of fcb
2011-06-27, by Christian Urban
completed proof in Classical; the fcb lemma works for any list of atoms (despite what was written earlier)
2011-06-27, by 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.
2011-06-27, by Christian Urban
renamed ds to dset (disagreement set)
2011-06-27, by Christian Urban
added small lemma about disagreement set
2011-06-27, by Christian Urban
merge
2011-06-27, by Cezary Kaliszyk
New-style fcb for multiple binders.
2011-06-27, by Cezary Kaliszyk
equality of lst_binder and a few helper lemmas
2011-06-27, by Cezary Kaliszyk
only one of the fcb precondistions are needed (probably the same with the perm-conditions)
2011-06-26, by Christian Urban
another change to the fcb2; this is needed in order to get all proofs through in Lambda.thy
2011-06-26, by Christian Urban
did all cases, except the multiple binder case
2011-06-25, by 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.
2011-06-25, by Christian Urban
except for the interated binder case, finished definition in Calssical.thy
2011-06-24, by Christian Urban
Make examples work with non-precompiled image
2011-06-24, by Cezary Kaliszyk
Remove Lambda_add.thy
2011-06-24, by Cezary Kaliszyk
The examples in Lambda_add can be defined by nominal_function directly
2011-06-24, by Cezary Kaliszyk
Theory name changes for JEdit
2011-06-24, by Cezary Kaliszyk
More usual names for substitution properties
2011-06-24, by Cezary Kaliszyk
Second Fixed Point Theorem
2011-06-24, by Cezary Kaliszyk
Speed-up the completeness proof.
2011-06-24, by Cezary Kaliszyk
the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
2011-06-23, by Christian Urban
added file
2011-06-23, by Christian Urban
expanded the example
2011-06-23, by 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
2011-06-23, by Christian Urban
tuned
2011-06-22, by Christian Urban
deleted some dead code
2011-06-22, by Christian Urban
some rudimentary infrastructure for storing data about nominal datatypes
2011-06-22, by Christian Urban
constants with the same names
2011-06-22, by Cezary Kaliszyk
Quotients/TODO addtion
2011-06-22, by Cezary Kaliszyk
Minor
2011-06-21, by Cezary Kaliszyk
merge
2011-06-21, by Cezary Kaliszyk
spelling
2011-06-21, by Cezary Kaliszyk
merge
2011-06-20, by Cezary Kaliszyk
Abs_set_fcb
2011-06-20, by Cezary Kaliszyk
function for let-rec
2011-06-20, by Cezary Kaliszyk
TODO/minor
2011-06-20, by Cezary Kaliszyk
Move lst_fcb to Nominal2_Abs
2011-06-20, by Cezary Kaliszyk
More minor TODOs
2011-06-20, by Cezary Kaliszyk
Update TODO
2011-06-20, by Cezary Kaliszyk
Let/minor
2011-06-20, by Cezary Kaliszyk
Update Quotient/TODO and remove some attic code
2011-06-20, by Cezary Kaliszyk
merge
2011-06-19, by Cezary Kaliszyk
little on cps2
2011-06-19, by Cezary Kaliszyk
got rid of the boolean flag in the raw_equivariance function
2011-06-16, by Christian Urban
Fix
2011-06-16, by Cezary Kaliszyk
merge
2011-06-16, by Cezary Kaliszyk
CPS3 can be defined with eqvt_rhs.
2011-06-16, by Cezary Kaliszyk
moved for the moment CPS translations into the example directory
2011-06-16, by Christian Urban
merged
2011-06-16, by Christian Urban
added eqvt_at and invariant for boths sides of the equations
2011-06-16, by Christian Urban
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.
2011-06-16, by Cezary Kaliszyk
added a test that every function must be of pt-sort
2011-06-16, by Christian Urban
all tests work again
2011-06-16, by Christian Urban
added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method
2011-06-15, by Christian Urban
added an abstract
2011-06-15, by Christian Urban
added a stub for function paper; "isabelle make fnpaper"
2011-06-15, by Christian Urban
merge
2011-06-15, by Cezary Kaliszyk
one TODO and one Problem?
2011-06-15, by Cezary Kaliszyk
merge
2011-06-15, by Cezary Kaliszyk
Some TODOs
2011-06-15, by Cezary Kaliszyk
merge
2011-06-15, by Cezary Kaliszyk
TypeSchemes work with 'default'.
2011-06-15, by Cezary Kaliszyk
tuned some proofs
2011-06-14, by Christian Urban
fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough
2011-06-14, by Christian Urban
tuned
2011-06-14, by Christian Urban
Move working examples before non-working ones
2011-06-10, by Cezary Kaliszyk
Optimized proofs and removed some garbage.
2011-06-10, by Cezary Kaliszyk
merge
2011-06-10, by Cezary Kaliszyk
Slightly modify fcb for list1 and put in common place.
2011-06-10, by Cezary Kaliszyk
Experiments with Let
2011-06-10, by Cezary Kaliszyk
Eval can be defined with additional freshness
2011-06-09, by Cezary Kaliszyk
Minor simplification
2011-06-09, by Cezary Kaliszyk
abs_res_fcb will be enough to finish the multiple-recursive proof, if we have a working 'default'.
2011-06-09, by Cezary Kaliszyk
More experiments with 'default'
2011-06-09, by Cezary Kaliszyk
Finished the proof with the invariant
2011-06-08, by Cezary Kaliszyk
Issue with 'default'
2011-06-08, by Cezary Kaliszyk
merged
2011-06-08, by Christian Urban
merged
2011-06-08, by Christian Urban
using the option "default" the function package allows one to give an explicit default value
2011-06-08, by Christian Urban
Simpler proof of TypeSchemes/substs
2011-06-08, by Cezary Kaliszyk
Simplify fcb_res
2011-06-08, by Cezary Kaliszyk
FCB for res binding and simplified proof of subst for type schemes
2011-06-08, by Cezary Kaliszyk
Simplify ln-trans proof
2011-06-08, by Cezary Kaliszyk
cbvs can be easily defined without an invariant
2011-06-08, by Cezary Kaliszyk
defined the "count-bound-variables-occurences" function which has an accumulator like trans
2011-06-07, by Christian Urban
merged
2011-06-07, by Christian Urban
remove garbage (proofs that assumes the invariant outside function)
2011-06-07, by Cezary Kaliszyk
Proof of trans with invariant
2011-06-07, by Cezary Kaliszyk
Testing invariant in Lambda_F_T
2011-06-07, by Cezary Kaliszyk
cleaned ups a bit the examples with the invariant framework; exported nominal_function_config datatype into separate structure and file
2011-06-07, by 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
2011-06-07, by Christian Urban
slightly stronger property in fundef_ex_prop
2011-06-06, by Christian Urban
added an option for an invariant (at the moment only a stub)
2011-06-05, by Christian Urban
added a more general lemma fro fundef_ex1
2011-06-05, by Christian Urban
Trying the induction on the graph
2011-06-04, by Cezary Kaliszyk
Finish and test the locale approach
2011-06-04, by Cezary Kaliszyk
FiniteSupp precondition in the function is enough to get rid of completeness obligationss
2011-06-03, by Cezary Kaliszyk
recursion combinator inside a locale
2011-06-03, by Christian Urban
merge
2011-06-03, by Cezary Kaliszyk
F for lambda used to define translation to locally nameless
2011-06-03, by Cezary Kaliszyk
typo
2011-06-02, by Christian Urban
removed dead code
2011-06-02, by Christian Urban
finished the missing obligations
2011-06-02, by Cezary Kaliszyk
merged
2011-06-02, by Christian Urban
a test with a recursion combinator defined on top of nominal_primrec
2011-06-02, by Christian Urban
Use FCB to simplify proof
2011-06-02, by Cezary Kaliszyk
merge
2011-06-02, by Cezary Kaliszyk
Remove SMT
2011-06-02, by Cezary Kaliszyk
hopefully final fix for ho-functions
2011-06-01, by Christian Urban
first test to fix the problem with free variables
2011-06-01, by Christian Urban
proved subst for All constructor in type schemes.
2011-06-01, by Cezary Kaliszyk
DB translation using index; easier to reason about.
2011-06-01, by Cezary Kaliszyk
Problem: free variables in the goal
2011-06-01, by Cezary Kaliszyk
fixed previous commit
2011-06-01, by Cezary Kaliszyk
equivariance of db_trans
2011-06-01, by Cezary Kaliszyk
fixed the problem with cps-like functions
2011-05-31, by Christian Urban
DeBruijn translation in a simplifier friendly way
2011-05-31, by Cezary Kaliszyk
map_term can be defined when equivariance is assumed
2011-05-31, by Cezary Kaliszyk
map_term is not a function the way it is defined
2011-05-31, by Cezary Kaliszyk
Defined translation from nominal to de-Bruijn; with a freshness condition for the lambda case.
2011-05-31, by Cezary Kaliszyk
Simple eqvt proofs with perm_simps for clarity
2011-05-31, by Cezary Kaliszyk
tuned last commit
2011-05-31, by Christian Urban
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
2011-05-31, by Christian Urban
updated to new Isabelle
2011-05-26, by Christian Urban
added eq_iff and distinct lemmas of nominal datatypes to the simplifier
2011-05-25, by Christian Urban
more on slides
2011-05-24, by Christian Urban
added slides for copenhagen
2011-05-22, by Christian Urban
added a problem with inductive_cases (reported by Randy)
2011-05-14, by Christian Urban
misc
2011-05-13, by Christian Urban
made the subtyping work again
2011-05-10, by Christian Urban
updated to new Isabelle (> 9 May)
2011-05-10, by Christian Urban
merged
2011-05-09, by Christian Urban
added two mutual recursive inductive definitions
2011-05-03, by Christian Urban
deleted two functions from the API
2011-05-03, by Christian Urban
proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
2011-05-03, by Christian Urban
more on pearl-paper
2011-05-09, by Christian Urban
more on pearl-paper
2011-05-04, by Christian Urban
updated Quotient paper so that it compiles again
2011-05-02, by Christian Urban
merged
2011-04-28, by Christian Urban
added slides for beijing
2011-04-28, by Christian Urban
more to the pearl paper
2011-04-22, by Christian Urban
updated to snapshot Isabelle 19 April
2011-04-19, by Christian Urban
merged
2011-04-18, by Christian Urban
added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
2011-04-18, by Christian Urban
New way of forward elimination of Abs1_eq and simplifications of the function obligation proofs.
2011-04-15, by Cezary Kaliszyk
merged
2011-04-13, by Christian Urban
introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
2011-04-13, by Christian Urban
shanghai slides
2011-04-12, by Christian Urban
pictures for slides
2011-04-11, by Christian Urban
Shanghai slides
2011-04-11, by Christian Urban
more paper
2011-04-10, by Christian Urban
eqvt of supp and fresh is proved using equivariance infrastructure
2011-04-10, by Christian Urban
more paper
2011-04-10, by Christian Urban
more on the paper
2011-04-09, by Christian Urban
tuned paper
2011-04-09, by Christian Urban
tuned paper
2011-04-09, by Christian Urban
typo
2011-04-09, by Christian Urban
more on paper
2011-04-08, by Christian Urban
eqvt_lambda without eta-expansion
2011-04-08, by Christian Urban
changed default preprocessor that does not catch variables only occuring on the right
2011-04-06, by Christian Urban
final version of slides
2011-03-31, by Christian Urban
more on the slides
2011-03-30, by Christian Urban
tuned IsaMakefile
2011-03-30, by Christian Urban
rearranged directories and updated to new Isabelle
2011-03-29, by Christian Urban
precise path to LaTeXsugar
2011-03-16, by Christian Urban
a lit bit more on the pearl-jv paper
2011-03-16, by Christian Urban
ported changes from function package....needs Isabelle 16 March or above
2011-03-16, by Christian Urban
more on the pearl paper
2011-03-15, by Christian Urban
equivariance for All and Ex can be proved in terms of their definition
2011-03-14, by Christian Urban
more on the paper
2011-03-11, by Christian Urban
merged
2011-03-08, by Christian Urban
more on the pearl paper
2011-03-08, by Christian Urban
distinct names at toplevel
2011-03-02, by Cezary Kaliszyk
merge
2011-03-02, by Cezary Kaliszyk
Pairing function
2011-03-02, by Cezary Kaliszyk
updated pearl papers
2011-03-02, by Christian Urban
a bit more tuning
2011-03-01, by Christian Urban
included old test cases for perm_simp into ROOT.ML file
2011-02-28, by Christian Urban
split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
2011-02-28, by Christian Urban
some slight polishing
2011-02-25, by Christian Urban
merged
2011-02-24, by Christian Urban
added a lemma about fresh_star and Abs
2011-02-24, by Christian Urban
Reduce the definition of trans to FCB; test that FCB can be proved with simp rules.
2011-02-23, by Cezary Kaliszyk
typeschemes/subst
2011-02-19, by Cezary Kaliszyk
further experiments with typeschemes subst
2011-02-17, by Cezary Kaliszyk
Finished the proof of a function that invents fresh variable names.
2011-02-17, by Cezary Kaliszyk
added eqvt for length
2011-02-16, by Christian Urban
added eqvt lemmas for filter and distinct
2011-02-16, by Christian Urban
added eqvt for cartesian products
2011-02-07, by Christian Urban
cleaned up the experiments so that the tests go through
2011-02-07, by Christian Urban
merge
2011-02-05, by Cezary Kaliszyk
Experiments defining a function on Let
2011-02-05, by Cezary Kaliszyk
updated TODO
2011-02-04, by Christian Urban
Lambda.thy which works with Nominal_Isabelle2011
2011-02-04, by Christian Urban
merged
2011-02-03, by Christian Urban
removed diagnostic code
2011-02-03, by Christian Urban
Only one of the subgoals is needed
2011-02-01, by Cezary Kaliszyk
Experiments with substitution on set+
2011-02-01, by Cezary Kaliszyk
More properties that relate abs_res and abs_set. Also abs_res with less binders.
2011-02-01, by Cezary Kaliszyk
alpha_res implies alpha_set :)
2011-01-30, by Cezary Kaliszyk
Showing that the binders difference is fresh for the left side solves the goal for 'set'.
2011-01-30, by Cezary Kaliszyk
Experiments with functions
2011-01-29, by Cezary Kaliszyk
some experiments
2011-01-27, by Christian Urban
the proofs with eqvt_at
2011-01-27, by Christian Urban
made eqvt-proof explicit in the function definitions
2011-01-25, by Christian Urban
merge
2011-01-25, by Cezary Kaliszyk
minor
2011-01-25, by Cezary Kaliszyk
Down as infixr
2011-01-25, by Cezary Kaliszyk
added some slides
2011-01-22, by Christian Urban
added Tutorial6
2011-01-23, by Christian Urban
cleaning up
2011-01-22, by Christian Urban
merged
2011-01-22, by Christian Urban
cleaned up Tutorial 3 with solutions
2011-01-22, by Christian Urban
Missing val.simps
2011-01-23, by Cezary Kaliszyk
merge
2011-01-23, by Cezary Kaliszyk
Tutorial 4s
2011-01-23, by Cezary Kaliszyk
cleaned up and solution section
2011-01-22, by Christian Urban
cleaned up tutorial1...added solution file
2011-01-22, by Christian Urban
better version of Tutorial 1
2011-01-22, by Christian Urban
better flow of proofs and definitions and proof
2011-01-21, by Christian Urban
separated type preservation and progress into a separate file
2011-01-21, by Christian Urban
substitution lemma in separate file
2011-01-21, by Christian Urban
added unbind example
2011-01-21, by Christian Urban
a bit tuning
2011-01-21, by Christian Urban
first split of tutorrial theory
2011-01-20, by Christian Urban
added a very rough version of the tutorial; all seems to work
2011-01-19, by Christian Urban
added obtain_fresh lemma; tuned Lambda.thy
2011-01-19, by Christian Urban
base file for the tutorial (contains definitions for heigt, subst and beta-reduction)
2011-01-19, by Christian Urban
ported some of the old proofs to serve as testcases
2011-01-19, by Christian Urban
added eqvt and supp lemma for removeAll (function from List.thy)
2011-01-19, by Christian Urban
theory name as it should be
2011-01-19, by Christian Urban
removed diagnostic code
2011-01-19, by Christian Urban
added Minimal file to test things
2011-01-19, by Christian Urban
defined height as a function that returns an integer
2011-01-19, by Christian Urban
deleted diagnostic code
2011-01-18, by Christian Urban
some tryes about substitution over type-schemes
2011-01-18, by Christian Urban
defined properly substitution
2011-01-18, by Christian Urban
derived stronger Abs_eq_iff2 theorems
2011-01-18, by Christian Urban
made alpha_abs_set_stronger1 stronger
2011-01-18, by Christian Urban
removed finiteness assumption from set_rename_perm
2011-01-18, by Christian Urban
alpha_abs_set_stronger1
2011-01-18, by Cezary Kaliszyk
alpha_abs_let_stronger is not true in the same form
2011-01-18, by Cezary Kaliszyk
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
2011-01-18, by Christian Urban
modified the renaming_perm lemmas
2011-01-18, by Christian Urban
added a translation function from lambda-terms to deBruijn terms (equivariance fails at the moment)
2011-01-17, by Christian Urban
added a few examples of functions to Lambda.thy
2011-01-17, by Christian Urban
exported nominal function code to external file
2011-01-17, by Christian Urban
removed old testing code from Lambda.thy
2011-01-17, by Christian Urban
moved high level code from LamTest into the main libraries.
2011-01-17, by Christian Urban
eliminated tracing code; added flag so that equivariance is only proved for the function graph, not the relation
2011-01-17, by Christian Urban
subst also works now
2011-01-15, by Christian Urban
nominal_function works now completely for frees and depth; still a propbelm with subst; no unproved assumptions
2011-01-15, by Christian Urban
strengthened renaming lemmas
2011-01-14, by Christian Urban
added eqvt_lemmas for subset and psubset
2011-01-13, by Christian Urban
a few lemmas about freshness for at and at_base
2011-01-10, by Christian Urban
added a property about finite support in the presense of eqvt_at
2011-01-10, by Christian Urban
instantiated fundef_ex1_eqvt_at theorem with the indction hypothesis
2011-01-09, by Christian Urban
solved subgoals for depth and subst function
2011-01-09, by Christian Urban
added eqvt_at premises in function definition - however not proved at the moment
2011-01-09, by Christian Urban
added one further lemma about equivariance of THE_default
2011-01-07, by Christian Urban
equivariance of THE_default under the uniqueness assumption
2011-01-07, by Christian Urban
derived equivariance for the function graph and function relation
2011-01-07, by Christian Urban
a modified function package where, as a test, True has been injected into the compatibility condictions
2011-01-06, by Christian Urban
removed last traces of debugging code
2011-01-06, by Christian Urban
removed debugging code abd introduced a guarded tracing function
2011-01-06, by Christian Urban
moved Weakening up....it does not compile when put at the last position
2011-01-06, by Christian Urban
tuned
2011-01-06, by Christian Urban
added weakening to the test cases
2011-01-06, by Christian Urban
cleaned up weakening proof and added a version with finit sets
2011-01-06, by Christian Urban
same
2011-01-06, by Christian Urban
some further lemmas for fsets
2011-01-06, by Christian Urban
made sure the raw datatypes and raw functions do not get any mixfix syntax
2011-01-06, by Christian Urban
exported the code into a separate file
2011-01-05, by Christian Urban
strong rule inductions; as an example the weakening lemma works
2011-01-05, by Christian Urban
final version of the ESOP paper; used set+ instead of res as requested by one reviewer
2011-01-04, by Christian Urban
file with most of the strong rule induction development
2011-01-03, by Christian Urban
simple cases for string rule inductions
2011-01-03, by Christian Urban
changed res keyword to set+ for restrictions; comment by a referee
2010-12-31, by Christian Urban
added proper case names for all induct and exhaust theorems
2010-12-31, by Christian Urban
added small example for strong inductions; functions still need a sorry
2010-12-31, by Christian Urban
removed local fix for bug in induction_schema; added setup method for strong inductions
2010-12-30, by Christian Urban
automated all strong induction lemmas
2010-12-28, by Christian Urban
proper application of induction_schema and strong_exhaust rules; needs local fix in induction_schema.ML
2010-12-28, by Christian Urban
generated goals for strong induction theorems.
2010-12-26, by Christian Urban
test with strong inductions
2010-12-23, by Christian Urban
moved all strong_exhaust code to nominal_dt_quot; tuned examples
2010-12-23, by Christian Urban
moved generic functions into nominal_library
2010-12-23, by Christian Urban
slight tuning
2010-12-22, by Christian Urban
slight tuning
2010-12-22, by Christian Urban
tuned examples
2010-12-22, by Christian Urban
added fold_right which produces the correct term for left-infix operators
2010-12-22, by Christian Urban
updated to Isabelle 22 December
2010-12-22, by Christian Urban
a bit tuning
2010-12-22, by Christian Urban
corrected premises of strong exhausts theorems
2010-12-22, by Christian Urban
properly exported strong exhaust theorem; cleaned up some examples
2010-12-22, by Christian Urban
all examples for strong exhausts work; recursive binders need to be treated differently; still unclean version with lots of diagnostic code
2010-12-21, by Christian Urban
one interesting case done
2010-12-19, by Christian Urban
a stronger statement for at_set_avoiding
2010-12-19, by Christian Urban
tuned
2010-12-17, by Christian Urban
tuned
2010-12-17, by Christian Urban
simple cases for strong inducts done; infrastructure for the difficult ones is there
2010-12-16, by Christian Urban
added theorem-rewriter conversion
2010-12-16, by Christian Urban
freshness theorem in strong exhausts; (temporarily includes a cheat_tac to make all tests go through)
2010-12-14, by Christian Urban
created strong_exhausts terms
2010-12-12, by Christian Urban
moved setify and listify functions into the library; introduced versions that have a type argument
2010-12-12, by Christian Urban
updated
2010-12-10, by Christian Urban
a bit more tuning of the paper
2010-12-09, by Christian Urban
brought the paper to 20 pages plus one page appendix
2010-12-09, by Christian Urban
first tests about exhaust
2010-12-08, by Christian Urban
moved some code into the nominal_library
2010-12-08, by Christian Urban
moved definition of raw bn-functions into nominal_dt_rawfuns
2010-12-08, by Christian Urban
kept the nested structure of constructors (belonging to one datatype)
2010-12-08, by Christian Urban
moved general theorems into the libraries
2010-12-07, by Christian Urban
automated permute_bn theorems
2010-12-07, by Christian Urban
updated to changes in Isabelle
2010-12-07, by Christian Urban
deleted nominal_dt_supp.ML
2010-12-06, by Christian Urban
moved code from nominal_dt_supp to nominal_dt_quot
2010-12-06, by Christian Urban
automated alpha_perm_bn theorems
2010-12-06, by Christian Urban
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
2010-12-06, by Christian Urban
updated to Isabelle 2nd December
2010-12-03, by Christian Urban
isarfied some of the high-level proofs
2010-11-29, by Christian Urban
added abs_rename_res lemma
2010-11-29, by Christian Urban
completed proofs in Foo2
2010-11-29, by Christian Urban
completed the strong exhausts rules for Foo2 using general lemmas
2010-11-28, by Christian Urban
tuned proof to reduce number of warnings
2010-11-27, by Christian Urban
disabled the Foo examples, because of heavy work
2010-11-27, by Christian Urban
slightly simplified the Foo2 tests and hint at a general lemma
2010-11-26, by Christian Urban
completely different method fro deriving the exhaust lemma
2010-11-26, by Christian Urban
merged
2010-11-26, by Christian Urban
merged
2010-11-25, by Christian Urban
added example from the F-ing paper by Rossberg, Russo and Dreyer
2010-11-24, by Christian Urban
implemented concrete suggestion of 3rd reviewer
2010-11-24, by Christian Urban
missing freshness assumptions
2010-11-26, by Cezary Kaliszyk
foo2 strong induction
2010-11-25, by Cezary Kaliszyk
foo2 full exhausts
2010-11-24, by Cezary Kaliszyk
Foo2 strong_exhaust for first variable.
2010-11-24, by Cezary Kaliszyk
single rename in let2
2010-11-22, by Cezary Kaliszyk
current isabelle
2010-11-22, by Cezary Kaliszyk
added example Foo2.thy
2010-11-21, by Christian Urban
tuned example
2010-11-15, by Christian Urban
proved that bn functions return a finite set
2010-11-15, by Christian Urban
added a test for the various shallow binders
2010-11-15, by Christian Urban
fixed bug in fv function where a shallow binder binds lists of names
2010-11-15, by Christian Urban
merged Nominal-General directory into Nominal; renamed Abs.thy to Nominal2_Abs.thy
2010-11-14, by Christian Urban
deleted special Nominal2_FSet theory
2010-11-14, by Christian Urban
moved rest of the lemmas from Nominal2_FSet to the TypeScheme example
2010-11-14, by Christian Urban
moved most material fron Nominal2_FSet into the Nominal_Base theory
2010-11-14, by Christian Urban
tuned example
2010-11-14, by Christian Urban
lifted permute_bn simp rules
2010-11-14, by Christian Urban
lifted permute_bn constants
2010-11-13, by Christian Urban
respectfulness for permute_bn functions
2010-11-13, by Christian Urban
automated permute_bn functions (raw ones first)
2010-11-12, by Christian Urban
adapted to changes by Florian on the quotient package and removed local fix for function package
2010-11-10, by Christian Urban
expanded the paper by uncommenting the comments and adding the appendix
2010-11-10, by Christian Urban
fixed locally the problem with the function package; all tests work again
2010-11-07, by Christian Urban
added a test about subtyping; disabled two tests, because of problem with function package
2010-11-06, by Christian Urban
small typo
2010-11-05, by Christian Urban
squeezed qpaper to 6 pages
2010-10-29, by Christian Urban
Qpaper / Move examples to commented out appendix
2010-10-29, by Cezary Kaliszyk
Unanonymize qpaper
2010-10-28, by Cezary Kaliszyk
FSet changes for Qpaper
2010-10-28, by Cezary Kaliszyk
Remove FSet and use the one from Isabelle
2010-10-28, by Cezary Kaliszyk
took out comment about map-types / adapted to recent changes
2010-10-19, by Christian Urban
use definitions instead of functions
2010-10-19, by Christian Urban
tuned
2010-10-18, by Christian Urban
used functions instead of definitions
2010-10-18, by Christian Urban
added missing style file
2010-10-18, by Christian Urban
Use the generalized compositional quotient theorem
2010-10-18, by Cezary Kaliszyk
fixed typo
2010-10-17, by Christian Urban
all tests work again
2010-10-17, by Christian Urban
some tuning
2010-10-17, by Christian Urban
naming scheme is now *_fset (not f*_)
2010-10-17, by Christian Urban
more cleaning
2010-10-15, by Christian Urban
further tuning
2010-10-15, by Christian Urban
renamed fminus_raw to diff_list
2010-10-15, by Christian Urban
renamed fcard_raw to card_list
2010-10-15, by Christian Urban
slight update
2010-10-15, by Christian Urban
Further reorganisation and cleaning
2010-10-15, by Christian Urban
further cleaning
2010-10-15, by Christian Urban
typo
2010-10-15, by Christian Urban
FSet: stronger fact in Isabelle.
2010-10-15, by Cezary Kaliszyk
FSet synchronizing
2010-10-15, by Cezary Kaliszyk
Synchronizing FSet further.
2010-10-15, by Cezary Kaliszyk
Partially merging changes from Isabelle
2010-10-15, by Cezary Kaliszyk
fixed the typo in the abstract and the problem with append (the type of map_k
2010-10-14, by Christian Urban
changed format of the pearl paper
2010-10-14, by Christian Urban
deleted some unused lemmas
2010-10-14, by Christian Urban
major reorganisation of fset (renamed fset_to_set to fset, changed the definition of list_eq and fcard_raw)
2010-10-14, by Christian Urban
more on the pearl paper
2010-10-13, by Christian Urban
added a section about abstractions
2010-10-12, by Christian Urban
tiny work on the pearl paper
2010-10-12, by Christian Urban
tuned
2010-10-08, by Christian Urban
added apendix to paper detailing one proof
2010-10-08, by Christian Urban
minor
2010-10-08, by Christian Urban
minor
2010-10-08, by Christian Urban
down to 20 pages
2010-10-08, by Christian Urban
minor
2010-10-07, by Cezary Kaliszyk
down to 21 pages and changed strong induction section
2010-10-06, by Christian Urban
tuned
2010-10-06, by Christian Urban
down to 22 pages
2010-10-06, by Christian Urban
down to 23 pages
2010-10-05, by Christian Urban
down to 24 pages and a bit
2010-10-05, by Christian Urban
llncs and more sqeezing
2010-10-05, by Christian Urban
first part of sqeezing everything into 20 pages (at the moment we have 26)
2010-10-04, by Christian Urban
changed to llncs
2010-10-04, by Christian Urban
merged
2010-10-01, by Christian Urban
minor experiments
2010-10-01, by Christian Urban
merged
2010-09-30, by Christian Urban
simplified exhaust proofs
2010-09-29, by Christian Urban
Made the paper to compile with the renamings.
2010-10-01, by Cezary Kaliszyk
merged
2010-09-29, by Christian Urban
worked example Foo1 with induct_schema
2010-09-29, by Christian Urban
merged
2010-09-29, by Christian Urban
use also induct_schema for the Let-example (permute_bn is used)
2010-09-29, by Christian Urban
test with induct_schema for simpler strong_ind proofs
2010-09-29, by Christian Urban
substitution definition with 'next_name'.
2010-09-29, by Cezary Kaliszyk
merged
2010-09-28, by Christian Urban
added Foo1 to explore a contrived example
2010-09-28, by Christian Urban
added postprocessed fresh-lemmas for constructors
2010-09-27, by Christian Urban
post-processed eq_iff and supp threormes according to the fv-supp equality
2010-09-27, by Christian Urban
more consistent naming in Abs.thy
2010-09-27, by Christian Urban
some experiments
2010-09-27, by Christian Urban
added simp rules for prod_fv and prod_alpha
2010-09-27, by Christian Urban
a few more words about Ott
2010-09-26, by Christian Urban
lifted size_thms and exported them as <name>.size
2010-09-25, by Christian Urban
cleaned up two examples
2010-09-25, by Christian Urban
added example about datatypes
2010-09-25, by Christian Urban
updated to Isabelle 22 Sept
2010-09-23, by Christian Urban
removed dead code
2010-09-22, by Christian Urban
fixed
2010-09-22, by Christian Urban
made supp proofs more robust by not using the standard induction; renamed some example files
2010-09-22, by Christian Urban
introduced a general procedure for structural inductions; simplified reflexivity proof
2010-09-20, by Christian Urban
updated to Isabelle Sept 16
2010-09-18, by Christian Urban
updated to Isabelle Sept 13
2010-09-18, by Christian Urban
tuned code
2010-09-12, by Christian Urban
tuned (to conform with indentation policy of Markus)
2010-09-11, by Christian Urban
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
2010-09-10, by Christian Urban
generated inducts rule by Project_Rule.projections
2010-09-05, by Christian Urban
added the definition supp_rel (support w.r.t. a relation)
2010-09-05, by Christian Urban
merged
2010-09-04, by Christian Urban
got rid of Nominal2_Supp (is now in Nomina2_Base)
2010-09-04, by Christian Urban
moved everything out of Nominal_Supp
2010-09-04, by Christian Urban
renamed alpha_gen -> alpha_set and Abs -> Abs_set etc
2010-09-04, by Christian Urban
moved a proof to Abs
2010-09-04, by Christian Urban
got rid of Nominal_Atoms (folded into Nominal2_Base)
2010-09-04, by Christian Urban
cleaned a bit various thy-files in Nominal-General
2010-09-04, by Christian Urban
adapted paper to changes
2010-09-03, by Christian Urban
made the fv-definition aggree more with alpha (needed in the support proofs)
2010-09-03, by Christian Urban
removed lemma finite_set (already in simpset)
2010-09-03, by Christian Urban
added supp_set lemma
2010-09-03, by Christian Urban
some experiments with support
2010-09-02, by Christian Urban
added eqvt-attribute for permute_abs lemmas
2010-09-02, by Christian Urban
slides of my talk
2010-08-31, by Christian Urban
merge
2010-08-30, by Cezary Kaliszyk
update qpaper to new isabelle
2010-08-30, by Cezary Kaliszyk
No need to unfold mem_def with rsp/prs (requires new isabelle).
2010-08-30, by Cezary Kaliszyk
Anonymize, change Quotient to Quot and fix indentation
2010-08-30, by Cezary Kaliszyk
renamed NewParser to Nominal2
2010-08-29, by Christian Urban
tuned
2010-08-29, by Christian Urban
updated todos
2010-08-29, by Christian Urban
added fs-instance proofs
2010-08-29, by Christian Urban
added proofs for fsupp properties
2010-08-29, by Christian Urban
fiexed problem with constructors that have no arguments
2010-08-29, by Christian Urban
proved supports lemmas
2010-08-29, by Christian Urban
slight cleaning
2010-08-28, by Christian Urban
updated to new Isabelle
2010-08-28, by Christian Urban
cut out most of the lifting section and cleaned up everything
2010-08-27, by Christian Urban
made all typographic changes
2010-08-27, by Christian Urban
first pass on section 1
2010-08-27, by Christian Urban
make copies of the "old" files
2010-08-27, by Christian Urban
Ball Bex can be lifted after unfolding.
2010-08-27, by Cezary Kaliszyk
"isabelle make test" makes all major examples....they work up to supp theorems (excluding)
2010-08-27, by Christian Urban
merged
2010-08-27, by Christian Urban
corrected bug with fv-function generation (that was the problem with recursive binders)
2010-08-27, by Christian Urban
minor
2010-08-26, by Cezary Kaliszyk
cleaned up (almost completely) the examples
2010-08-26, by Christian Urban
cleaning of unused files and code
2010-08-25, by Christian Urban
automatic lifting
2010-08-25, by Christian Urban
everything now lifts as expected
2010-08-25, by Christian Urban
now every lemma lifts (even with type variables)
2010-08-25, by Christian Urban
can now deal with type variables in nominal datatype definitions
2010-08-25, by Christian Urban
updated to new Isabelle
2010-08-22, by Christian Urban
merged
2010-08-22, by Christian Urban
updated to new Isabelle
2010-08-22, by Christian Urban
not needed anymore
2010-08-21, by Christian Urban
moved lifting code from Lift.thy to nominal_dt_quot.ML
2010-08-21, by Christian Urban
nominal_datatypes with type variables do not work
2010-08-21, by 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
2010-08-21, by Christian Urban
Clarifications to FIXMEs.
2010-08-20, by Cezary Kaliszyk
Finished adding remarks from the reviewers.
2010-08-20, by Cezary Kaliszyk
few remaining remarks as fixme's.
2010-08-20, by Cezary Kaliszyk
used @{const_name} hopefully everywhere
2010-08-19, by Christian Urban
Intuition behind REL
2010-08-19, by Cezary Kaliszyk
add missing mathpartir
2010-08-19, by Cezary Kaliszyk
Add 2 FIXMEs
2010-08-19, by Cezary Kaliszyk
The type does determine respectfulness, the constant without an instantiated type does not.
2010-08-19, by Cezary Kaliszyk
Add the SAC stylesheet and updated root file.
2010-08-19, by Cezary Kaliszyk
TODO
2010-08-19, by Cezary Kaliszyk
further comments from the referees
2010-08-19, by Cezary Kaliszyk
fixes for referees
2010-08-19, by Cezary Kaliszyk
put everything in a "timeit"
2010-08-18, by Christian Urban
improved runtime slightly, by constructing an explicit size measure for the function definitions
2010-08-18, by Christian Urban
more tuning of the code
2010-08-17, by Christian Urban
deleted unused code
2010-08-17, by Christian Urban
improved code
2010-08-17, by Christian Urban
can also lift the various eqvt lemmas for bn, fv, fv_bn and size
2010-08-17, by Christian Urban
also able to lift the bn_defs
2010-08-17, by Christian Urban
added rsp-lemmas for alpha_bns
2010-08-17, by Christian Urban
cezary made the eq_iff lemmas to lift (still needs some infrastructure in quotient)
2010-08-16, by Christian Urban
pinpointed the problem
2010-08-16, by Christian Urban
modified the code for class instantiations (with help from Florian)
2010-08-16, by Christian Urban
defined qperms and qsizes
2010-08-15, by Christian Urban
simplified code
2010-08-15, by Christian Urban
improved code
2010-08-14, by Christian Urban
more experiments with lifting
2010-08-14, by Christian Urban
updated to Isabelle 12th Aug
2010-08-12, by Christian Urban
rsp for constructors
2010-08-11, by Christian Urban
updated to Isabelle 11 Aug
2010-08-11, by Christian Urban
added a function that transforms the helper-rsp lemmas into real rsp lemmas
2010-08-11, by Christian Urban
proved rsp-helper lemmas of size functions
2010-08-08, by Christian Urban
tuning
2010-07-31, by Christian Urban
further simplification with alpha_prove
2010-07-31, by Christian Urban
introduced a general alpha_prove method
2010-07-31, by Christian Urban
equivariance for size
2010-07-30, by Christian Urban
helper lemmas for rsp-lemmas
2010-07-29, by Christian Urban
tests
2010-07-27, by Christian Urban
cleaned up a bit Abs.thy
2010-07-27, by Christian Urban
fixed order of fold_union to make alpha and fv agree
2010-07-27, by Christian Urban
small cleaning
2010-07-26, by Christian Urban
added paper by james; some minor cleaning
2010-07-25, by Christian Urban
samll changes
2010-07-23, by Christian Urban
made compatible
2010-07-23, by Christian Urban
added
2010-07-23, by Christian Urban
updated to new Isabelle; made FSet more "quiet"
2010-07-22, by Christian Urban
merged
2010-07-20, by Christian Urban
minor
2010-07-19, by Christian Urban
minor polishing
2010-07-19, by Christian Urban
quote for a new paper
2010-07-19, by Christian Urban
corrected lambda-preservation theorem
2010-07-19, by Christian Urban
minor
2010-07-19, by Christian Urban
minor things on the paper
2010-07-18, by Christian Urban
merged
2010-07-18, by Christian Urban
minor things
2010-07-18, by Christian Urban
some test with quotient
2010-07-18, by Christian Urban
some minor changes
2010-07-17, by Christian Urban
changes suggested by Peter Homeier
2010-07-17, by Christian Urban
tests
2010-07-17, by Christian Urban
submitted version
2010-07-16, by Christian Urban
more paper
2010-07-16, by Christian Urban
more on the paper
2010-07-16, by Christian Urban
more on the paper
2010-07-16, by Christian Urban
a bit more to the paper
2010-07-15, by Christian Urban
more on the paper
2010-07-14, by Christian Urban
more on slides
2010-07-13, by Christian Urban
slides
2010-07-13, by Christian Urban
more on slides
2010-07-12, by Christian Urban
slides
2010-07-11, by Christian Urban
slides
2010-07-11, by Christian Urban
more on slides
2010-07-10, by Christian Urban
more on slides
2010-07-10, by Christian Urban
added material for slides
2010-07-10, by Christian Urban
fixed
2010-07-09, by Christian Urban
before examples
2010-07-09, by Christian Urban
finished alpha-section
2010-07-09, by Christian Urban
more on the paper
2010-07-07, by Christian Urban
more on the paper
2010-07-07, by Christian Urban
more on the paper
2010-07-02, by Christian Urban
finished fv-section
2010-07-02, by Christian Urban
more on the paper
2010-07-01, by Christian Urban
spell check
2010-07-01, by Christian Urban
more work on the paper
2010-06-30, by Christian Urban
removed an "eqvt"-warning
2010-06-29, by Christian Urban
more quotient-definitions
2010-06-28, by Christian Urban
slight cleaning
2010-06-28, by Christian Urban
fixed according to changes in quotient
2010-06-27, by Christian Urban
added definition of the quotient types
2010-06-24, by Christian Urban
fixed according to changes in quotient
2010-06-24, by Christian Urban
added comment about partial equivalence relations
2010-06-24, by Christian Urban
even further polishing of the qpaper
2010-06-24, by Christian Urban
polished paper again (and took out some claims about Homeier's package)
2010-06-23, by Christian Urban
some slight polishing on the paper
2010-06-23, by Christian Urban
merged cezary's changes
2010-06-23, by Christian Urban
whitespace
2010-06-23, by Christian Urban
Un-do the second change to SingleLet.
2010-06-23, by Cezary Kaliszyk
merge
2010-06-23, by Cezary Kaliszyk
Changes for PER and list_all2 committed to Isabelle
2010-06-23, by Cezary Kaliszyk
changes for partial-equivalence quotient package
2010-06-18, by Cezary Kaliszyk
deleted compose-lemmas in Abs (not needed anymore)
2010-06-23, by Christian Urban
deleted equivp_hack
2010-06-23, by Christian Urban
proved eqvip theorems for alphas
2010-06-22, by Christian Urban
cleaned up the FSet (noise was introduced by error)
2010-06-22, by Christian Urban
prove that alpha implies alpha_bn (needed for rsp proofs)
2010-06-22, by Christian Urban
further post-submission tuning
2010-06-21, by Christian Urban
merged with main line
2010-06-21, by Christian Urban
merged
2010-06-21, by Christian Urban
also symmetry
2010-06-11, by Christian Urban
merged
2010-06-10, by Christian Urban
premerge
2010-06-10, by Christian Urban
transitivity proofs done
2010-06-09, by Christian Urban
merged
2010-06-07, by Christian Urban
work on transitivity proof
2010-06-07, by Christian Urban
added uminus_eqvt
2010-06-03, by Christian Urban
fixed problem with eqvt proofs
2010-06-03, by Christian Urban
fixed problem with bn_info
2010-06-02, by Christian Urban
merged
2010-06-01, by Christian Urban
equivariance done
2010-06-01, by Christian Urban
smaller code for raw-eqvt proofs
2010-06-01, by Christian Urban
all raw definitions are defined using function
2010-05-31, by Christian Urban
merged
2010-05-27, by Christian Urban
intermediate state
2010-05-27, by Christian Urban
merged
2010-05-26, by Christian Urban
added FSet to the correct paper
2010-05-26, by Christian Urban
added slides
2010-05-25, by Christian Urban
tuned
2010-05-24, by Christian Urban
tuned
2010-05-24, by Christian Urban
alpha works now
2010-05-24, by Christian Urban
started to work on alpha
2010-05-23, by Christian Urban
properly exported bn_descr
2010-05-22, by Christian Urban
hving a working fv-definition without the export
2010-05-21, by Christian Urban
tuned
2010-05-21, by Christian Urban
proper parser for "exclude:"
2010-05-21, by Christian Urban
tuned
2010-05-20, by Christian Urban
moved some mk_union and mk_diff into the library
2010-05-20, by Christian Urban
new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
2010-05-20, by Christian Urban
some post-submission polishing
2010-06-21, by Christian Urban
added a few points that need to be looked at the next version of the qpaper
2010-06-21, by Christian Urban
eliminated a quot_thm flag
2010-06-21, by Christian Urban
fixed example
2010-06-20, by Christian Urban
small addition to the acknowledgement
2010-06-20, by Christian Urban
qpaper / address FIXMEs.
2010-06-17, by Cezary Kaliszyk
forgot to save
2010-06-17, by Cezary Kaliszyk
Fix regularization. Two "FIXME" left in introduction. Minor spellings.
2010-06-17, by Cezary Kaliszyk
polished everything and submitted
2010-06-17, by Christian Urban
conclusion done
2010-06-16, by Christian Urban
Answer questions in comments
2010-06-16, by Cezary Kaliszyk
tuned
2010-06-16, by Christian Urban
finished section 4, but put some things I do not understand on comment
2010-06-16, by Christian Urban
4 almost finished
2010-06-16, by Christian Urban
cleaned up definitions
2010-06-15, by Christian Urban
merge
2010-06-15, by Cezary Kaliszyk
qpaper/Rewrite section5
2010-06-15, by Cezary Kaliszyk
merged
2010-06-15, by Christian Urban
tuned everytinh up to section 4
2010-06-15, by Christian Urban
Definition of Respects.
2010-06-15, by Cezary Kaliszyk
conclusion
2010-06-15, by Cezary Kaliszyk
Qpaper / Clarify the typing system and composition of quotients issue.
2010-06-15, by Cezary Kaliszyk
Remove only reference to 'equivp'.
2010-06-15, by Cezary Kaliszyk
merge
2010-06-15, by Cezary Kaliszyk
qpaper/ackno
2010-06-15, by Cezary Kaliszyk
tuned
2010-06-15, by Christian Urban
qpaper
2010-06-15, by Cezary Kaliszyk
qpaper / hol4
2010-06-15, by Cezary Kaliszyk
qpaper/related work
2010-06-15, by Cezary Kaliszyk
finished preliminary section
2010-06-15, by Christian Urban
typo
2010-06-14, by Christian Urban
some slight tuning of the preliminary section
2010-06-14, by Christian Urban
merge
2010-06-14, by Cezary Kaliszyk
qpaper
2010-06-14, by Cezary Kaliszyk
merged
2010-06-14, by Christian Urban
tuned
2010-06-14, by Christian Urban
Qpaper / beginnig of sec5
2010-06-14, by Cezary Kaliszyk
merge
2010-06-14, by Cezary Kaliszyk
qpaper/unfold the ball_reg_right statement
2010-06-14, by Cezary Kaliszyk
merged
2010-06-14, by Christian Urban
some tuning and start work on section 4
2010-06-14, by Christian Urban
qpaper
2010-06-14, by Cezary Kaliszyk
qpaper / INJ
2010-06-14, by Cezary Kaliszyk
qpaper / REG
2010-06-14, by Cezary Kaliszyk
qpaper / minor
2010-06-14, by Cezary Kaliszyk
qpaper/various
2010-06-14, by Cezary Kaliszyk
qpaper
2010-06-14, by Cezary Kaliszyk
qpaper/more on example
2010-06-14, by Cezary Kaliszyk
qpaper/examples
2010-06-14, by Cezary Kaliszyk
completed proof and started section about respectfulness and preservation
2010-06-14, by Christian Urban
more on the qpaper
2010-06-13, by Christian Urban
tuned
2010-06-13, by Christian Urban
more on the constant lifting section
2010-06-13, by Christian Urban
something about the quotient ype definitions
2010-06-13, by Christian Urban
added some examples
2010-06-13, by Christian Urban
improved definition of ABS and REP
2010-06-13, by Christian Urban
qpaper.
2010-06-13, by Cezary Kaliszyk
some spelling
2010-06-13, by Cezary Kaliszyk
minor
2010-06-13, by Cezary Kaliszyk
qpaper / tuning in preservation and general display
2010-06-13, by Cezary Kaliszyk
polishing of ABS/REP
2010-06-13, by Christian Urban
some slight tuning of the intro
2010-06-12, by Christian Urban
Fix integer relation.
2010-06-12, by Cezary Kaliszyk
completed the intro (except minor things)
2010-06-12, by Christian Urban
more intro
2010-06-11, by Christian Urban
more on the qpaper
2010-06-11, by Christian Urban
even more on the qpaper (intro almost done)
2010-06-11, by Christian Urban
more to the introduction of the qpaper
2010-06-11, by Christian Urban
adapted to the official sigplan style file (this gives us more space)
2010-06-10, by Christian Urban
added to the popl-paper a pointer to work by Altenkirch
2010-06-10, by Christian Urban
more on the qpaper
2010-06-10, by Christian Urban
new title for POPL paper
2010-06-07, by Christian Urban
more work on intro and abstract (done for today)
2010-06-07, by Christian Urban
a bit more in the introduction and abstract
2010-06-07, by Christian Urban
improved abstract, some tuning
2010-06-07, by Christian Urban
Qpaper / minor on cleaning
2010-06-06, by Cezary Kaliszyk
qpaper / injection proof.
2010-06-05, by Cezary Kaliszyk
qpaper / example interaction
2010-06-05, by Cezary Kaliszyk
Qpaper/regularization proof.
2010-06-05, by Cezary Kaliszyk
qpaper
2010-06-05, by Cezary Kaliszyk
Qpaper/more.
2010-06-02, by Cezary Kaliszyk
Qpaper/Minor
2010-06-02, by Cezary Kaliszyk
added larry's quote
2010-06-01, by Christian Urban
added larry's paper
2010-06-01, by Christian Urban
tuned
2010-06-01, by Christian Urban
first version of the abstract
2010-05-29, by Christian Urban
merged
2010-05-27, by Christian Urban
fixed bug where perm_simp 'forgets' how to prove equivariance for the empty set
2010-05-27, by Christian Urban
qpaper / lemmas used in proofs
2010-05-27, by Cezary Kaliszyk
qpaper / injection statement
2010-05-27, by Cezary Kaliszyk
qpaper / regularize
2010-05-27, by Cezary Kaliszyk
qpaper / a bit about prs
2010-05-27, by Cezary Kaliszyk
Functionalized the ABS/REP definition.
2010-05-27, by Cezary Kaliszyk
qpaper / lifting introduction
2010-05-26, by Cezary Kaliszyk
merged
2010-05-26, by Cezary Kaliszyk
fixed compile error
2010-05-26, by Christian Urban
qpaper / composition of quotients.
2010-05-26, by Cezary Kaliszyk
qpaper
2010-05-26, by Cezary Kaliszyk
qpaper..
2010-05-26, by Cezary Kaliszyk
qpaper.
2010-05-26, by Cezary Kaliszyk
Name some respectfullness
2010-05-26, by Cezary Kaliszyk
added FSet to the correct paper
2010-05-26, by Christian Urban
merged
2010-05-26, by Christian Urban
added FSet
2010-05-26, by Christian Urban
qpaper
2010-05-26, by Cezary Kaliszyk
qpaper
2010-05-26, by Cezary Kaliszyk
Substitution Lemma for TypeSchemes.
2010-05-25, by Cezary Kaliszyk
Simplified the proof
2010-05-25, by Cezary Kaliszyk
A lemma about substitution in TypeSchemes.
2010-05-25, by Cezary Kaliszyk
reversing the direction of fresh_star
2010-05-25, by Cezary Kaliszyk
overlapping deep binders proof
2010-05-25, by Cezary Kaliszyk
edits from the reviewers
2010-05-25, by Christian Urban
tuned paper
2010-05-24, by Christian Urban
changed qpaper to lncs-style
2010-05-23, by Christian Urban
Match_Lam defined on Quotient Level.
2010-05-21, by Cezary Kaliszyk
More on Function-defined subst.
2010-05-21, by Cezary Kaliszyk
Isabelle renamings
2010-05-21, by Cezary Kaliszyk
merge
2010-05-21, by Cezary Kaliszyk
Renamings.
2010-05-21, by Cezary Kaliszyk
Renamings
2010-05-21, by Cezary Kaliszyk
merge (non-trival)
2010-05-21, by Cezary Kaliszyk
Previously uncommited direct subst definition changes.
2010-05-21, by Cezary Kaliszyk
Function experiments
2010-05-21, by Cezary Kaliszyk
merged
2010-05-19, by Christian Urban
added comments about pottiers work
2010-05-19, by Christian Urban
more subst experiments
2010-05-19, by Cezary Kaliszyk
More subst experminets
2010-05-19, by Cezary Kaliszyk
more on subst
2010-05-18, by Cezary Kaliszyk
Single variable substitution
2010-05-18, by Cezary Kaliszyk
subst fix
2010-05-18, by Cezary Kaliszyk
subst experiments
2010-05-18, by Cezary Kaliszyk
soem minor tuning
2010-05-18, by Christian Urban
Fix broken add
2010-05-18, by Cezary Kaliszyk
add missing .bib
2010-05-18, by Cezary Kaliszyk
merge
2010-05-18, by Cezary Kaliszyk
starting bibliography
2010-05-18, by Cezary Kaliszyk
merged
2010-05-17, by Christian Urban
updated to new Isabelle (More_Conv -> Conv)
2010-05-17, by Christian Urban
made this example to work again
2010-05-17, by Christian Urban
merge
2010-05-17, by Cezary Kaliszyk
alpha_alphabn for bindings in a type under bn.
2010-05-17, by Cezary Kaliszyk
minor tuning
2010-05-17, by Christian Urban
Ex4 does work, and I don't see the difference between the alphas.
2010-05-17, by Cezary Kaliszyk
slight tuning
2010-05-17, by Christian Urban
somewhat simplified the main parsing function; failed to move a Note-statement to define_raw_perms
2010-05-17, by 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
2010-05-16, by Christian Urban
tuned paper
2010-05-16, by Christian Urban
tuned paper
2010-05-15, by Christian Urban
tuned a bit the paper
2010-05-14, by Christian Urban
started a new file for the parser to make some experiments
2010-05-14, by Christian Urban
moved old parser and fv into attic
2010-05-14, by Christian Urban
polished example
2010-05-14, by Christian Urban
merged
2010-05-14, by Christian Urban
tuned a bit the paper
2010-05-14, by Christian Urban
Proper fv/alpha for multiple compound binders
2010-05-14, by Cezary Kaliszyk
SingleLetFoo with everything.
2010-05-14, by Cezary Kaliszyk
Fv for multiple binding functions
2010-05-14, by Cezary Kaliszyk
added a more instructive example - has some problems with fv though
2010-05-13, by Christian Urban
added flip_eqvt and swap_eqvt to the equivariance lists
2010-05-13, by Christian Urban
tuned the paper
2010-05-13, by Christian Urban
properly declared outer keyword
2010-05-13, by Christian Urban
added an example which goes outside our current speciifcation
2010-05-13, by Christian Urban
made out of STEPS a configuration value so that it can be set individually in each file
2010-05-13, by Christian Urban
tuned eqvt-proofs about prod_rel and prod_fv
2010-05-13, by Christian Urban
removed internal functions from the signature (they are not needed anymore)
2010-05-13, by Christian Urban
added term4 back to the examples
2010-05-13, by Christian Urban
Make Term4 use 'equivariance'.
2010-05-13, by Cezary Kaliszyk
fixed the examples for the new eqvt-procedure....temporarily disabled Manual/Term4.thy
2010-05-12, by Christian Urban
merged
2010-05-12, by Christian Urban
moved the data-transformation into the parser
2010-05-12, by Christian Urban
added a test whether some of the constants already equivariant (then the procedure has to fail).
2010-05-12, by Christian Urban
include set_simps and append_simps in fv_rsp
2010-05-12, by Cezary Kaliszyk
Move alpha_eqvt to unused.
2010-05-12, by Cezary Kaliszyk
Use equivariance instead of alpha_eqvt
2010-05-12, by Cezary Kaliszyk
merge
2010-05-12, by Cezary Kaliszyk
merge
2010-05-12, by Cezary Kaliszyk
fvbv_rsp include prod_rel.simps
2010-05-12, by Cezary Kaliszyk
better ML-interface (returning only a list of theorems and a context)
2010-05-12, by Christian Urban
merge
2010-05-12, by Cezary Kaliszyk
Use raw_induct instead of induct
2010-05-12, by Cezary Kaliszyk
ingnored parameters in equivariance; added a proper interface to be called from ML
2010-05-12, by Christian Urban
properly exported defined bn-functions
2010-05-12, by Christian Urban
Include raw permutation definitions in eqvt
2010-05-11, by Cezary Kaliszyk
Declare alpha_gen_eqvt as eqvt and change the proofs that used 'eqvts[symmetric]'
2010-05-11, by Cezary Kaliszyk
a bit for the introduction of the q-paper
2010-05-11, by Christian Urban
added some of the quotient literature; a bit more to the qpaper
2010-05-11, by Christian Urban
fixed a problem with non-existant alphas2
2010-05-10, by Christian Urban
added comment about bind_set
2010-05-10, by Christian Urban
fixing bind_set problem
2010-05-10, by Christian Urban
merge
2010-05-10, by Cezary Kaliszyk
Term8 comment
2010-05-10, by Cezary Kaliszyk
merge
2010-05-10, by Cezary Kaliszyk
Restore set bindings in CoreHaskell
2010-05-10, by Cezary Kaliszyk
Recursive examples with relation composition
2010-05-10, by Cezary Kaliszyk
merge
2010-05-10, by Cezary Kaliszyk
prod_rel and prod_fv eqvt and mono
2010-05-10, by Cezary Kaliszyk
ExLetRec
2010-05-10, by Cezary Kaliszyk
merge
2010-05-10, by Cezary Kaliszyk
Parser changes for compound relations
2010-05-10, by Cezary Kaliszyk
merge
2010-05-10, by Cezary Kaliszyk
Use mk_compound_fv' and mk_compound_rel'
2010-05-10, by Cezary Kaliszyk
merge
2010-05-10, by Cezary Kaliszyk
Membership in a pair of lists.
2010-05-10, by Cezary Kaliszyk
Synchronize FSet with repository
2010-05-10, by Cezary Kaliszyk
tuned file names for examples
2010-05-09, by Christian Urban
cleaned up a bit the examples; added equivariance to all examples
2010-05-09, by Christian Urban
fixed the problem with alpha containing splits
2010-05-09, by 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
2010-05-09, by Christian Urban
Manually added some newer keywords from the distribution
2010-05-07, by Cezary Kaliszyk
Regularize experiments
2010-05-07, by Cezary Kaliszyk
alpha_eqvt_tac with prod_rel and prod_fv simps
2010-05-06, by Cezary Kaliszyk
mem => member
2010-05-06, by Cezary Kaliszyk
merge
2010-05-06, by Cezary Kaliszyk
Fixes for new Isabelle
2010-05-06, by Cezary Kaliszyk
compound versions with prod_rel and prod_fun, not made default yet.
2010-05-06, by Cezary Kaliszyk
prod_rel and prod_fv simps
2010-05-06, by Cezary Kaliszyk
mem => member
2010-05-06, by Cezary Kaliszyk
prod_rel.simps and Fixed for new isabelle
2010-05-06, by Cezary Kaliszyk
Fixes for new isabelle
2010-05-06, by Cezary Kaliszyk
prod_fv and its respectfullness and preservation.
2010-05-06, by Cezary Kaliszyk
Experiments with equivariance.
2010-05-06, by Cezary Kaliszyk
merged
2010-05-05, by Christian Urban
a bit mor on the pearl journal paper
2010-05-05, by Christian Urban
solved the problem with equivariance by first eta-normalising the goal
2010-05-05, by Christian Urban
Some cleaning in Term4
2010-05-05, by Cezary Kaliszyk
"isabelle make" compiles all examples with newparser/newfv/newalpha only.
2010-05-04, by Cezary Kaliszyk
Move Term4 to NewParser
2010-05-04, by Cezary Kaliszyk
Fix Term4 for permutation signature change
2010-05-04, by Cezary Kaliszyk
Move LF to NewParser. Just works.
2010-05-04, by Cezary Kaliszyk
merge
2010-05-04, by Cezary Kaliszyk
ExLetMult
2010-05-04, by Cezary Kaliszyk
Ex1Rec.
2010-05-04, by Cezary Kaliszyk
merge
2010-05-04, by Cezary Kaliszyk
merge
2010-05-04, by Cezary Kaliszyk
ExPS3 in NewParser
2010-05-04, by Cezary Kaliszyk
Move ExPS8 to new parser.
2010-05-04, by Cezary Kaliszyk
Fix for new isabelle
2010-05-04, by Cezary Kaliszyk
merge
2010-05-04, by Cezary Kaliszyk
Minor
2010-05-04, by Cezary Kaliszyk
increased step counter so that all steps go through
2010-05-04, by Christian Urban
fixed my error with define_raw_fv
2010-05-04, by Christian Urban
tuned and added some comments to the code; added also an exception for early exit of the nominal2_cmd function
2010-05-04, by Christian Urban
Separate Term8, as it may work soon.
2010-05-04, by Cezary Kaliszyk
moved CoreHaskell to NewParser.
2010-05-04, by Cezary Kaliszyk
ExPS7 in NewParser
2010-05-04, by Cezary Kaliszyk
Move ExLeroy to New Parser
2010-05-04, by Cezary Kaliszyk
Move 2 more to NewParser
2010-05-04, by Cezary Kaliszyk
Move TypeSchemes to NewParser
2010-05-04, by Cezary Kaliszyk
Move ExLet to NewParser.
2010-05-04, by Cezary Kaliszyk
tuned
2010-05-04, by Christian Urban
roll back of the last commit (there was a difference)
2010-05-04, by Christian Urban
tuned
2010-05-04, by 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
2010-05-04, by Christian Urban
merged
2010-05-04, by Christian Urban
some preliminary changes to the pearl-jv paper
2010-05-04, by Christian Urban
some preliminary notes of the abstract (qpaper); still need to see the motivating example
2010-05-03, by Christian Urban
Added cheats to classical
2010-05-03, by Cezary Kaliszyk
Ex2 moved to new parser.
2010-05-03, by Cezary Kaliszyk
alpha_eqvt_tac fixed to work when the existential is not at the top level.
2010-05-03, by Cezary Kaliszyk
SingleLet and Ex3 work with NewParser.
2010-05-03, by Cezary Kaliszyk
Comment
2010-05-03, by Cezary Kaliszyk
Another example where only alpha_eqvt fails.
2010-05-03, by Cezary Kaliszyk
Register only non-looping rules in eq_iff
2010-05-03, by Cezary Kaliszyk
Equivariance fails for single let?
2010-05-03, by Cezary Kaliszyk
NewParser
2010-05-03, by Cezary Kaliszyk
Introduce eq_iff_simp to match the one from Parser.
2010-05-03, by Cezary Kaliszyk
remove tracing
2010-05-03, by Cezary Kaliszyk
Cheat support equations in new parser
2010-05-03, by Cezary Kaliszyk
Remove dependency on NewFv
2010-05-03, by Cezary Kaliszyk
Fix Parser
2010-05-03, by Cezary Kaliszyk
Add explicit cheats in NewParser and comment out the examples for outside use.
2010-05-03, by Cezary Kaliszyk
Fix Datatype_Aux calls in NewParser.
2010-05-03, by Cezary Kaliszyk
Move old fv_alpha_export to Fv.
2010-05-03, by Cezary Kaliszyk
moved old parser and old fv back into their original places; isabelle make works again
2010-05-03, by Christian Urban
slight tuning
2010-05-03, by Christian Urban
simplified the supp-of-finite-sets proof
2010-05-02, by Christian Urban
tried to add some comments in the huge(!) nominal2_cmd function
2010-05-02, by Christian Urban
replaced make_pair with library function HOLogic.mk_prod
2010-05-02, by Christian Urban
removed duplicate eqvt attribute
2010-05-02, by 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)
2010-05-02, by Christian Urban
merged
2010-05-01, by Christian Urban
tuned
2010-05-01, by Christian Urban
replaced hide by the new hide_const
2010-04-30, by Christian Urban
generalised the fs-instance lemma (not just fsets of atoms are finitely supported, but also fsets of finitely supported elements)
2010-04-30, by Christian Urban
added lemmas establishing the support of finite sets of finitely supported elements
2010-04-30, by Christian Urban
added eqvt-lemmas for Bex, Ball and Union
2010-04-30, by Christian Urban
NewParser with Parser functionality, but some cheats included since the order of datayupes is wrong.
2010-04-30, by Cezary Kaliszyk
Merged nominal_datatype into NewParser until eqvts
2010-04-30, by Cezary Kaliszyk
more parser/new parser synchronization.
2010-04-30, by Cezary Kaliszyk
Simplify old parser for integration
2010-04-30, by Cezary Kaliszyk
merge
2010-04-30, by Cezary Kaliszyk
Change signature of fv and alpha generation.
2010-04-30, by Cezary Kaliszyk
reorganised eqvt-file (now uses perm_simp already)
2010-04-30, by Christian Urban
qpaper
2010-04-30, by Cezary Kaliszyk
merge
2010-04-29, by Cezary Kaliszyk
New Alpha.
2010-04-29, by Cezary Kaliszyk
Minimal cleaning in LamEx
2010-04-29, by Cezary Kaliszyk
Remove things moved to the isabelle distribution
2010-04-29, by Cezary Kaliszyk
Unify and give only one name to 'setify', 'listify' and 'set'
2010-04-29, by Cezary Kaliszyk
Fixing the definitions in the Parser.
2010-04-29, by Cezary Kaliszyk
Some of the exceptions that the parser should check in TODO.
2010-04-29, by Cezary Kaliszyk
Extracting the fv body function and exporting the terms.
2010-04-29, by Cezary Kaliszyk
Fix for recursive binders.
2010-04-29, by Cezary Kaliszyk
revert 0c9ef14e9ba4
2010-04-29, by Cezary Kaliszyk
Support in positive position and atoms in negative positions.
2010-04-29, by Cezary Kaliszyk
merge
2010-04-29, by Cezary Kaliszyk
Include support of unknown datatypes in new fv
2010-04-29, by Cezary Kaliszyk
merged
2010-04-29, by Christian Urban
added basic functions for constructing supp-terms
2010-04-29, by Christian Urban
quotient paper
2010-04-29, by Cezary Kaliszyk
added missing latex-style file
2010-04-29, by Christian Urban
merged
2010-04-29, by Christian Urban
added stub for quotient paper; call with isabelle make qpaper
2010-04-29, by Christian Urban
Cleaning of Int and FSet Examples
2010-04-28, by Cezary Kaliszyk
use the more general type-class at_base
2010-04-28, by Christian Urban
deleted left-over code
2010-04-28, by Christian Urban
simpliied and moved the remaining lemmas about the atom-function to Nominal2_Base
2010-04-28, by Christian Urban
use sort at_base instead of at
2010-04-28, by Christian Urban
white spaces
2010-04-28, by Christian Urban
avoided repeated dest of dt_info
2010-04-28, by Christian Urban
tuned
2010-04-28, by Christian Urban
factured out common functionality of prefixing the dt-names with a string
2010-04-28, by Christian Urban
closed Datatype_Aux; replaced nth_dtyp by the function used in Perm.thy
2010-04-28, by Christian Urban
added some further problemetic tests
2010-04-27, by Christian Urban
some tuning
2010-04-27, by Christian Urban
moved mk_atom into the library; that meant that concrete atom classes need to be in Nominal2_Base
2010-04-27, by Christian Urban
merged
2010-04-27, by Christian Urban
Rewrote FV code and included the function package.
2010-04-27, by Cezary Kaliszyk
merge
2010-04-27, by Cezary Kaliszyk
Function in Core Haskell
2010-04-27, by Cezary Kaliszyk
one more pass over the paper
2010-04-27, by Christian Urban
more polishing on the paper
2010-04-27, by Christian Urban
merged
2010-04-26, by Christian Urban
some changes to the paper
2010-04-26, by Christian Urban
rewrote eqvts_raw to be a symtab, that can be looked up
2010-04-26, by Christian Urban
merge ???
2010-04-26, by Cezary Kaliszyk
infix for In
2010-04-21, by Cezary Kaliszyk
eliminated command so that all compiles
2010-04-26, by Christian Urban
changed theorem_i to theorem....requires new Isabelle
2010-04-26, by Christian Urban
tuned
2010-04-25, by Christian Urban
tuned and cleaned
2010-04-25, by Christian Urban
tuned and made to compile
2010-04-25, by Christian Urban
added definition of raw-permutations to the new-parser
2010-04-25, by Christian Urban
tuned
2010-04-25, by Christian Urban
slight tuning
2010-04-25, by Christian Urban
added a comment about a function where I am not sure who wrote it.
2010-04-24, by Christian Urban
merged
2010-04-24, by Christian Urban
Minor
2010-04-23, by Cezary Kaliszyk
Minor cleaning of IntEx
2010-04-23, by Cezary Kaliszyk
Further cleaning of proofs in FSet
2010-04-23, by Cezary Kaliszyk
Update term8
2010-04-22, by Cezary Kaliszyk
Converted 'thm' to a lemma.
2010-04-22, by Cezary Kaliszyk
Moved working Fset3 properties to FSet.
2010-04-22, by Cezary Kaliszyk
tuned parser
2010-04-22, by Christian Urban
moved lemmas from FSet.thy to do with atom to Nominal2_Base, and to do with 'a::at set to Nominal2_Atoms; moved Nominal2_Eqvt.thy one up to be loaded before Nominal2_Atoms
2010-04-22, by Christian Urban
tuned proofs
2010-04-21, by Christian Urban
merged
2010-04-21, by Christian Urban
moved some lemmas into the right places
2010-04-21, by Christian Urban
minor
2010-04-21, by Cezary Kaliszyk
merge
2010-04-21, by Cezary Kaliszyk
append_rsp2 + isarification
2010-04-21, by Cezary Kaliszyk
some small changes
2010-04-21, by Christian Urban
merged
2010-04-21, by Christian Urban
deleted the incomplete proof about pairs of abstractions
2010-04-21, by Christian Urban
added a variant of the induction principle for permutations
2010-04-21, by Christian Urban
merge
2010-04-21, by Cezary Kaliszyk
More about concat
2010-04-21, by Cezary Kaliszyk
merged
2010-04-21, by Christian Urban
incomplete tests
2010-04-21, by Christian Urban
added an improved version of the induction principle for permutations
2010-04-21, by Christian Urban
Working lifting of concat with inline proofs of second level preservation.
2010-04-21, by Cezary Kaliszyk
FSet3 cleaning part2
2010-04-21, by Cezary Kaliszyk
merge
2010-04-21, by Cezary Kaliszyk
Remove the part already in FSet and leave the experiments
2010-04-21, by Cezary Kaliszyk
merged
2010-04-21, by Christian Urban
removed a sorry
2010-04-21, by Christian Urban
renamed Ex1.thy to SingleLet.thy
2010-04-20, by Christian Urban
tuning of the code
2010-04-20, by Christian Urban
Reorder FSet
2010-04-21, by Cezary Kaliszyk
merge
2010-04-21, by Cezary Kaliszyk
lattice properties.
2010-04-21, by Cezary Kaliszyk
All lifted in Term4. Requires new isabelle.
2010-04-20, by Cezary Kaliszyk
fsets are distributive lattices.
2010-04-20, by Cezary Kaliszyk
Fix of comment
2010-04-20, by Cezary Kaliszyk
reordered code
2010-04-20, by Christian Urban
renamed "_empty" and "_append" to "_zero" and "_plus"
2010-04-20, by Christian Urban
removed dead code (nominal cannot deal with argument types of constructors that are functions)
2010-04-20, by Christian Urban
added comment about abstraction in raw permuations
2010-04-20, by Christian Urban
optimised the code of define_raw_perm
2010-04-20, by Christian Urban
deleting function perm_arg in favour of the library function mk_perm
2010-04-19, by Christian Urban
merged
2010-04-19, by Christian Urban
tuned; fleshed out some library functions about permutations; closed Datatype_Aux structure (increases readability)
2010-04-19, by Christian Urban
FSet is a semi-lattice
2010-04-19, by Cezary Kaliszyk
merge
2010-04-19, by Cezary Kaliszyk
Putting FSet in bot typeclass.
2010-04-19, by Cezary Kaliszyk
reorder
2010-04-19, by Cezary Kaliszyk
merged
2010-04-19, by Christian Urban
small updates to the paper; remaining points in PAPER-TODO
2010-04-19, by Christian Urban
sub_list definition and respects
2010-04-19, by Cezary Kaliszyk
Alternate list_eq and equivalence
2010-04-19, by Cezary Kaliszyk
Some new lemmas
2010-04-19, by Cezary Kaliszyk
More cleaning
2010-04-19, by Cezary Kaliszyk
remove more metis
2010-04-19, by Cezary Kaliszyk
more metis cleaning
2010-04-19, by Cezary Kaliszyk
Getting rid of 'metis'.
2010-04-19, by Cezary Kaliszyk
merge
2010-04-19, by Cezary Kaliszyk
Remove 'defer'.
2010-04-19, by Cezary Kaliszyk
merged
2010-04-19, by Christian Urban
tuned proofs
2010-04-19, by Christian Urban
2 more lifted lemmas needed for second representation
2010-04-19, by Cezary Kaliszyk
Accept non-equality eqvt rules in support proofs.
2010-04-19, by Cezary Kaliszyk
merge
2010-04-19, by Cezary Kaliszyk
Locations of files in Parser
2010-04-19, by Cezary Kaliszyk
merge
2010-04-19, by Cezary Kaliszyk
minor FSet3 edits.
2010-04-19, by Cezary Kaliszyk
tuned
2010-04-18, by Christian Urban
moved some general function into nominal_library.ML
2010-04-18, by Christian Urban
tuned; transformation functions now take a context, a thm and return a thm
2010-04-18, by Christian Urban
tuned
2010-04-18, by Christian Urban
equivariance for alpha_raw in CoreHaskell is automatically derived
2010-04-18, by Christian Urban
preliminary parser for perm_simp metod
2010-04-18, by Christian Urban
automatic proofs for equivariance of alphas
2010-04-16, by Christian Urban
Finished proof in Lambda.thy
2010-04-16, by Cezary Kaliszyk
merged
2010-04-16, by Christian Urban
attempt to manual prove eqvt for alpha
2010-04-16, by Christian Urban
Lifting in Term4.
2010-04-16, by Cezary Kaliszyk
some tuning of eqvt-infrastructure
2010-04-16, by Christian Urban
some tuning of proofs
2010-04-15, by Christian Urban
typo
2010-04-15, by Christian Urban
merged
2010-04-15, by Christian Urban
half of the pair-abs-equivalence
2010-04-15, by Christian Urban
More on Manual/Trm4
2010-04-15, by Cezary Kaliszyk
alpha4_equivp and constant lifting.
2010-04-15, by Cezary Kaliszyk
alpha4_eqvt and alpha4_reflp
2010-04-15, by Cezary Kaliszyk
fv_eqvt in term4
2010-04-15, by Cezary Kaliszyk
Updating in Term4.
2010-04-15, by Cezary Kaliszyk
merge
2010-04-15, by Cezary Kaliszyk
Prove insert_rsp2
2010-04-15, by Cezary Kaliszyk
merged
2010-04-15, by Christian Urban
changed header
2010-04-15, by Christian Urban
Minor paper fixes.
2010-04-15, by Cezary Kaliszyk
temporary fix for CoreHaskell
2010-04-14, by Christian Urban
deleted offending [eqvt]-attribute in Abs; Lambda works again, but there is now a problem in CoreHaskell
2010-04-14, by Christian Urban
merge
2010-04-14, by Cezary Kaliszyk
Fix the 'subscript' error.
2010-04-14, by Cezary Kaliszyk
merged
2010-04-14, by Christian Urban
thmdecls can deal with lemmas like alpha_gen which contain pairs or tuples
2010-04-14, by Christian Urban
merge
2010-04-14, by Cezary Kaliszyk
merge
2010-04-14, by Cezary Kaliszyk
Separate alpha_definition.
2010-04-14, by Cezary Kaliszyk
Fix spelling in theory header
2010-04-14, by Cezary Kaliszyk
Separate define_fv.
2010-04-14, by Cezary Kaliszyk
tuned and removed dead code
2010-04-14, by Christian Urban
moved a couple of more functions to the library
2010-04-14, by Christian Urban
added a library for basic nominal functions; separated nominal_eqvt file
2010-04-14, by Christian Urban
merged
2010-04-14, by Christian Urban
first working version of the automatic equivariance procedure
2010-04-14, by Christian Urban
Initial cleaning/reorganization in Fv.
2010-04-14, by Cezary Kaliszyk
merged
2010-04-14, by Christian Urban
preliminary tests
2010-04-14, by Christian Urban
deleted test
2010-04-14, by Christian Urban
merge
2010-04-14, by Cezary Kaliszyk
merge part: delete_rsp
2010-04-14, by Cezary Kaliszyk
merge part1: none_memb_nil
2010-04-14, by Cezary Kaliszyk
added header and more tuning
2010-04-14, by Christian Urban
more tuning
2010-04-14, by Christian Urban
tuned
2010-04-14, by Christian Urban
Working FSet with additional lemmas.
2010-04-13, by Cezary Kaliszyk
Much more in FSet (currently non-working)
2010-04-13, by Cezary Kaliszyk
made everything to compile
2010-04-13, by Christian Urban
merged
2010-04-13, by Christian Urban
some small tunings (incompleted work in Lambda.thy)
2010-04-13, by Christian Urban
moved equivariance of map into Nominal2_Eqvt file
2010-04-13, by Christian Urban
early ott paper
2010-04-12, by Christian Urban
Porting lemmas from Quotient package FSet to new FSet.
2010-04-12, by Cezary Kaliszyk
added alpha-caml paper
2010-04-12, by Christian Urban
implemented in thmdecls the case where eqvt-lemmas are of the form _ ==> _
2010-04-12, by Christian Urban
fixed bug in thmdecls with destructing Trueprop; some initial infrastructure for eqvt-theorems of the form _ ==> _
2010-04-11, by Christian Urban
folded changes from the conference version
2010-04-11, by Christian Urban
added TODO item about parser creating syntax for the wrong type
2010-04-11, by Christian Urban
corrected imports header
2010-04-11, by Christian Urban
tuned
2010-04-11, by Christian Urban
a few tests
2010-04-11, by Christian Urban
added eqvt rules that are more standard
2010-04-11, by Christian Urban
used warning instead of tracing (does not seem to produce stable output)
2010-04-11, by Christian Urban
added small ittems about equivaraince of alpha_gens and name of lam.perm
2010-04-11, by Christian Urban
added more robust tracing infrastructure; a strict version of the eqvt_tac raises an error if not all permutations cannot be analysed
2010-04-11, by Christian Urban
changed the eqvt-tac to move only outermost permutations inside; added tracing infrastructure for the eqvt-tac
2010-04-09, by Christian Urban
rewrite paragraph introducing equivariance, add citation to Pitts03
2010-04-09, by Brian Huffman
edit 'contributions' section so we do not just quote directly from the reviewer
2010-04-09, by Brian Huffman
renamed ExLam to Lambda and completed the proof of the strong ind principle; tuned paper
2010-04-09, by Christian Urban
clarified comment about distinct lists in th efuture work section
2010-04-08, by Christian Urban
tuned type-schemes example
2010-04-08, by Christian Urban
updated (comment about weirdo example)
2010-04-08, by Christian Urban
check whether the "weirdo" example from the binding bestiary works with shallow binders
2010-04-08, by Christian Urban
properly separated the example from my PhD and gave the correct alpha-equivalence relation (according to the paper)
2010-04-08, by Christian Urban
merged
2010-04-08, by Christian Urban
some further changes
2010-04-08, by Christian Urban
merged
2010-04-08, by Brian Huffman
change some wording in conclusion
2010-04-08, by Brian Huffman
remove extra word
2010-04-08, by Brian Huffman
merged
2010-04-08, by Christian Urban
added new paper directory for further work
2010-04-08, by Christian Urban
use qualified name as string in concrete atom example
2010-04-08, by Brian Huffman
merged
2010-04-08, by Brian Huffman
simplify instance proof
2010-04-08, by Brian Huffman
polish explanation of additive group syntax
2010-04-07, by Brian Huffman
final version of the pearl paper
2010-04-08, by Christian Urban
my final version of the paper
2010-04-07, by Christian Urban
added an induction principle for permutations; removed add_perm construction
2010-04-07, by Christian Urban
isarfied proof about existence of a permutation list
2010-04-06, by Christian Urban
added reference to E. Gunter's work
2010-04-06, by Christian Urban
typos in paper
2010-04-06, by Christian Urban
separated general nominal theory into separate folder
2010-04-04, by Christian Urban
added README and moved examples into separate directory
2010-04-03, by Christian Urban
merged pearl paper with this repository; started litrature subdirectory
2010-04-03, by Christian Urban
submitted version (just in time ;o)
2010-04-02, by Christian Urban
first complete version (slightly less than 3h more to go)
2010-04-02, by Christian Urban
tuned
2010-04-02, by Christian Urban
tuned strong ind section
2010-04-02, by Christian Urban
polished infrastruct section
2010-04-02, by Christian Urban
completed lifting section
2010-04-02, by Christian Urban
more on the lifting section
2010-04-02, by Christian Urban
more on the strong induction section
2010-04-02, by Christian Urban
completed conclusion
2010-04-01, by Christian Urban
merged
2010-04-01, by Christian Urban
merged
2010-04-01, by Christian Urban
updated related work section
2010-04-01, by Christian Urban
fv_fv_bn
2010-04-01, by Cezary Kaliszyk
Update fv_bn definition for bindings allowed in types for which bn is present.
2010-04-01, by Cezary Kaliszyk
fv_perm_bn
2010-04-01, by Cezary Kaliszyk
Minor formula fixes.
2010-04-01, by Cezary Kaliszyk
fixed alpha_bn
2010-04-01, by Christian Urban
current state
2010-04-01, by Christian Urban
merged
2010-04-01, by Christian Urban
added alpha_bn definition
2010-04-01, by Christian Urban
hfill for right aligning single table cells.
2010-04-01, by Cezary Kaliszyk
Cleaning the strong induction example.
2010-04-01, by Cezary Kaliszyk
minor
2010-04-01, by Cezary Kaliszyk
Fighting with space in displaying strong induction...
2010-04-01, by Cezary Kaliszyk
starting strong induction
2010-04-01, by Cezary Kaliszyk
General paper minor fixes.
2010-04-01, by Cezary Kaliszyk
Forgot to save before commit.
2010-04-01, by Cezary Kaliszyk
Let with multiple bindings.
2010-04-01, by Cezary Kaliszyk
Fill the space below the figure.
2010-04-01, by Cezary Kaliszyk
last commit for now.
2010-04-01, by Christian Urban
more on the conclusion
2010-04-01, by Christian Urban
completed related work section
2010-04-01, by Christian Urban
more on the paper
2010-04-01, by Christian Urban
added an item about alpha-equivalence (the existential should be closer to the abstraction)
2010-04-01, by Christian Urban
polished everything up to TODO
2010-03-31, by Christian Urban
merged
2010-03-31, by Christian Urban
added alpha-definition for ~~ty
2010-03-31, by Christian Urban
permute_bn
2010-03-31, by Cezary Kaliszyk
abbreviations for \<otimes> and \<oplus>
2010-03-31, by Christian Urban
merged
2010-03-31, by Christian Urban
a test with let having multiple bodies
2010-03-31, by Christian Urban
polished and removed tys from bn-functions.
2010-03-31, by Christian Urban
merge
2010-03-31, by Cezary Kaliszyk
More on paper
2010-03-31, by Cezary Kaliszyk
started to polish alpha-equivalence section, but needs more work
2010-03-31, by Christian Urban
started with a related work section
2010-03-31, by Christian Urban
polished and added an example for fvars
2010-03-30, by Christian Urban
cleaned up the section about fv's
2010-03-30, by Christian Urban
tuned beginning of section 4
2010-03-30, by Christian Urban
More on section 5.
2010-03-30, by Cezary Kaliszyk
More on section 5.
2010-03-30, by Cezary Kaliszyk
merged
2010-03-30, by Christian Urban
removed "raw" distinction
2010-03-30, by Christian Urban
More on Section 5
2010-03-30, by Cezary Kaliszyk
Beginning of section 5.
2010-03-30, by Cezary Kaliszyk
merged
2010-03-30, by Christian Urban
Avoid mentioning other nominal datatypes as it makes things too complicated.
2010-03-30, by Cezary Kaliszyk
merged
2010-03-30, by Christian Urban
close the missing parenthesis on both sides.
2010-03-30, by Cezary Kaliszyk
merged
2010-03-30, by Christian Urban
changes to section 2
2010-03-30, by Christian Urban
Clean alpha
2010-03-30, by Cezary Kaliszyk
clean fv_bn
2010-03-30, by Cezary Kaliszyk
alpha_bn
2010-03-30, by Cezary Kaliszyk
Change @{text} to @{term}
2010-03-30, by Cezary Kaliszyk
alpha
2010-03-30, by Cezary Kaliszyk
more
2010-03-30, by Cezary Kaliszyk
fv and fv_bn
2010-03-30, by Cezary Kaliszyk
more of the paper
2010-03-30, by Christian Urban
merged
2010-03-29, by Christian Urban
Updated strong induction to modified definitions.
2010-03-29, by Cezary Kaliszyk
Initial renaming
2010-03-29, by Cezary Kaliszyk
small changes in the core-haskell spec
2010-03-29, by Christian Urban
Update according to paper
2010-03-29, by Cezary Kaliszyk
merge
2010-03-29, by Cezary Kaliszyk
merge
2010-03-29, by Cezary Kaliszyk
Changed to Lists.
2010-03-29, by Cezary Kaliszyk
clarified core-haskell example
2010-03-29, by Christian Urban
spell check
2010-03-29, by Christian Urban
merge
2010-03-29, by Cezary Kaliszyk
Abs_gen and Abs_let simplifications.
2010-03-29, by Cezary Kaliszyk
more on the paper
2010-03-29, by Christian Urban
fixed a problem due to a change in type-def (needs new Isabelle)
2010-03-29, by Christian Urban
merged
2010-03-29, by Christian Urban
more on the paper
2010-03-29, by Christian Urban
got rid of the aux-function on the raw level, by defining it with function on the quotient level
2010-03-28, by Christian Urban
Lets finally abstract lists.
2010-03-27, by Cezary Kaliszyk
Core Haskell can now use proper strings.
2010-03-27, by Cezary Kaliszyk
Automatically lift theorems and constants only using the new quotient types. Requires new Isabelle.
2010-03-27, by Cezary Kaliszyk
Remove list_eq notation.
2010-03-27, by Cezary Kaliszyk
Get lifted types information from the quotient package.
2010-03-27, by Cezary Kaliszyk
Equivariance when bn functions are lists.
2010-03-27, by Cezary Kaliszyk
Accepts lists in FV.
2010-03-27, by Cezary Kaliszyk
Parsing of list-bn functions into components.
2010-03-27, by Cezary Kaliszyk
Automatically compute support if only one type of Abs is present in the type.
2010-03-27, by Cezary Kaliszyk
Manually proved TySch support; All properties of TySch now true.
2010-03-27, by Cezary Kaliszyk
Generalize Abs_eq_iff.
2010-03-27, by Cezary Kaliszyk
Minor fix.
2010-03-27, by Cezary Kaliszyk
New compose lemmas. Reverted alpha_gen sym/trans changes. Equivp for alpha_res should work now.
2010-03-27, by Cezary Kaliszyk
Initial proof modifications for alpha_res
2010-03-27, by Cezary Kaliszyk
merge
2010-03-27, by Cezary Kaliszyk
Fv/Alpha now takes into account Alpha_Type given from the parser.
2010-03-27, by Cezary Kaliszyk
Minor cleaning.
2010-03-27, by Cezary Kaliszyk
merged
2010-03-27, by Christian Urban
more on the paper
2010-03-27, by Christian Urban
Removed some warnings.
2010-03-27, by Cezary Kaliszyk
merge
2010-03-26, by Cezary Kaliszyk
Modified abs_gen_sym and abs_gen_trans so it becomes usable in the proofs.
2010-03-26, by Cezary Kaliszyk
merged
2010-03-26, by Christian Urban
more on the paper
2010-03-26, by Christian Urban
simplification
2010-03-26, by Christian Urban
merge
2010-03-26, by Cezary Kaliszyk
Describe 'nominal_datatype2'.
2010-03-26, by Cezary Kaliszyk
Fixed renamings.
2010-03-26, by Cezary Kaliszyk
merged
2010-03-26, by Christian Urban
Removed remaining cheats + some cleaning.
2010-03-26, by Cezary Kaliszyk
Extract PS7 and PS8 from Test. PS7 needs the same fix as Core Haskell.
2010-03-26, by Cezary Kaliszyk
Update cheats in TODO.
2010-03-26, by Cezary Kaliszyk
Removed another cheat and cleaned the code a bit.
2010-03-26, by Cezary Kaliszyk
Fix Manual/LamEx for experiments.
2010-03-26, by Cezary Kaliszyk
Proper bn_rsp, for bn functions calling each other.
2010-03-25, by Cezary Kaliszyk
Gathering things to prove by induction together; removed cheat_bn_eqvt.
2010-03-25, by Cezary Kaliszyk
Update TODO
2010-03-25, by Cezary Kaliszyk
Showed ACons_subst.
2010-03-25, by Cezary Kaliszyk
Only ACons_subst left to show.
2010-03-25, by Cezary Kaliszyk
Solved all boring subgoals, and looking at properly defning permute_bv
2010-03-25, by Cezary Kaliszyk
One more copy-and-paste in core-haskell.
2010-03-25, by Cezary Kaliszyk
Properly defined permute_bn. No more sorry's in Let strong induction.
2010-03-25, by Cezary Kaliszyk
Showed Let substitution.
2010-03-25, by Cezary Kaliszyk
Only let substitution is left.
2010-03-25, by Cezary Kaliszyk
further in the proof
2010-03-25, by Cezary Kaliszyk
trying to prove the string induction for let.
2010-03-25, by Cezary Kaliszyk
added experiemental permute_bn
2010-03-25, by Christian Urban
first attempt of strong induction for lets with assignments
2010-03-25, by Christian Urban
more on the paper
2010-03-25, by Christian Urban
more on the paper
2010-03-24, by Christian Urban
Further in the strong induction proof.
2010-03-24, by Cezary Kaliszyk
Solved one of the strong-induction goals.
2010-03-24, by Cezary Kaliszyk
avoiding for atom.
2010-03-24, by Cezary Kaliszyk
Started proving strong induction.
2010-03-24, by Cezary Kaliszyk
stating the strong induction; further.
2010-03-24, by Cezary Kaliszyk
Working on stating induct.
2010-03-24, by Cezary Kaliszyk
some tuning; possible fix for strange paper generation
2010-03-24, by Christian Urban
more on the paper
2010-03-24, by Christian Urban
merge
2010-03-24, by Cezary Kaliszyk
Showed support of Core Haskell
2010-03-24, by Cezary Kaliszyk
Support proof modification for Core Haskell.
2010-03-24, by Cezary Kaliszyk
Experiments with Core Haskell support.
2010-03-24, by Cezary Kaliszyk
Export all the cheats needed for Core Haskell.
2010-03-24, by Cezary Kaliszyk
Compute Fv for non-recursive bn functions calling other bn functions
2010-03-24, by Cezary Kaliszyk
Core Haskell experiments.
2010-03-24, by Cezary Kaliszyk
tuned paper
2010-03-24, by Christian Urban
more of the paper
2010-03-23, by Christian Urban
merged
2010-03-23, by Christian Urban
more tuning in the paper
2010-03-23, by Christian Urban
merge
2010-03-23, by Cezary Kaliszyk
Parsing bn functions that call other bn functions and transmitting this information to fv/alpha.
2010-03-23, by Cezary Kaliszyk
merged
2010-03-23, by Christian Urban
more tuning
2010-03-23, by Christian Urban
tuned paper
2010-03-23, by Christian Urban
more on the paper
2010-03-23, by Christian Urban
merge
2010-03-23, by Cezary Kaliszyk
Modification to Core Haskell to make it accepted with an empty binding function.
2010-03-23, by Cezary Kaliszyk
merged
2010-03-23, by Christian Urban
tuned paper
2010-03-23, by Christian Urban
Initial list unfoldings in Core Haskell.
2010-03-23, by Cezary Kaliszyk
compiles
2010-03-23, by Cezary Kaliszyk
More modification needed for compilation
2010-03-23, by Cezary Kaliszyk
Moved let properties from Term5 to ExLetRec.
2010-03-23, by Cezary Kaliszyk
Move Let properties to ExLet
2010-03-23, by Cezary Kaliszyk
Added missing file
2010-03-23, by Cezary Kaliszyk
More reorganization.
2010-03-23, by Cezary Kaliszyk
Move Leroy out of Test, rename accordingly.
2010-03-23, by Cezary Kaliszyk
Term1 is identical to Example 3
2010-03-23, by Cezary Kaliszyk
Move example3 out.
2010-03-23, by Cezary Kaliszyk
Move Ex1 and Ex2 out of Test
2010-03-23, by Cezary Kaliszyk
Move examples which create more permutations out
2010-03-23, by Cezary Kaliszyk
Move LamEx out of Test.
2010-03-23, by Cezary Kaliszyk
Move lambda examples to manual
2010-03-23, by Cezary Kaliszyk
Move manual examples to a subdirectory.
2010-03-23, by Cezary Kaliszyk
Removed compat tests.
2010-03-23, by Cezary Kaliszyk
merge
2010-03-23, by Cezary Kaliszyk
Move Non-respectful examples to NotRsp
2010-03-23, by Cezary Kaliszyk
merged
2010-03-23, by Christian Urban
more on the paper
2010-03-23, by Christian Urban
Move the comment to appropriate place.
2010-03-23, by Cezary Kaliszyk
Remove compose_eqvt
2010-03-23, by Cezary Kaliszyk
sym proof with compose.
2010-03-22, by Cezary Kaliszyk
Marked the place where a compose lemma applies.
2010-03-22, by Cezary Kaliszyk
merge
2010-03-22, by Cezary Kaliszyk
equivp_cheat can be removed for all one-permutation examples.
2010-03-22, by Cezary Kaliszyk
merged
2010-03-22, by Christian Urban
more on the paper
2010-03-22, by Christian Urban
merged
2010-03-22, by Christian Urban
tuned paper
2010-03-22, by Christian Urban
Got rid of alpha_bn_rsp_cheat.
2010-03-22, by Cezary Kaliszyk
alpha_bn_rsp_pre automatized.
2010-03-22, by Cezary Kaliszyk
merge
2010-03-22, by Cezary Kaliszyk
fv_rsp proved automatically.
2010-03-22, by Cezary Kaliszyk
more on the paper
2010-03-22, by Christian Urban
merged
2010-03-22, by Christian Urban
tuned paper
2010-03-22, by Christian Urban
some tuning
2010-03-22, by Christian Urban
Strong induction for Type Schemes.
2010-03-22, by Cezary Kaliszyk
Fixed missing colon.
2010-03-22, by Cezary Kaliszyk
tuned paper
2010-03-21, by Christian Urban
merged
2010-03-20, by Christian Urban
proved at_set_avoiding2 which is needed for strong induction principles
2010-03-20, by Christian Urban
moved lemmas supp_perm_eq and exists_perm to Nominal2_Supp
2010-03-20, by Christian Urban
Size experiments.
2010-03-20, by Cezary Kaliszyk
Use 'alpha_bn_refl' to get rid of one of the sorrys.
2010-03-20, by Cezary Kaliszyk
Build alpha-->alphabn implications
2010-03-20, by Cezary Kaliszyk
Prove reflp for all relations.
2010-03-20, by Cezary Kaliszyk
started cleaning up and introduced 3 versions of ~~gen
2010-03-20, by Christian Urban
moved infinite_Un into mainstream Isabelle; moved permute_boolI/E lemmas
2010-03-20, by Christian Urban
more work on the paper
2010-03-19, by Christian Urban
Described automatically created funs.
2010-03-19, by Cezary Kaliszyk
merge
2010-03-19, by Cezary Kaliszyk
Automatically derive support for datatypes with at-most one binding per constructor.
2010-03-19, by Cezary Kaliszyk
picture
2010-03-19, by Christian Urban
merged
2010-03-19, by Christian Urban
polished
2010-03-19, by Christian Urban
Update Test to use fset.
2010-03-19, by Cezary Kaliszyk
merge
2010-03-19, by Cezary Kaliszyk
Use fs typeclass in showing finite support + some cheat cleaning.
2010-03-19, by Cezary Kaliszyk
merged
2010-03-19, by Christian Urban
more one the paper
2010-03-19, by Christian Urban
Keep only one copy of infinite_Un.
2010-03-19, by Cezary Kaliszyk
Added a missing 'import'.
2010-03-19, by Cezary Kaliszyk
Showed the instance: fset::(at) fs
2010-03-19, by Cezary Kaliszyk
merge
2010-03-19, by Cezary Kaliszyk
Remove atom_decl from the parser.
2010-03-19, by Cezary Kaliszyk
TySch strong induction looks ok.
2010-03-19, by Cezary Kaliszyk
Working on TySch strong induction.
2010-03-19, by Cezary Kaliszyk
Something is wrong with the statement of strong induction for TySch, as the All case is trivial and Fun case unprovable...
2010-03-19, by Cezary Kaliszyk
merged
2010-03-19, by Christian Urban
more tuning on the paper
2010-03-19, by Christian Urban
The nominal infrastructure for fset. 'fs' missing, but not needed so far.
2010-03-19, by Cezary Kaliszyk
A few more theorems in FSet.
2010-03-19, by Cezary Kaliszyk
merge 2
2010-03-19, by Cezary Kaliszyk
merge 1
2010-03-19, by Cezary Kaliszyk
support of fset_to_set, support of fmap_atom.
2010-03-19, by Cezary Kaliszyk
merged
2010-03-18, by Christian Urban
more tuning on the paper
2010-03-18, by Christian Urban
added item about size functions
2010-03-18, by Christian Urban
merge
2010-03-18, by Cezary Kaliszyk
Reached strong_induction in fset-based TySch. Will not work until isabelle changes are pushed.
2010-03-18, by Cezary Kaliszyk
tuned
2010-03-18, by Christian Urban
another little bit for the introduction
2010-03-18, by Christian Urban
Leroy96 supp=fv and fixes to make it compile
2010-03-18, by Cezary Kaliszyk
merged
2010-03-18, by Christian Urban
more of the introduction
2010-03-18, by Christian Urban
merge
2010-03-18, by Cezary Kaliszyk
Added a cleaned version of FSet.
2010-03-18, by Cezary Kaliszyk
corrected the strong induction principle in the lambda-calculus case; gave a second (oartial) version that is more elegant
2010-03-18, by Christian Urban
Continued description of alpha.
2010-03-18, by Cezary Kaliszyk
Rename "_property" to ".property"
2010-03-18, by Cezary Kaliszyk
First part of the description of alpha_ty.
2010-03-18, by Cezary Kaliszyk
Description of generation of alpha_bn.
2010-03-18, by Cezary Kaliszyk
case names also for _induct
2010-03-18, by Cezary Kaliszyk
Case_Names for _inducts. Does not work for _induct yet.
2010-03-18, by Cezary Kaliszyk
Added fv,bn,distinct,perm to the simplifier.
2010-03-18, by Cezary Kaliszyk
merge
2010-03-18, by Cezary Kaliszyk
Simplified the description.
2010-03-18, by Cezary Kaliszyk
merged
2010-03-18, by Christian Urban
slightly more in the paper
2010-03-18, by Christian Urban
Update the description of the generation of fv function.
2010-03-18, by Cezary Kaliszyk
fv_bn may need to call other fv_bns.
2010-03-18, by Cezary Kaliszyk
Update TODO.
2010-03-18, by Cezary Kaliszyk
Which proofs need a 'sorry'.
2010-03-18, by Cezary Kaliszyk
added TODO
2010-03-18, by Christian Urban
vixed variable names
2010-03-18, by Christian Urban
simplified strong induction proof by using flip
2010-03-18, by Christian Urban
Rename bound variables + minor cleaning.
2010-03-18, by Cezary Kaliszyk
Move most of the exporting out of the parser.
2010-03-18, by Cezary Kaliszyk
Prove pseudo-inject (eq-iff) on the exported level and rename appropriately.
2010-03-18, by Cezary Kaliszyk
Prove eqvts on exported terms.
2010-03-18, by Cezary Kaliszyk
Clean 'Lift', start working only on exported things in Parser.
2010-03-18, by Cezary Kaliszyk
slightly more of the paper
2010-03-18, by Christian Urban
merged
2010-03-17, by Christian Urban
paper uses now a heap file - does not compile so long anymore
2010-03-17, by Christian Urban
merge
2010-03-17, by Cezary Kaliszyk
compose_sym2 works also for term5
2010-03-17, by Cezary Kaliszyk
Updated Term1, including statement of strong induction.
2010-03-17, by Cezary Kaliszyk
Proper compose_sym2
2010-03-17, by Cezary Kaliszyk
merged
2010-03-17, by Christian Urban
temporarily disabled tests in Nominal/ROOT
2010-03-17, by Christian Urban
made paper to compile
2010-03-17, by Christian Urban
added partial proof for the strong induction principle
2010-03-17, by Christian Urban
Trying to find a compose lemma for 2 arguments.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
2010-03-17, by Cezary Kaliszyk
merged
2010-03-17, by Christian Urban
added proof of supp/fv for type schemes
2010-03-17, by Christian Urban
Updated Type Schemes to automatic lifting. One goal is not true because of the restriction.
2010-03-17, by Cezary Kaliszyk
Remove Term5a, since it is now identical to Term5.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
Finished all proofs in Term5 and Term5n.
2010-03-17, by Cezary Kaliszyk
added partial proof of supp for type schemes
2010-03-17, by Christian Urban
Fix in alpha; support of the recursive Let works :)
2010-03-17, by Cezary Kaliszyk
The recursive supp just has one equation too much.
2010-03-17, by Cezary Kaliszyk
Fix for the change of alpha_gen.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
Generate compound FV and Alpha for recursive bindings.
2010-03-17, by Cezary Kaliszyk
Lifting theorems with compound fv and compound alpha.
2010-03-17, by Cezary Kaliszyk
commented out examples that should not work; but for example type-scheme example should work
2010-03-17, by Christian Urban
added another supp-proof for the non-recursive case
2010-03-17, by Christian Urban
Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
2010-03-16, by Cezary Kaliszyk
merge
2010-03-16, by Cezary Kaliszyk
The old recursive alpha works fine.
2010-03-16, by Cezary Kaliszyk
added the final unfolded result
2010-03-16, by Christian Urban
merge and proof of support for non-recursive case
2010-03-16, by Christian Urban
Added Term5 non-recursive. The bug is there only for the recursive case.
2010-03-16, by Cezary Kaliszyk
Alpha is wrong.
2010-03-16, by Cezary Kaliszyk
alpha_bn doesn't need the permutation in non-recursive case.
2010-03-16, by Cezary Kaliszyk
alpha5_transp and equivp
2010-03-16, by Cezary Kaliszyk
alpha5_symp proved.
2010-03-16, by Cezary Kaliszyk
FV_bn generated for recursive functions as well, and used in main fv for bindings.
2010-03-16, by Cezary Kaliszyk
The proof in 'Test' gets simpler.
2010-03-16, by Cezary Kaliszyk
Removed pi o bn = bn' assumption in alpha
2010-03-16, by Cezary Kaliszyk
merged (confirmed to work with Isabelle from 6th March)
2010-03-15, by Christian Urban
another synchronisation
2010-03-15, by Christian Urban
proof for support when bn-function is present, but fb_function is empty
2010-03-15, by Christian Urban
fv_eqvt_cheat no longer needed.
2010-03-15, by Cezary Kaliszyk
derive "inducts" from "induct" instead of lifting again is much faster.
2010-03-15, by Cezary Kaliszyk
build_eqvts works with recursive case if proper induction rule is used.
2010-03-15, by Cezary Kaliszyk
cheat_alpha_eqvt no longer needed; the proofs work.
2010-03-15, by Cezary Kaliszyk
LF works with new alpha...?
2010-03-15, by Cezary Kaliszyk
explicit flag "cheat_equivp"
2010-03-15, by Cezary Kaliszyk
Prove alpha_gen_compose_eqvt
2010-03-15, by Cezary Kaliszyk
Use eqvt.
2010-03-15, by Cezary Kaliszyk
added preliminary test version....but Test works now
2010-03-15, by Christian Urban
added an eqvt-proof for bi
2010-03-15, by Christian Urban
synchronised with main hg-repository; used add_typedef_global in nominal_atoms
2010-03-15, by Christian Urban
localised the typedef in Attic (requires new Isabelle)
2010-03-14, by Christian Urban
started supp-fv proofs (is going to work)
2010-03-13, by Christian Urban
Even with pattern simplified to a single clause, the supp equation doesn't seem true.
2010-03-12, by Cezary Kaliszyk
Still don't know how to prove supp=fv for simplest Let...
2010-03-12, by Cezary Kaliszyk
Do not fail if the finite support proof fails.
2010-03-11, by Cezary Kaliszyk
generalised the supp for atoms to all concrete atoms (not just names)
2010-03-11, by Christian Urban
support of atoms at the end of Abs.thy
2010-03-11, by Christian Urban
Trying to prove atom_image_fresh_swap
2010-03-11, by Cezary Kaliszyk
Finite_support proof no longer needed in LF.
2010-03-11, by Cezary Kaliszyk
Show that the new types are in finite support typeclass.
2010-03-11, by Cezary Kaliszyk
mk_supports_eq and supports_tac.
2010-03-11, by Cezary Kaliszyk
merge
2010-03-11, by Cezary Kaliszyk
Fixes for term1 for new alpha. Still not able to show support equations.
2010-03-11, by Cezary Kaliszyk
merged
2010-03-11, by Christian Urban
finally the proof that new and old alpha agree
2010-03-11, by Christian Urban
Remove "_raw" from lifted theorems.
2010-03-11, by Cezary Kaliszyk
looking at trm5_equivp
2010-03-11, by Cezary Kaliszyk
The cheats described explicitely.
2010-03-11, by Cezary Kaliszyk
The alpha5_eqvt tactic works if I manage to build the goal.
2010-03-11, by Cezary Kaliszyk
With the 4 cheats, all examples fully lift.
2010-03-11, by Cezary Kaliszyk
Lift alpha_bn_constants.
2010-03-11, by Cezary Kaliszyk
Lifting constants.
2010-03-11, by Cezary Kaliszyk
Proper error message.
2010-03-11, by Cezary Kaliszyk
Lifting constants works for all examples.
2010-03-11, by Cezary Kaliszyk
Remove tracing from fv/alpha.
2010-03-11, by Cezary Kaliszyk
Equivp working only on the standard alpha-equivalences.
2010-03-11, by Cezary Kaliszyk
explicit cheat_fv_eqvt
2010-03-11, by Cezary Kaliszyk
extract build_eqvts_tac.
2010-03-11, by Cezary Kaliszyk
build_eqvts no longer requires permutations.
2010-03-11, by Cezary Kaliszyk
Add explicit alpha_eqvt_cheat.
2010-03-11, by Cezary Kaliszyk
Export tactic out of alpha_eqvt.
2010-03-11, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
More tries about the proofs in trm5
2010-03-10, by Cezary Kaliszyk
merged
2010-03-10, by Christian Urban
almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining)
2010-03-10, by Christian Urban
alpha_equivp for trm5
2010-03-10, by Cezary Kaliszyk
Undoing mistakenly committed parser experiments.
2010-03-10, by Cezary Kaliszyk
alpha_eqvt for recursive term1.
2010-03-10, by Cezary Kaliszyk
Looking at alpha_eqvt for term5, not much progress.
2010-03-10, by Cezary Kaliszyk
Reordered examples in Test.
2010-03-10, by Cezary Kaliszyk
Allows multiple bindings with same lhs.
2010-03-10, by Cezary Kaliszyk
Linked parser to fv and alpha.
2010-03-10, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
A minor fix for shallow binders. LF works again.
2010-03-10, by Cezary Kaliszyk
merged
2010-03-10, by Christian Urban
parser produces ordered bn-fun information
2010-03-10, by Christian Urban
Testing equalities in trm5, all seems good.
2010-03-10, by Cezary Kaliszyk
Fv&Alpha seem to work.
2010-03-10, by Cezary Kaliszyk
include alpha in the definitions.
2010-03-10, by Cezary Kaliszyk
Filled the algorithm for alpha_bn_arg
2010-03-10, by Cezary Kaliszyk
rhs of alpha_bn, and template for the arguments.
2010-03-10, by Cezary Kaliszyk
alpha_bn_constr template
2010-03-10, by Cezary Kaliszyk
exported template for alpha_bn
2010-03-10, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
Use alpha_bns in normal alpha defs.
2010-03-10, by Cezary Kaliszyk
alpha_bn_frees
2010-03-10, by Cezary Kaliszyk
merged
2010-03-09, by Christian Urban
added bn-information, but it is not yet ordered according to the dts
2010-03-09, by Christian Urban
Separate lists for separate constructors, to match bn_eqs.
2010-03-09, by Cezary Kaliszyk
All examples should work.
2010-03-09, by Cezary Kaliszyk
Fix to get old alpha.
2010-03-09, by Cezary Kaliszyk
Separate primrecs in Fv.
2010-03-09, by Cezary Kaliszyk
A version of Fv that takes into account recursive and non-recursive bindings.
2010-03-09, by Cezary Kaliszyk
Trying to prove that old alpha is the same as new recursive one. Lets still to do.
2010-03-09, by Cezary Kaliszyk
fv_bi and alpha_bi
2010-03-09, by Cezary Kaliszyk
merged
2010-03-09, by Christian Urban
added first test about new compat
2010-03-09, by Christian Urban
fv_compat
2010-03-09, by Cezary Kaliszyk
added another compat example
2010-03-09, by Christian Urban
added a test-file for compatibility
2010-03-08, by Christian Urban
added compat definitions to some examples
2010-03-08, by Christian Urban
Proper recognition of atoms and atom sets.
2010-03-08, by Cezary Kaliszyk
deleted comments about "weird"
2010-03-08, by Christian Urban
merged
2010-03-08, by Christian Urban
updated to new Isabelle
2010-03-08, by Christian Urban
Term5 written as nominal_datatype is the recursive let.
2010-03-08, by Cezary Kaliszyk
With restricted_nominal=1, exp7 and exp8 work. Not sure about proving bn_rsp there.
2010-03-08, by Cezary Kaliszyk
More fine-grained nominal restriction for debugging.
2010-03-08, by Cezary Kaliszyk
Fix permutation addition.
2010-03-08, by Cezary Kaliszyk
Update the comments
2010-03-08, by Cezary Kaliszyk
Gather bindings with same binder, and generate only one permutation for them.
2010-03-08, by Cezary Kaliszyk
Undo effects of simp.
2010-03-08, by Cezary Kaliszyk
merged
2010-03-07, by Christian Urban
updated to renamings in Isabelle
2010-03-07, by Christian Urban
merged
2010-03-04, by Christian Urban
merged
2010-03-04, by Christian Urban
more proofs in Abs and work on Core Haskell
2010-03-04, by Christian Urban
added a lemma that permutations can be represented as sums of swapping
2010-03-03, by Christian Urban
Still unable to show supp=fv for let with one existential.
2010-03-05, by Cezary Kaliszyk
Ported LF to the parser interface.
2010-03-05, by Cezary Kaliszyk
merge
2010-03-05, by Cezary Kaliszyk
Lift fv and bn eqvts; no need to lift alpha_eqvt.
2010-03-05, by Cezary Kaliszyk
Not much progress about the single existential let case.
2010-03-05, by Cezary Kaliszyk
Fixed LF for one quantifier over 2 premises.
2010-03-05, by Cezary Kaliszyk
Trying to fix the proofs for the single existential... So far failed.
2010-03-05, by Cezary Kaliszyk
Lift distinct.
2010-03-04, by Cezary Kaliszyk
Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
2010-03-04, by Cezary Kaliszyk
Lift BV,FV,Permutations and injection :).
2010-03-04, by Cezary Kaliszyk
Comment out Weird and Phd until we have an idea how to handle multiple permutations. Transp that works for multiple existentials.
2010-03-04, by Cezary Kaliszyk
A version that just leaves the supp/\supp goal. Obviously not true.
2010-03-04, by Cezary Kaliszyk
Prove symp and transp of weird without the supp /\ supp = {} assumption.
2010-03-04, by Cezary Kaliszyk
merge
2010-03-03, by Cezary Kaliszyk
Experiments with proving weird transp
2010-03-03, by Cezary Kaliszyk
Code for solving symp goals with multiple existentials.
2010-03-03, by Cezary Kaliszyk
reflp for multiple quantifiers.
2010-03-03, by Cezary Kaliszyk
fixed mess in Test.thy
2010-03-03, by Christian Urban
Fix eqvt for multiple quantifiers.
2010-03-03, by Cezary Kaliszyk
only tuned
2010-03-03, by Christian Urban
merged
2010-03-03, by Christian Urban
start of paper - does not compile yet
2010-03-03, by Christian Urban
added ACM style file for ICFP
2010-03-03, by Christian Urban
weird eqvt
2010-03-03, by Cezary Kaliszyk
Add the supp intersection conditions.
2010-03-03, by Cezary Kaliszyk
Comment out the part that does not work with 2 quantifiers.
2010-03-02, by Cezary Kaliszyk
Fixes for the fv problem and alpha problem.
2010-03-02, by Cezary Kaliszyk
merged
2010-03-02, by Christian Urban
preliinary test about alpha-weirdo
2010-03-02, by Christian Urban
Another problem with permutations in alpha and possibly also in fv
2010-03-02, by Christian Urban
potential problem with the phd-example, where two permutations are generated, but only one is used
2010-03-02, by Christian Urban
Some tests around Term4. Not sure how to fix the generated fv function.
2010-03-02, by Cezary Kaliszyk
merge
2010-03-02, by Cezary Kaliszyk
Porting from Lift to Parser; until defining the Quotient type.
2010-03-02, by Cezary Kaliszyk
Add image_eqvt and atom_eqvt to eqvt bases.
2010-03-02, by Cezary Kaliszyk
Include the raw eqvt lemmas.
2010-03-02, by Cezary Kaliszyk
merged
2010-03-02, by Christian Urban
added some more examples from Peter Sewell's bestiary
2010-03-02, by Christian Urban
merge
2010-03-02, by Cezary Kaliszyk
Minor
2010-03-02, by Cezary Kaliszyk
Working bv_eqvt
2010-03-02, by Cezary Kaliszyk
Moving wrappers out of Lift.
2010-03-02, by Cezary Kaliszyk
merged
2010-03-02, by Christian Urban
added distinctness of perms
2010-03-02, by Christian Urban
updated (added lemma about commuting permutations)
2010-03-02, by Christian Urban
Change type schemes to name set.
2010-03-02, by Cezary Kaliszyk
More fixes for new alpha, the whole lift script should now work again.
2010-03-02, by Cezary Kaliszyk
Length fix for nested recursions.
2010-03-02, by Cezary Kaliszyk
Fix equivp.
2010-03-02, by Cezary Kaliszyk
Fixed eqvt code.
2010-03-02, by Cezary Kaliszyk
most tests work - the ones that do not I commented out
2010-03-02, by Christian Urban
merge
2010-03-02, by Cezary Kaliszyk
Add a check of fv_functions.
2010-03-02, by Cezary Kaliszyk
some tuning
2010-03-02, by Christian Urban
Link calls to Raw permutations, FV definition and alpha_definition into the parser.
2010-03-02, by Cezary Kaliszyk
merged
2010-03-02, by Christian Urban
rawified the bind specs (ready to be used now)
2010-03-02, by Christian Urban
merge
2010-03-01, by Cezary Kaliszyk
Trying to prove equivariance.
2010-03-01, by Cezary Kaliszyk
modified for new binding format - hope it is the intended one
2010-03-01, by Christian Urban
further code-refactoring in the parser
2010-03-01, by Christian Urban
The new alpha-equivalence and testing in Trm2 and Trm5.
2010-03-01, by Cezary Kaliszyk
slight simplification of the raw-decl generation
2010-03-01, by Christian Urban
Example that shows that current alpha is wrong.
2010-03-01, by Cezary Kaliszyk
added example from my phd
2010-03-01, by Christian Urban
streamlined parser
2010-02-27, by Christian Urban
generated the "binding list" from the input; at the moment it is only printed out as tracing; does not yet include the "bind itself binders"
2010-02-26, by Christian Urban
More about the general lifting procedure.
2010-02-26, by Cezary Kaliszyk
Update TODO
2010-02-26, by Cezary Kaliszyk
Progress with general lifting procedure.
2010-02-26, by Cezary Kaliszyk
RSP of perms can be shown in one go.
2010-02-26, by Cezary Kaliszyk
Change in signature of prove_const_rsp for general lifting.
2010-02-26, by Cezary Kaliszyk
Permutation and FV_Alpha interface change.
2010-02-26, by Cezary Kaliszyk
To call quotient it is enough to export the alpha frees to proper constants and their respective equivp theorems.
2010-02-26, by Cezary Kaliszyk
merge
2010-02-25, by Cezary Kaliszyk
Preparing the generalized lifting procedure
2010-02-25, by Cezary Kaliszyk
merged
2010-02-25, by Christian Urban
added ott-example about Leroy96
2010-02-25, by Christian Urban
Forgot to add one file.
2010-02-25, by Cezary Kaliszyk
Split Terms into separate files and add them to tests.
2010-02-25, by Cezary Kaliszyk
merge
2010-02-25, by Cezary Kaliszyk
Move the eqvt code out of Terms and fixed induction for single-rule examples.
2010-02-25, by Cezary Kaliszyk
merged
2010-02-25, by Christian Urban
a few simplifications
2010-02-25, by Christian Urban
first attempt to make sense out of the core-haskell definition
2010-02-25, by Christian Urban
Code for proving eqvt, still in Terms.
2010-02-25, by Cezary Kaliszyk
Use eqvt infrastructure.
2010-02-25, by Cezary Kaliszyk
Simple function eqvt code.
2010-02-25, by Cezary Kaliszyk
added IsaMakefile...but so far included only a test for the parser
2010-02-25, by Christian Urban
moved Quot package to Attic (still compiles there with "isabelle make")
2010-02-25, by Christian Urban
merged
2010-02-25, by Christian Urban
moved Nominal to "toplevel"
2010-02-25, by Christian Urban
Export perm_frees.
2010-02-25, by Cezary Kaliszyk
Restructuring the code in Perm
2010-02-24, by Cezary Kaliszyk
Simplified and finised eqvt proofs for t1 and t5
2010-02-24, by Cezary Kaliszyk
merge
2010-02-24, by Cezary Kaliszyk
Define lifted perms.
2010-02-24, by Cezary Kaliszyk
merged
2010-02-24, by Christian Urban
parsing and definition of raw datatype and bv-function work (not very beautiful)
2010-02-24, by Christian Urban
With permute_rsp we can lift the instance proofs :).
2010-02-24, by Cezary Kaliszyk
Note the instance proofs, since they can be easily lifted.
2010-02-24, by Cezary Kaliszyk
More refactoring and removed references to the global simpset in Perm.
2010-02-24, by Cezary Kaliszyk
Factor-out 'prove_perm_empty'; I plan to use it in defining permutations on the lifted type.
2010-02-24, by Cezary Kaliszyk
Regularize finite support proof for trm1
2010-02-24, by Cezary Kaliszyk
Made the fv-supp proof much more straightforward.
2010-02-24, by Cezary Kaliszyk
Regularize the proofs about finite support.
2010-02-24, by Cezary Kaliszyk
Respects of permute and constructors.
2010-02-24, by Cezary Kaliszyk
Generate fv_rsp automatically.
2010-02-24, by Cezary Kaliszyk
Define the constants automatically.
2010-02-24, by Cezary Kaliszyk
Rename also the lifted types to non-capital.
2010-02-24, by Cezary Kaliszyk
Use the infrastructure in LF. Much shorter :).
2010-02-24, by Cezary Kaliszyk
Final synchronization of names.
2010-02-24, by Cezary Kaliszyk
LF renaming part 3 (proper names of alpha equvalences)
2010-02-24, by Cezary Kaliszyk
LF renaming part 2 (proper fv functions)
2010-02-24, by Cezary Kaliszyk
merge
2010-02-24, by Cezary Kaliszyk
LF renaming part1.
2010-02-24, by Cezary Kaliszyk
merged
2010-02-24, by Christian Urban
parsing of function definitions almost works now; still an error with undefined constants
2010-02-24, by Christian Urban
merge
2010-02-23, by Cezary Kaliszyk
rsp for bv; the only issue is that it requires an appropriate induction principle.
2010-02-23, by Cezary Kaliszyk
merged
2010-02-23, by Christian Urban
declarartion of the raw datatype already works; raw binding functions throw an exception about mutual recursive types
2010-02-23, by Christian Urban
rsp infrastructure.
2010-02-23, by Cezary Kaliszyk
merge
2010-02-23, by Cezary Kaliszyk
Progress towards automatic rsp of constants and fv.
2010-02-23, by Cezary Kaliszyk
merged
2010-02-23, by Christian Urban
"raw"-ified the term-constructors and types given in the specification
2010-02-23, by Christian Urban
Looking at proving the rsp rules automatically.
2010-02-23, by Cezary Kaliszyk
Minor beutification.
2010-02-23, by Cezary Kaliszyk
Define the quotient from ML
2010-02-23, by Cezary Kaliszyk
All works in LF but will require renaming.
2010-02-23, by Cezary Kaliszyk
Reordering in LF.
2010-02-23, by Cezary Kaliszyk
Fixes for auxiliary datatypes.
2010-02-23, by Cezary Kaliszyk
Fixed pseudo_injectivity for trm4
2010-02-22, by Cezary Kaliszyk
Testing auto equivp code.
2010-02-22, by Cezary Kaliszyk
A tactic for final equivp
2010-02-22, by Cezary Kaliszyk
More equivp infrastructure.
2010-02-22, by Cezary Kaliszyk
tactify transp
2010-02-22, by Cezary Kaliszyk
export the reflp and symp tacs.
2010-02-22, by Cezary Kaliszyk
Generalize atom_trans and atom_sym.
2010-02-22, by Cezary Kaliszyk
Some progress about transp
2010-02-22, by Cezary Kaliszyk
alpha-symmetric addons.
2010-02-22, by Cezary Kaliszyk
alpha reflexivity
2010-02-22, by Cezary Kaliszyk
Renaming.
2010-02-22, by Cezary Kaliszyk
Added missing description.
2010-02-22, by Cezary Kaliszyk
Added Brian's suggestion.
2010-02-22, by Cezary Kaliszyk
Update TODO
2010-02-22, by Cezary Kaliszyk
Removed bindings 'in itself' where possible.
2010-02-21, by Cezary Kaliszyk
Some adaptation
2010-02-20, by Cezary Kaliszyk
proof cleaning and standardizing.
2010-02-19, by Cezary Kaliszyk
Automatic production and proving of pseudo-injectivity.
2010-02-19, by Cezary Kaliszyk
Experiments for the pseudo-injectivity tactic.
2010-02-19, by Cezary Kaliszyk
merge
2010-02-19, by Cezary Kaliszyk
Constructing alpha_inj goal.
2010-02-19, by Cezary Kaliszyk
merged
2010-02-18, by Christian Urban
start work with the parser
2010-02-18, by Christian Urban
Full alpha equivalence + testing in terms. Some differ but it seems the generated version is more correct.
2010-02-18, by Cezary Kaliszyk
First (non-working) version of alpha-equivalence
2010-02-18, by Cezary Kaliszyk
Description of the fv procedure.
2010-02-18, by Cezary Kaliszyk
Testing auto constant lifting.
2010-02-18, by Cezary Kaliszyk
Fix for new Isabelle (primrec)
2010-02-18, by Cezary Kaliszyk
Automatic lifting of constants.
2010-02-18, by Cezary Kaliszyk
Changed back to original version of trm5
2010-02-18, by Cezary Kaliszyk
The alternate version of trm5 with additional binding. All proofs work the same.
2010-02-18, by Cezary Kaliszyk
Code for handling atom sets.
2010-02-18, by Cezary Kaliszyk
Replace Terms by Terms2.
2010-02-18, by Cezary Kaliszyk
Fixed proofs in Terms2 and found a mistake in Terms.
2010-02-18, by Cezary Kaliszyk
Terms2 with bindings for binders synchronized with bindings they are used in.
2010-02-17, by Cezary Kaliszyk
Cleaning of proofs in Terms.
2010-02-17, by Cezary Kaliszyk
Testing Fv
2010-02-17, by Cezary Kaliszyk
Fix the strong induction principle.
2010-02-17, by Cezary Kaliszyk
Reorder
2010-02-17, by Cezary Kaliszyk
Add bindings of recursive types by free_variables.
2010-02-17, by Cezary Kaliszyk
Bindings adapted to multiple defined datatypes.
2010-02-17, by Cezary Kaliszyk
Reorganization
2010-02-17, by Cezary Kaliszyk
Now should work.
2010-02-17, by Cezary Kaliszyk
Some optimizations and fixes.
2010-02-17, by Cezary Kaliszyk
Simplified format of bindings.
2010-02-17, by Cezary Kaliszyk
Tested the Perm code; works everywhere in Terms.
2010-02-17, by Cezary Kaliszyk
Wrapped the permutation code.
2010-02-17, by Cezary Kaliszyk
Description of intended bindings.
2010-02-17, by Cezary Kaliszyk
Code for generating the fv function, no bindings yet.
2010-02-17, by Cezary Kaliszyk
merge
2010-02-17, by Cezary Kaliszyk
indent
2010-02-17, by Cezary Kaliszyk
merge
2010-02-17, by Cezary Kaliszyk
Simplifying perm_eq
2010-02-17, by Cezary Kaliszyk
merge
2010-02-16, by Cezary Kaliszyk
indenting
2010-02-16, by Cezary Kaliszyk
Minor
2010-02-16, by Cezary Kaliszyk
Merge
2010-02-16, by Cezary Kaliszyk
Ported Stefan's permutation code, still needs some localizing.
2010-02-16, by Cezary Kaliszyk
merge
2010-02-15, by Cezary Kaliszyk
Removed varifyT.
2010-02-15, by Cezary Kaliszyk
merged
2010-02-15, by Christian Urban
2-spaces rule (where it makes sense)
2010-02-15, by Christian Urban
merge
2010-02-15, by Cezary Kaliszyk
Fixed the definition of less and finished the missing proof.
2010-02-15, by Cezary Kaliszyk
further tuning
2010-02-15, by Christian Urban
small tuning
2010-02-15, by Christian Urban
tuned the parsing and testing code in quotient_def.ML; cleaned out old stuff in AbsRepTest.thy
2010-02-15, by Christian Urban
der_bname -> derived_bname
2010-02-15, by Cezary Kaliszyk
Names of files.
2010-02-15, by Cezary Kaliszyk
Finished introducing the binding.
2010-02-15, by Cezary Kaliszyk
Synchronize the commands.
2010-02-15, by Cezary Kaliszyk
Passing the binding to quotient_def
2010-02-15, by Cezary Kaliszyk
Added a binding to the parser.
2010-02-15, by Cezary Kaliszyk
Second inline
2010-02-15, by Cezary Kaliszyk
remove one-line wrapper.
2010-02-15, by Cezary Kaliszyk
Undid the read_terms change; now compiles.
2010-02-12, by Cezary Kaliszyk
merge
2010-02-12, by Cezary Kaliszyk
renamed 'as' to 'is' everywhere.
2010-02-12, by Cezary Kaliszyk
"is" defined as the keyword
2010-02-12, by Cezary Kaliszyk
moved "strange" lemma to quotient_tacs; marked a number of lemmas as unused; tuned
2010-02-12, by Christian Urban
The lattice instantiations are gone from Isabelle/Main, so
2010-02-12, by Cezary Kaliszyk
the lam/bla example.
2010-02-11, by Cezary Kaliszyk
Finished a working foo/bar.
2010-02-11, by Cezary Kaliszyk
fv_foo is not regular.
2010-02-11, by Cezary Kaliszyk
Testing foo/bar
2010-02-11, by Cezary Kaliszyk
Even when bv = fv it still doesn't lift.
2010-02-11, by Cezary Kaliszyk
Added the missing syntax file
2010-02-11, by Cezary Kaliszyk
Notation available locally
2010-02-11, by Cezary Kaliszyk
Main renaming + fixes for new Isabelle in IntEx2.
2010-02-11, by Cezary Kaliszyk
Merging QuotBase into QuotMain.
2010-02-11, by Cezary Kaliszyk
removed dead code
2010-02-10, by Christian Urban
cleaned a bit
2010-02-10, by Christian Urban
lowercase locale
2010-02-10, by Cezary Kaliszyk
hg-added the added file.
2010-02-10, by Cezary Kaliszyk
Changes from Makarius's code review + some noticed fixes.
2010-02-10, by Cezary Kaliszyk
example with a respectful bn function defined over the type itself
2010-02-10, by Cezary Kaliszyk
Finishe the renaming.
2010-02-10, by Cezary Kaliszyk
Another mistake found with OTT.
2010-02-10, by Cezary Kaliszyk
merge
2010-02-10, by Cezary Kaliszyk
Fixed rbv6, when translating to OTT.
2010-02-10, by Cezary Kaliszyk
Some cleaning of proofs.
2010-02-10, by Cezary Kaliszyk
merged again
2010-02-10, by Christian Urban
merged
2010-02-10, by Christian Urban
more minor space and bracket modifications.
2010-02-10, by Cezary Kaliszyk
More changes according to the standards.
2010-02-10, by Cezary Kaliszyk
A concrete example, with a proof that rbv is not regular and
2010-02-10, by Cezary Kaliszyk
proper declaration of types and terms during parsing (removes the varifyT when storing data)
2010-02-09, by Christian Urban
merged
2010-02-09, by Christian Urban
slight correction
2010-02-09, by Christian Urban
merge
2010-02-09, by Cezary Kaliszyk
More about trm6
2010-02-09, by Cezary Kaliszyk
merged
2010-02-09, by Christian Urban
the specifications of the respects.
2010-02-09, by Cezary Kaliszyk
trm6 with the 'Foo' constructor.
2010-02-09, by Cezary Kaliszyk
removing unnecessary brackets
2010-02-09, by Cezary Kaliszyk
More indentation cleaning.
2010-02-09, by Cezary Kaliszyk
'exc' -> 'exn' and more name and space cleaning.
2010-02-09, by Cezary Kaliszyk
Fully qualified exception names.
2010-02-09, by Cezary Kaliszyk
merge
2010-02-09, by Cezary Kaliszyk
More indentation, names and todo cleaning in the quotient package
2010-02-09, by Cezary Kaliszyk
merged
2010-02-09, by Christian Urban
a few more attempts to show the equivalence between old and new way of defining alpha-equivalence
2010-02-09, by Christian Urban
minor tuning
2010-02-09, by Christian Urban
Explicitly marked what is bound.
2010-02-09, by Cezary Kaliszyk
Cleaning and updating in Terms.
2010-02-09, by Cezary Kaliszyk
Looking at the trm2 example
2010-02-09, by Cezary Kaliszyk
Fixed pattern matching, now the test in Abs works correctly.
2010-02-09, by Cezary Kaliszyk
added a test case
2010-02-08, by Christian Urban
merged
2010-02-08, by Christian Urban
moved some lemmas to Nominal; updated all files
2010-02-08, by Christian Urban
merge
2010-02-08, by Cezary Kaliszyk
Comments.
2010-02-08, by Cezary Kaliszyk
slightly tuned
2010-02-08, by Christian Urban
Proper context fixes lifting inside instantiations.
2010-02-08, by Cezary Kaliszyk
Fixed the context import/export and simplified LFex.
2010-02-08, by Cezary Kaliszyk
added 2 papers about core haskell
2010-02-08, by Christian Urban
fixed lemma name
2010-02-07, by Christian Urban
updated to latest Nominal2
2010-02-07, by Christian Urban
minor
2010-02-06, by Christian Urban
some tuning
2010-02-06, by Christian Urban
merge
2010-02-05, by Cezary Kaliszyk
merge
2010-02-05, by Cezary Kaliszyk
Fixes for Bex1 removal.
2010-02-05, by Cezary Kaliszyk
Cleaned Terms using [lifted] and found a workaround for the instantiation problem.
2010-02-05, by Cezary Kaliszyk
A procedure that properly instantiates the types too.
2010-02-05, by Cezary Kaliszyk
More code abstracted away
2010-02-05, by Cezary Kaliszyk
A bit more intelligent and cleaner code.
2010-02-05, by Cezary Kaliszyk
merge
2010-02-05, by Cezary Kaliszyk
A proper version of the attribute
2010-02-05, by Cezary Kaliszyk
merged
2010-02-05, by Christian Urban
eqvts and eqvts_raw are separate thm-lists; otherwise permute_eqvt is problematic as it causes looks in eqvts
2010-02-05, by Christian Urban
The automatic lifting translation function, still with dummy types,
2010-02-04, by Cezary Kaliszyk
Quotdata_dest needed for lifting theorem translation.
2010-02-04, by Cezary Kaliszyk
fixed (permute_eqvt in eqvts makes this simpset always looping)
2010-02-04, by Christian Urban
rollback of the test
2010-02-04, by Christian Urban
linked versions - instead of copies
2010-02-04, by Christian Urban
merged
2010-02-04, by Christian Urban
restored the old behaviour of having an eqvts list; the transformed theorems are stored in eqvts_raw
2010-02-04, by Christian Urban
More let-rec experiments
2010-02-03, by Cezary Kaliszyk
proposal for an alpha equivalence
2010-02-03, by Christian Urban
Lets different.
2010-02-03, by Cezary Kaliszyk
Simplified the proof.
2010-02-03, by Cezary Kaliszyk
merged
2010-02-03, by Christian Urban
proved that bv for lists respects alpha for terms
2010-02-03, by Christian Urban
Finished remains on the let proof.
2010-02-03, by Cezary Kaliszyk
merge
2010-02-03, by Cezary Kaliszyk
Lets are ok.
2010-02-03, by Cezary Kaliszyk
merged
2010-02-03, by Christian Urban
added type-scheme example
2010-02-03, by Christian Urban
merge
2010-02-03, by Cezary Kaliszyk
Definitions for trm5
2010-02-03, by Cezary Kaliszyk
another adaptation for the eqvt-change
2010-02-03, by Christian Urban
merged
2010-02-03, by Christian Urban
fixed proofs that broke because of eqvt
2010-02-03, by Christian Urban
Minor fix.
2010-02-03, by Cezary Kaliszyk
merge
2010-02-03, by Cezary Kaliszyk
alpha5 pseudo-injective
2010-02-03, by Cezary Kaliszyk
less
more
|
(0)
-1920
tip