Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1000
-480
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.
merged
2011-07-11, by Christian Urban
some more experiments with let and bns
2011-07-11, by Christian Urban
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
less
more
|
(0)
-1000
-480
tip