Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1000
-960
+960
+1000
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.
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
fixed proofs in Abs.thy
2010-02-03, by Christian Urban
merged
2010-02-03, by Christian Urban
added a first eqvt_tac which pushes permutations inside terms
2010-02-03, by Christian Urban
The alpha-equivalence relation for let-rec. Not sure if correct...
2010-02-03, by Cezary Kaliszyk
Starting with a let-rec example.
2010-02-03, by Cezary Kaliszyk
Minor
2010-02-03, by Cezary Kaliszyk
Some cleaning and eqvt proof
2010-02-03, by Cezary Kaliszyk
The trm1_support lemma explicitly and stated a strong induction principle.
2010-02-03, by Cezary Kaliszyk
More ingredients in Terms.
2010-02-03, by Cezary Kaliszyk
Finished the supp_fv proof; first proof that analyses the structure of 'Let' :)
2010-02-02, by Cezary Kaliszyk
More in Terms
2010-02-02, by Cezary Kaliszyk
First experiments in Terms.
2010-02-02, by Cezary Kaliszyk
LF ported to alpha_gen, equivp solved and one of the missing proofs in support<-> fv solved. Still some supp properties left.
2010-02-02, by Cezary Kaliszyk
Disambiguating the syntax.
2010-02-02, by Cezary Kaliszyk
Minor uncommited changes from LamEx2.
2010-02-02, by Cezary Kaliszyk
Some equivariance machinery that comes useful in LF.
2010-02-02, by Cezary Kaliszyk
Generalized the eqvt proof for single binders.
2010-02-02, by Cezary Kaliszyk
With induct instead of induct_tac, just one induction is sufficient.
2010-02-02, by Cezary Kaliszyk
General alpha_gen_trans for one-variable abstraction.
2010-02-02, by Cezary Kaliszyk
With unfolding Rep/Abs_eqvt no longer needed.
2010-02-02, by Cezary Kaliszyk
Lam2 finished apart from Rep_eqvt.
2010-02-02, by Cezary Kaliszyk
merge
2010-02-01, by Cezary Kaliszyk
All should be ok now.
2010-02-01, by Cezary Kaliszyk
repaired according to changes in Abs.thy
2010-02-01, by Christian Urban
added a single-binder alpha equivalence; showed one half of the equivalence proof between general and single binder case
2010-02-01, by Christian Urban
cleaned
2010-02-01, by Christian Urban
updated from huffman
2010-02-01, by Christian Urban
updated from nominal-huffman
2010-02-01, by Christian Urban
Fixed wrong rename.
2010-02-01, by Cezary Kaliszyk
merge
2010-02-01, by Cezary Kaliszyk
Lambda based on alpha_gen, under construction.
2010-02-01, by Cezary Kaliszyk
updated from huffman - repo
2010-02-01, by Christian Urban
renamed Abst/abst to Abs/abs
2010-02-01, by Christian Urban
got rid of RAbst type - is now just pairs
2010-02-01, by Christian Urban
Monotonicity of ~~gen, needed for using it in inductive definitions.
2010-02-01, by Cezary Kaliszyk
The current state of fv vs supp proofs in LF.
2010-02-01, by Cezary Kaliszyk
merge
2010-02-01, by Cezary Kaliszyk
More proofs in the LF example.
2010-02-01, by Cezary Kaliszyk
merged
2010-02-01, by Christian Urban
slight tuning
2010-02-01, by Christian Urban
renamed function according to the name of the constant
2010-02-01, by Christian Urban
fixed problem with Bex1_rel renaming
2010-02-01, by Christian Urban
Ported LF to the generic lambda and solved the simpler _supp cases.
2010-02-01, by Cezary Kaliszyk
merged
2010-01-30, by Christian Urban
introduced a generic alpha (but not sure whether it is helpful)
2010-01-30, by Christian Urban
More in the LF example in the new nominal way, all is clear until support.
2010-01-29, by Cezary Kaliszyk
Fixed the induction problem + some more proofs.
2010-01-29, by Cezary Kaliszyk
equivariance of rfv and alpha.
2010-01-29, by Cezary Kaliszyk
Added the experiments with fun and function.
2010-01-29, by Cezary Kaliszyk
now also final step is proved - the supp of lambdas is now completely characterised
2010-01-29, by Christian Urban
the supp of a lambda can now be characterised, *provided* the notion of free variables coincides with support on lambda terms
2010-01-29, by Christian Urban
improved the proof slightly by defining alpha as a function and completely characterised the equality between two abstractions
2010-01-28, by Christian Urban
merged
2010-01-28, by Christian Urban
general abstraction operator and complete characterisation of its support and freshness
2010-01-28, by Christian Urban
Ported existing part of LF to new permutations and alphas.
2010-01-28, by Cezary Kaliszyk
attempt of a general abstraction operator
2010-01-28, by Christian Urban
attempt to prove equivalence between alpha definitions
2010-01-28, by Christian Urban
End of renaming.
2010-01-28, by Cezary Kaliszyk
Minor when looking at lam.distinct and lam.inject
2010-01-28, by Cezary Kaliszyk
Renamed Bexeq to Bex1_rel
2010-01-28, by Cezary Kaliszyk
Substracting bounds from free variables.
2010-01-28, by Cezary Kaliszyk
Improper interface for datatype and function packages and proper interface lateron.
2010-01-28, by Cezary Kaliszyk
merged
2010-01-28, by Christian Urban
minor
2010-01-28, by Christian Urban
test about supp/freshness for lam (old proofs work in principle - for single binders)
2010-01-28, by Christian Urban
Recommited the changes for nitpick
2010-01-28, by Cezary Kaliszyk
Correct types which fixes the printing.
2010-01-27, by Cezary Kaliszyk
fv for subterms
2010-01-27, by Cezary Kaliszyk
Fix the problem with later examples. Maybe need to go back to textual specifications.
2010-01-27, by Cezary Kaliszyk
Some processing of variables in constructors to get free variables.
2010-01-27, by Cezary Kaliszyk
Parsing of the input as terms and types, and passing them as such to the function package.
2010-01-27, by Cezary Kaliszyk
Undid the parsing, as it is not possible with thy->lthy interaction.
2010-01-27, by Cezary Kaliszyk
merge
2010-01-27, by Cezary Kaliszyk
Some cleaning of thy vs lthy vs context.
2010-01-27, by Cezary Kaliszyk
merged
2010-01-27, by Christian Urban
tuned comment
2010-01-27, by Christian Urban
completely ported
2010-01-27, by Christian Urban
Another string in the specification.
2010-01-27, by Cezary Kaliszyk
Variable takes a 'name'.
2010-01-27, by Cezary Kaliszyk
merge
2010-01-27, by Cezary Kaliszyk
When commenting discovered a missing case of Babs->Abs regularization.
2010-01-27, by Cezary Kaliszyk
merged
2010-01-27, by Christian Urban
mostly ported Terms.thy to new Nominal
2010-01-27, by Christian Urban
merge
2010-01-27, by Cezary Kaliszyk
Commenting regularize
2010-01-27, by Cezary Kaliszyk
very rough example file for how nominal2 specification can be parsed
2010-01-27, by Christian Urban
reordered cases in regularize (will be merged into two cases)
2010-01-27, by Christian Urban
use of equiv_relation_chk in quotient_term
2010-01-27, by Christian Urban
some slight tuning
2010-01-27, by Christian Urban
added Terms to Nominal - Instantiation of two types does not work (ask Florian)
2010-01-27, by Christian Urban
added another example with indirect recursion over lists
2010-01-27, by Christian Urban
just moved obsolete material into Attic
2010-01-26, by Christian Urban
added an LamEx example together with the new nominal infrastructure
2010-01-26, by Christian Urban
Bex1_Bexeq_regular.
2010-01-26, by Cezary Kaliszyk
Hom Theorem with exists unique
2010-01-26, by Cezary Kaliszyk
2 cases for regularize with split, lemmas with split now lift.
2010-01-26, by Cezary Kaliszyk
Simpler statement that has the problem.
2010-01-26, by Cezary Kaliszyk
Found a term that does not regularize.
2010-01-26, by Cezary Kaliszyk
A triple is still ok.
2010-01-26, by Cezary Kaliszyk
Combined the simpsets in clean_tac and updated the comment. Now cleaning of splits does work.
2010-01-26, by Cezary Kaliszyk
Changed the lambda_prs_simple_conv to use id_apply, now last eq_reflection can be removed from id_simps.
2010-01-26, by Cezary Kaliszyk
Sigma cleaning works with split_prs (still manual proof).
2010-01-26, by Cezary Kaliszyk
tuned
2010-01-26, by Christian Urban
merged
2010-01-26, by Christian Urban
cleaning of QuotProd; a little cleaning of QuotList
2010-01-26, by Christian Urban
added prs and rsp lemmas for Inl and Inr
2010-01-26, by Christian Urban
used split_option_all lemma
2010-01-26, by Christian Urban
used the internal Option.map instead of custom option_map
2010-01-26, by Christian Urban
Generalized split_prs and split_rsp
2010-01-26, by Cezary Kaliszyk
All eq_reflections apart from the one of 'id_apply' can be removed.
2010-01-26, by Cezary Kaliszyk
continued
2010-01-26, by Cezary Kaliszyk
More eqreflection/equiv cleaning.
2010-01-26, by Cezary Kaliszyk
more eq_reflection & other cleaning.
2010-01-26, by Cezary Kaliszyk
Removing more eq_reflections.
2010-01-26, by Cezary Kaliszyk
ids *cannot* be object equalities
2010-01-25, by Christian Urban
re-inserted lemma in QuotList
2010-01-25, by Christian Urban
added prs and rsp lemmas for Some and None
2010-01-25, by Christian Urban
tuned proofs (mainly in QuotProd)
2010-01-25, by Christian Urban
properly commented out the "unused lemmas section" and moved actually used lemmas elsewhere; added two minor items to the TODO list
2010-01-25, by Christian Urban
renamed QuotScript to QuotBase
2010-01-25, by Christian Urban
cleaned some theorems
2010-01-25, by Christian Urban
test with splits
2010-01-24, by Christian Urban
The alpha equivalence relations for structures in 'Terms'
2010-01-23, by Cezary Kaliszyk
More experiments with defining the homomorphism directly, lifting of 'distinct' and of 'exhaust'.
2010-01-23, by Cezary Kaliszyk
Trying to define hom for the lifted type directly.
2010-01-23, by Cezary Kaliszyk
Proper alpha equivalence for Sigma calculus.
2010-01-22, by Cezary Kaliszyk
Changed fun_map and rel_map to definitions.
2010-01-21, by Cezary Kaliszyk
Lifted Peter's Sigma lemma with Ex1.
2010-01-21, by Cezary Kaliszyk
Automatic injection of Bexeq
2010-01-21, by Cezary Kaliszyk
Automatic cleaning of Bexeq<->Ex1 theorems.
2010-01-21, by Cezary Kaliszyk
Using Bexeq_rsp, and manually lifted lemma with Ex1.
2010-01-21, by Cezary Kaliszyk
Bexeq definition, Ex1_prs lemma, Bex1_rsp lemma, compiles.
2010-01-21, by Cezary Kaliszyk
The missing rule.
2010-01-21, by Cezary Kaliszyk
Ex1 -> Bex1 Regularization, Preparing Exeq.
2010-01-21, by Cezary Kaliszyk
Added the Sigma Calculus example
2010-01-20, by Cezary Kaliszyk
Better error messages for non matching quantifiers.
2010-01-20, by Cezary Kaliszyk
Statement of term1_hom_rsp
2010-01-20, by Cezary Kaliszyk
proved that the function is a function
2010-01-20, by Christian Urban
term1_hom as a function
2010-01-20, by Cezary Kaliszyk
A version of hom with quantifiers.
2010-01-19, by Cezary Kaliszyk
added permutation functions for the raw calculi
2010-01-17, by Christian Urban
fixed broken (partial) proof
2010-01-16, by Christian Urban
used "new" alpha-equivalence relation (according to new scheme); proved equivalence theorems and so on
2010-01-16, by Christian Urban
liftin and lifing_tac can now lift several "and"-separated goals at once; the raw-theorems have to be given in the order of goals
2010-01-16, by Christian Urban
added a partial proof under which conditions rlam_rec Respects alpha...I guess something like this is true; this means the Hom lemmas need to have preconditions
2010-01-15, by Christian Urban
tried to witness the hom-lemma with the recursion combinator from rlam....does not work yet completely
2010-01-15, by Christian Urban
merged
2010-01-15, by Christian Urban
added free_variable function (do not know about the algorithm yet)
2010-01-15, by Christian Urban
hom lifted to hom', so it is true. Infrastructure for partially regularized quantifiers. Nicer errors for regularize.
2010-01-15, by Cezary Kaliszyk
slight tuning of relation_error
2010-01-15, by Christian Urban
Appropriate respects and a statement of the lifted hom lemma
2010-01-15, by Cezary Kaliszyk
recursion-hom for lambda
2010-01-15, by Christian Urban
Incorrect version of the homomorphism lemma
2010-01-15, by Cezary Kaliszyk
trivial
2010-01-14, by Christian Urban
tuned quotient_typ.ML
2010-01-14, by Christian Urban
tuned quotient_def.ML and cleaned somewhat LamEx.thy
2010-01-14, by Christian Urban
a few more lemmas...except supp of lambda-abstractions
2010-01-14, by Christian Urban
removed one sorry
2010-01-14, by Christian Urban
nearly all of the proof
2010-01-14, by Christian Urban
right generalisation
2010-01-14, by Christian Urban
First subgoal.
2010-01-14, by Cezary Kaliszyk
setup for strong induction
2010-01-14, by Christian Urban
exported absrep_const for nitpick.
2010-01-14, by Cezary Kaliszyk
minor
2010-01-14, by Cezary Kaliszyk
Simplified matches_typ.
2010-01-14, by Cezary Kaliszyk
added bound-variable functions to terms
2010-01-14, by Christian Urban
merged
2010-01-14, by Christian Urban
added 3 calculi with interesting binding structure
2010-01-14, by Christian Urban
produce defs with lthy, like prs and ids
2010-01-14, by Cezary Kaliszyk
Remove SOLVED from quotient_tac. Move atomize_eqv to 'Unused'.
2010-01-14, by Cezary Kaliszyk
Finished organising an efficient datastructure for qconst_info.
2010-01-14, by Cezary Kaliszyk
Undid changes from symtab to termtab, since we need to lookup specialized types.
2010-01-14, by Cezary Kaliszyk
Moved the matches_typ function outside a?d simplified it.
2010-01-13, by Cezary Kaliszyk
one more item in the list of Markus
2010-01-13, by Christian Urban
Put relation_error as a separate function.
2010-01-13, by Cezary Kaliszyk
Better error message for definition failure.
2010-01-13, by Cezary Kaliszyk
merge
2010-01-13, by Cezary Kaliszyk
Stored Termtab for constant information.
2010-01-13, by Cezary Kaliszyk
merged
2010-01-13, by Christian Urban
deleted SOLVED'
2010-01-13, by Christian Urban
Removed the 'oops' in IntEx.
2010-01-13, by Cezary Kaliszyk
tuned
2010-01-13, by Christian Urban
added SOLVED' which is now part of Isabelle....must be removed eventually
2010-01-13, by Christian Urban
merged
2010-01-13, by Christian Urban
tuned
2010-01-13, by Christian Urban
absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
2010-01-13, by Christian Urban
More indenting, bracket removing and comment restructuring.
2010-01-12, by Cezary Kaliszyk
Finished replacing OO by OOO
2010-01-12, by Cezary Kaliszyk
Change OO to OOO in FSet3.
2010-01-12, by Cezary Kaliszyk
minor comment editing
2010-01-12, by Cezary Kaliszyk
modifying comments/indentation in quotient_term.ml
2010-01-12, by Cezary Kaliszyk
Cleaning comments, indentation etc in quotient_tacs.
2010-01-12, by Cezary Kaliszyk
No more exception handling in rep_abs_rsp_tac
2010-01-12, by Cezary Kaliszyk
handle all is no longer necessary in lambda_prs.
2010-01-12, by Cezary Kaliszyk
removed 3 hacks.
2010-01-12, by Cezary Kaliszyk
Updated some comments.
2010-01-12, by Cezary Kaliszyk
merge
2010-01-12, by Cezary Kaliszyk
Removed exception handling from equals_rsp_tac.
2010-01-12, by Cezary Kaliszyk
added an abbreviation for OOO
2010-01-11, by Christian Urban
merge
2010-01-11, by Cezary Kaliszyk
Undid the non-working part.
2010-01-11, by Cezary Kaliszyk
started to adhere to Wenzel-Standard
2010-01-11, by Christian Urban
Changing exceptions to 'try', part 1.
2010-01-11, by Cezary Kaliszyk
removed quotdata_lookup_type
2010-01-11, by Cezary Kaliszyk
Fix for testing matching constants in regularize.
2010-01-11, by Cezary Kaliszyk
tuned previous commit further
2010-01-11, by Christian Urban
the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
2010-01-11, by Christian Urban
introduced separate match function
2010-01-09, by Christian Urban
removed obsolete equiv_relation and rnamed new_equiv_relation
2010-01-09, by Christian Urban
New_relations, all works again including concat examples.
2010-01-08, by Cezary Kaliszyk
map and rel simps for all quotients; needed when changing the relations to aggregate ones.
2010-01-08, by Cezary Kaliszyk
id_simps needs to be taken out not used directly, otherwise the new lemmas are not there.
2010-01-08, by Cezary Kaliszyk
Experimients with fconcat_insert
2010-01-08, by Cezary Kaliszyk
Modifications for new_equiv_rel, part2
2010-01-08, by Cezary Kaliszyk
Modifictaions for new_relation.
2010-01-08, by Cezary Kaliszyk
Proved concat_empty.
2010-01-08, by Cezary Kaliszyk
Replacing equivp by reflp in the assumptions leads to non-provable subgoals in the gen_pre lemmas.
2010-01-07, by Cezary Kaliszyk
some cleaning.
2010-01-07, by Cezary Kaliszyk
First generalization.
2010-01-07, by Cezary Kaliszyk
The working proof of the special case.
2010-01-07, by Cezary Kaliszyk
Reduced the proof to two simple but not obvious to prove facts.
2010-01-07, by Cezary Kaliszyk
More cleaning and commenting AbsRepTest. Now tests work; just slow.
2010-01-07, by Cezary Kaliszyk
cleaning in AbsRepTest.
2010-01-07, by Cezary Kaliszyk
Further in the proof
2010-01-06, by Cezary Kaliszyk
Tried to prove the lemma manually; only left with quotient proofs.
2010-01-06, by Cezary Kaliszyk
Sledgehammer bug.
2010-01-06, by Cezary Kaliszyk
merge
2010-01-05, by Cezary Kaliszyk
Trying the proof
2010-01-05, by Cezary Kaliszyk
merged
2010-01-05, by Christian Urban
Struggling with composition
2010-01-05, by Cezary Kaliszyk
Trying to state composition quotient.
2010-01-05, by Cezary Kaliszyk
proper handling of error messages (code copy - maybe this can be avoided)
2010-01-05, by Christian Urban
added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
2010-01-05, by Christian Urban
Readded 'regularize_to_injection' which I believe will be needed.
2010-01-05, by Cezary Kaliszyk
added a warning to the quotient_type definition, if a map function is missing
2010-01-02, by Christian Urban
tuned
2010-01-01, by Christian Urban
a slight change to abs/rep generation
2010-01-01, by Christian Urban
tuned
2010-01-01, by Christian Urban
fixed comment errors
2010-01-01, by Christian Urban
some slight tuning
2010-01-01, by Christian Urban
renamed transfer to transform (Markus)
2009-12-31, by Christian Urban
some small changes
2009-12-30, by cu
added a functor that allows checking what is added to the theorem lists
2009-12-27, by Christian Urban
corrected wrong [quot_respect] attribute; tuned
2009-12-26, by Christian Urban
renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
2009-12-26, by Christian Urban
added an item about when the same quotient constant is defined twice (throws a bind exception in quoteint_def.ML)
2009-12-26, by Christian Urban
as expected problems occure when lifting concat lemmas
2009-12-26, by Christian Urban
tuned
2009-12-26, by Christian Urban
commeted the absrep function
2009-12-26, by Christian Urban
generalised absrep function; needs consolidation
2009-12-26, by Christian Urban
tuned
2009-12-25, by Christian Urban
added sanity checks for quotient_type
2009-12-25, by Christian Urban
made the quotient_type definition more like typedef; now type variables need to be explicitly given
2009-12-24, by Christian Urban
used Local_Theory.declaration for storing quotdata
2009-12-24, by Christian Urban
tuning
2009-12-23, by Christian Urban
renamed some fields in the info records
2009-12-23, by Christian Urban
modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
2009-12-23, by Christian Urban
cleaed a bit function mk_typedef_main
2009-12-23, by Christian Urban
renamed QUOT_TYPE to Quot_Type
2009-12-23, by Christian Urban
explicit handling of mem_def, avoiding the use of the simplifier; this fixes some quotient_type definitions
2009-12-23, by Christian Urban
corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
2009-12-23, by Christian Urban
added "Highest Priority" category; and tuned slightly code
2009-12-22, by Christian Urban
added a print_maps command; updated the keyword file accordingly
2009-12-22, by Christian Urban
renamed get_fun to absrep_fun; introduced explicit checked versions of the term functions
2009-12-22, by Christian Urban
tuned
2009-12-22, by Christian Urban
moved get_fun into quotient_term; this simplifies the overall including structure of the package
2009-12-22, by Christian Urban
tuned comments; renamed QUOT_TRUE to Quot_True; atomize_eqv seems to not be neccessary (has it been added to Isabelle)...it is now comented out and everything still works
2009-12-22, by Christian Urban
on the hunt for what condition raises which exception in the CLEVER CODE of calculate_inst
2009-12-22, by Christian Urban
simplified calculate_instance; worked around some clever code; clever code is unfortunately still there...needs to be removed
2009-12-22, by Christian Urban
used eq_reflection not with OF, but directly in @{thm ...}
2009-12-21, by Christian Urban
cleaned a bit calculate_inst a bit; eta-contraction seems to be not necessary? (all examples go through)
2009-12-21, by Christian Urban
get_fun needed change to cope with "('a fset) fset" types...this needs composition (op o); now id_simps contains also id_o and o_id, and map_id is also added in QuotList.thy; regularize and cleaning needed to be hacked (indicated by "HACK")...THIS NEEDS ATTENTION!!!; except two lemmas in IntEx, all examples go through; added considerable material to FSet3; tuned FIXME-TODO
2009-12-21, by Christian Urban
on suggestion of Tobias renamed "quotient_def" to "quotient_definition"; needs new keyword file
2009-12-20, by Christian Urban
renamed "quotient" command to "quotient_type"; needs new keyword file to be installed
2009-12-20, by Christian Urban
this file is now obsolete; replaced by isar-keywords-quot.el
2009-12-20, by Christian Urban
with "isabelle make keywords" you can create automatically a "quot" keywordfile, provided all Logics are in place
2009-12-20, by Christian Urban
added a very old paper about Quotients in Isabelle (related work)
2009-12-19, by Christian Urban
avoided global "open"s - replaced by local "open"s
2009-12-19, by Christian Urban
small tuning
2009-12-19, by Christian Urban
various tunings; map_lookup now raises an exception; addition to FIXME-TODO
2009-12-19, by Christian Urban
minor cleaning
2009-12-17, by Christian Urban
moved the QuotMain code into two ML-files
2009-12-17, by Christian Urban
complete fix for IsaMakefile
2009-12-16, by Christian Urban
first fix
2009-12-16, by Christian Urban
merged
2009-12-16, by Christian Urban
added a paper for possible notes
2009-12-16, by Christian Urban
Removed lambdas on the right hand side. This fixes all 'PROBLEM' comments.
2009-12-16, by Cezary Kaliszyk
lambda_prs & solve_quotient_assum cleaned.
2009-12-15, by Cezary Kaliszyk
some commenting
2009-12-15, by Christian Urban
Fixed previous commit.
2009-12-14, by Cezary Kaliszyk
merge
2009-12-14, by Cezary Kaliszyk
Moved DETERM inside Repeat & added SOLVE around quotient_tac.
2009-12-14, by Cezary Kaliszyk
merge.
2009-12-14, by Cezary Kaliszyk
FIXME/TODO.
2009-12-14, by Cezary Kaliszyk
reply to question in code
2009-12-14, by Cezary Kaliszyk
Reply in code.
2009-12-14, by Cezary Kaliszyk
Replies to questions from the weekend: Uncommenting the renamed theorem commented out in 734.
2009-12-14, by Cezary Kaliszyk
a few code annotations
2009-12-13, by Christian Urban
another pass on apply_rsp
2009-12-13, by Christian Urban
managed to simplify apply_rsp
2009-12-13, by Christian Urban
tried to simplify apply_rsp_tac; failed at the moment; added some questions
2009-12-12, by Christian Urban
some trivial changes
2009-12-12, by Christian Urban
trivial cleaning of make_inst
2009-12-12, by Christian Urban
tried to improve test; but fails
2009-12-12, by Christian Urban
merged
2009-12-12, by Christian Urban
annotated some questions to the code; some simple changes
2009-12-12, by Christian Urban
Answering the question in code.
2009-12-12, by Cezary Kaliszyk
merged
2009-12-12, by Christian Urban
trivial
2009-12-12, by Christian Urban
tuned code
2009-12-12, by Christian Urban
Minor
2009-12-12, by Cezary Kaliszyk
Some proofs.
2009-12-12, by Cezary Kaliszyk
Proof of finite_set_storng_cases_raw.
2009-12-12, by Cezary Kaliszyk
A bracket was missing; with it proved the 'definitely false' lemma.
2009-12-12, by Cezary Kaliszyk
renamed quotient.ML to quotient_typ.ML
2009-12-12, by Christian Urban
merged
2009-12-11, by Christian Urban
tuned
2009-12-11, by Christian Urban
started to have a look at it; redefined the relation
2009-12-11, by Christian Urban
More name and indentation cleaning.
2009-12-11, by Cezary Kaliszyk
Merge + Added LarryInt & Fset3 to tests.
2009-12-11, by Cezary Kaliszyk
Renaming
2009-12-11, by Cezary Kaliszyk
merged
2009-12-11, by Christian Urban
deleted struct_match by Pattern.match (fixes a problem in LarryInt)
2009-12-11, by Christian Urban
FSet3 minor fixes + cases
2009-12-11, by Cezary Kaliszyk
added Int example from Larry
2009-12-11, by Christian Urban
Added FSet3 with a formalisation of finite sets based on Michael's one.
2009-12-11, by Cezary Kaliszyk
Updated TODO list together.
2009-12-11, by Cezary Kaliszyk
Merge
2009-12-11, by Cezary Kaliszyk
More theorem renaming.
2009-12-11, by Cezary Kaliszyk
Renamed theorems in IntEx2 to conform to names in Int.
2009-12-11, by Cezary Kaliszyk
Updated comments.
2009-12-11, by Cezary Kaliszyk
merged
2009-12-11, by Christian Urban
tuned
2009-12-11, by Christian Urban
renamed Larrys example
2009-12-11, by Christian Urban
New syntax for definitions.
2009-12-11, by Cezary Kaliszyk
changed error message
2009-12-11, by Christian Urban
reformulated the lemma lifting_procedure as ML value; gave better warning message for injection case
2009-12-11, by Christian Urban
slightly tuned
2009-12-10, by Christian Urban
merged
2009-12-10, by Christian Urban
added Larry's theory; introduced lemma equivpI; added something to the TODO about error messages
2009-12-10, by Christian Urban
added maps-printout and tuned some comments
2009-12-10, by Christian Urban
Option and Sum quotients.
2009-12-10, by Cezary Kaliszyk
Regularized the hard lemma.
2009-12-10, by Cezary Kaliszyk
Simplification of Babses for regularize; will probably become injection
2009-12-10, by Cezary Kaliszyk
Found the problem with ttt3.
2009-12-10, by Cezary Kaliszyk
minor
2009-12-10, by Cezary Kaliszyk
Moved Unused part of locale to Unused QuotMain.
2009-12-10, by Cezary Kaliszyk
Moved 'int_induct' to IntEx to keep IntEx2 being just theory of integers in order.
2009-12-10, by Cezary Kaliszyk
Removed 'Presburger' as it introduces int & other minor cleaning in Int2.
2009-12-10, by Cezary Kaliszyk
more tuning
2009-12-10, by Christian Urban
tuned
2009-12-10, by Christian Urban
simplified the instantiation of QUOT_TRUE in procedure_tac
2009-12-10, by Christian Urban
completed previous commit
2009-12-10, by Christian Urban
deleted DT/NDT diagnostic code
2009-12-10, by Christian Urban
moved the interpretation code into Unused.thy
2009-12-10, by Christian Urban
added an attempt to get a finite set theory
2009-12-10, by Christian Urban
removed memb and used standard mem (member from List.thy)
2009-12-10, by Christian Urban
merged
2009-12-10, by Christian Urban
simplified proofs
2009-12-10, by Christian Urban
removed quot_respect attribute of a non-standard lemma
2009-12-10, by Christian Urban
With int_of_nat as a quotient_def, lemmas about it can be easily lifted.
2009-12-10, by Cezary Kaliszyk
merged
2009-12-10, by Christian Urban
naming in this file cannot be made to agree to the original (PROBLEM?)
2009-12-10, by Christian Urban
Lifted some kind of induction.
2009-12-10, by Cezary Kaliszyk
more proofs in IntEx2
2009-12-09, by Christian Urban
Finished one proof in IntEx2.
2009-12-09, by Cezary Kaliszyk
slightly more on IntEx2
2009-12-09, by Christian Urban
proved (with a lot of pain) that times_raw is respectful
2009-12-09, by Christian Urban
merged
2009-12-09, by Christian Urban
fixed minor stupidity
2009-12-09, by Christian Urban
Exception handling.
2009-12-09, by Cezary Kaliszyk
Code cleaning.
2009-12-09, by Cezary Kaliszyk
merge
2009-12-09, by Cezary Kaliszyk
foldr_rsp.
2009-12-09, by Cezary Kaliszyk
tuned
2009-12-09, by Christian Urban
merge
2009-12-09, by Cezary Kaliszyk
Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants.
2009-12-09, by Cezary Kaliszyk
deleted make_inst3
2009-12-09, by Christian Urban
tuned
2009-12-09, by Christian Urban
tuned
2009-12-09, by Christian Urban
moved function and tuned comment
2009-12-09, by Christian Urban
improved fun_map_conv
2009-12-09, by Christian Urban
Arbitrary number of fun_map_tacs.
2009-12-09, by Cezary Kaliszyk
Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work.
2009-12-09, by Cezary Kaliszyk
tuned code
2009-12-09, by Christian Urban
tuned the examples and flagged the problematic cleaning lemmas in FSet
2009-12-09, by Christian Urban
merged
2009-12-08, by Christian Urban
implemented cleaning strategy with fun_map.simps on non-bounded variables; still a few rough edges
2009-12-08, by Christian Urban
merge
2009-12-08, by Cezary Kaliszyk
manually cleaned the hard lemma.
2009-12-08, by Cezary Kaliszyk
merged
2009-12-08, by Christian Urban
decoupled QuotProd from QuotMain and also started new cleaning strategy
2009-12-08, by Christian Urban
merge
2009-12-08, by Cezary Kaliszyk
An example which is hard to lift because of the interplay between lambda_prs and unfolding.
2009-12-08, by Cezary Kaliszyk
proper formulation of all preservation theorems
2009-12-08, by Christian Urban
started to reformulate preserve lemmas
2009-12-08, by Christian Urban
properly set up the prs_rules
2009-12-08, by Christian Urban
merged
2009-12-08, by Christian Urban
added preserve rules to the cleaning_tac
2009-12-08, by Christian Urban
merge
2009-12-08, by Cezary Kaliszyk
cleaning.
2009-12-08, by Cezary Kaliszyk
merged
2009-12-08, by Christian Urban
chnaged syntax to "lifting theorem"
2009-12-08, by Christian Urban
changed names of attributes
2009-12-08, by Christian Urban
merge
2009-12-08, by Cezary Kaliszyk
Manual regularization of a goal in FSet.
2009-12-08, by Cezary Kaliszyk
merged
2009-12-08, by Christian Urban
added methods for the lifting_tac and the other tacs
2009-12-08, by Christian Urban
make_inst3
2009-12-08, by Cezary Kaliszyk
Merge
2009-12-08, by Cezary Kaliszyk
trans2 replaced with equals_rsp_tac
2009-12-08, by Cezary Kaliszyk
corrected name of FSet in ROOT.ML
2009-12-08, by Christian Urban
Made fset work again to test all.
2009-12-08, by Cezary Kaliszyk
Finished the proof of ttt2 and found bug in regularize when trying ttt3.
2009-12-08, by Cezary Kaliszyk
Another lambda example theorem proved. Seems it starts working properly.
2009-12-08, by Cezary Kaliszyk
Removed pattern from quot_rel_rsp, since list_rel and all used introduced ones cannot be patterned
2009-12-08, by Cezary Kaliszyk
Proper checked map_rsp.
2009-12-08, by Cezary Kaliszyk
Nitpick found a counterexample for one lemma.
2009-12-08, by Cezary Kaliszyk
Added a 'rep_abs' in inj_repabs_trm of babs; and proved two lam examples.
2009-12-08, by Cezary Kaliszyk
It also regularizes.
2009-12-08, by Cezary Kaliszyk
inj_repabs also works.
2009-12-08, by Cezary Kaliszyk
merge
2009-12-08, by Cezary Kaliszyk
An example of working cleaning for lambda lifting. Still not sure why Babs helps.
2009-12-08, by Cezary Kaliszyk
tuned
2009-12-08, by Christian Urban
the lift_tac produces a warning message if one of the three automatic proofs fails
2009-12-08, by Christian Urban
added a thm list for ids
2009-12-08, by Christian Urban
removed a fixme: map_info is now checked
2009-12-08, by Christian Urban
tuning of the code
2009-12-07, by Christian Urban
merged
2009-12-07, by Christian Urban
removed "global" data and lookup functions; had to move a tactic out from the inj_repabs_match tactic since apply_rsp interferes with a trans2 rule for ===>
2009-12-07, by Christian Urban
3 lambda examples in FSet. In the last one regularize_term fails.
2009-12-07, by Cezary Kaliszyk
Handling of errors in lambda_prs_conv.
2009-12-07, by Cezary Kaliszyk
babs_prs
2009-12-07, by Cezary Kaliszyk
clarified the function examples
2009-12-07, by Christian Urban
first attempt to deal with Babs in regularise and cleaning (not yet working)
2009-12-07, by Christian Urban
isabelle make tests all examples
2009-12-07, by Christian Urban
merge
2009-12-07, by Cezary Kaliszyk
make_inst for lambda_prs where the second quotient is not identity.
2009-12-07, by Cezary Kaliszyk
added "end" to each example theory
2009-12-07, by Christian Urban
List moved after QuotMain
2009-12-07, by Cezary Kaliszyk
cleaning
2009-12-07, by Christian Urban
final move
2009-12-07, by Christian Urban
directory re-arrangement
2009-12-07, by Christian Urban
inj_repabs_tac handles Babs now.
2009-12-07, by Cezary Kaliszyk
Fix of regularize for babs and proof of babs_rsp.
2009-12-07, by Cezary Kaliszyk
Using pair_prs; debugging the error in regularize of a lambda.
2009-12-07, by Cezary Kaliszyk
QuotProd with product_quotient and a 3 respects and preserves lemmas.
2009-12-07, by Cezary Kaliszyk
merge
2009-12-07, by Cezary Kaliszyk
3 new example thms in MyInt; reveal problems with handling of lambdas; regularize fails with "Loose Bound".
2009-12-07, by Cezary Kaliszyk
simplified the regularize simproc
2009-12-07, by Christian Urban
now simpler regularize_tac with added solver works
2009-12-07, by Christian Urban
removed usage of HOL_basic_ss by using a slighly extended version of empty_ss
2009-12-07, by Christian Urban
merged
2009-12-07, by Christian Urban
fixed examples
2009-12-07, by Christian Urban
Fix IntEx2 for equiv_list
2009-12-07, by Cezary Kaliszyk
merged
2009-12-06, by Christian Urban
working state again
2009-12-06, by Christian Urban
added a theorem list for equivalence theorems
2009-12-06, by Christian Urban
Merge
2009-12-06, by Cezary Kaliszyk
Name changes.
2009-12-06, by Cezary Kaliszyk
Solved all quotient goals.
2009-12-06, by Cezary Kaliszyk
updated Isabelle and deleted mono rules
2009-12-06, by Christian Urban
more tuning of the code
2009-12-06, by Christian Urban
puting code in separate sections
2009-12-06, by Christian Urban
Handle 'find_qt_asm' exception. Now all inj_repabs_goals should be solved automatically.
2009-12-06, by Cezary Kaliszyk
merge
2009-12-06, by Cezary Kaliszyk
Simpler definition code that works with any type maps.
2009-12-06, by Cezary Kaliszyk
working on lambda_prs with examples; polished code of clean_tac
2009-12-06, by Christian Urban
renamed lambda_allex_prs
2009-12-06, by Christian Urban
added more to IntEx2
2009-12-06, by Christian Urban
merged
2009-12-06, by Christian Urban
added new example for Ints; regularise does not work in all instances
2009-12-06, by Christian Urban
Definitions folded first.
2009-12-06, by Cezary Kaliszyk
Used symmetric definitions. Moved quotient_rsp to QuotMain.
2009-12-05, by Cezary Kaliszyk
Proved foldl_rsp and ho_map_rsp
2009-12-05, by Cezary Kaliszyk
moved all_prs and ex_prs out from the conversion into the simplifier
2009-12-05, by Christian Urban
further cleaning
2009-12-05, by Christian Urban
Merge
2009-12-05, by Cezary Kaliszyk
Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx.
2009-12-05, by Cezary Kaliszyk
simplified inj_repabs_trm
2009-12-05, by Christian Urban
merged
2009-12-05, by Christian Urban
merged
2009-12-05, by Christian Urban
merged
2009-12-05, by Christian Urban
simpler version of clean_tac
2009-12-05, by Christian Urban
Handling of respects in the fast inj_repabs_tac; includes respects with quotient assumptions.
2009-12-05, by Cezary Kaliszyk
Solutions to IntEx tests.
2009-12-05, by Cezary Kaliszyk
made some slight simplifications to the examples
2009-12-05, by Christian Urban
added three examples to IntEx for testing ideas - regularisation and injection seem to be not quite right yet
2009-12-05, by Christian Urban
tuned code
2009-12-05, by Christian Urban
merged
2009-12-04, by Christian Urban
not yet quite functional treatment of constants
2009-12-04, by Christian Urban
Changed FOCUS to SUBGOAL in rep_abs_rsp_tac; another 20% speedup :)
2009-12-04, by Cezary Kaliszyk
Changing FOCUS to CSUBGOAL (part 1)
2009-12-04, by Cezary Kaliszyk
abs_rep as ==
2009-12-04, by Cezary Kaliszyk
Cleaning the Quotients file
2009-12-04, by Cezary Kaliszyk
Minor renames and moving
2009-12-04, by Cezary Kaliszyk
Cleaning/review of QuotScript.
2009-12-04, by Cezary Kaliszyk
More cleaning
2009-12-04, by Cezary Kaliszyk
less
more
|
(0)
-1000
-960
+960
+1000
tip