Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1000
-120
+120
+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.
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
less
more
|
(0)
-1000
-120
+120
+1000
tip