2009-12-09 |
Cezary Kaliszyk |
Finished one proof in IntEx2.
|
changeset |
files
|
2009-12-09 |
Christian Urban |
slightly more on IntEx2
|
changeset |
files
|
2009-12-09 |
Christian Urban |
proved (with a lot of pain) that times_raw is respectful
|
changeset |
files
|
2009-12-09 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-09 |
Christian Urban |
fixed minor stupidity
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
Exception handling.
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
Code cleaning.
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
foldr_rsp.
|
changeset |
files
|
2009-12-09 |
Christian Urban |
tuned
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants.
|
changeset |
files
|
2009-12-09 |
Christian Urban |
deleted make_inst3
|
changeset |
files
|
2009-12-09 |
Christian Urban |
tuned
|
changeset |
files
|
2009-12-09 |
Christian Urban |
tuned
|
changeset |
files
|
2009-12-09 |
Christian Urban |
moved function and tuned comment
|
changeset |
files
|
2009-12-09 |
Christian Urban |
improved fun_map_conv
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
Arbitrary number of fun_map_tacs.
|
changeset |
files
|
2009-12-09 |
Cezary Kaliszyk |
Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
tuned code
|
changeset |
files
|
2009-12-08 |
Christian Urban |
tuned the examples and flagged the problematic cleaning lemmas in FSet
|
changeset |
files
|
2009-12-08 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-08 |
Christian Urban |
implemented cleaning strategy with fun_map.simps on non-bounded variables; still a few rough edges
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
manually cleaned the hard lemma.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-08 |
Christian Urban |
decoupled QuotProd from QuotMain and also started new cleaning strategy
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
An example which is hard to lift because of the interplay between lambda_prs and unfolding.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
proper formulation of all preservation theorems
|
changeset |
files
|
2009-12-08 |
Christian Urban |
started to reformulate preserve lemmas
|
changeset |
files
|
2009-12-08 |
Christian Urban |
properly set up the prs_rules
|
changeset |
files
|
2009-12-08 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-08 |
Christian Urban |
added preserve rules to the cleaning_tac
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
cleaning.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-08 |
Christian Urban |
chnaged syntax to "lifting theorem"
|
changeset |
files
|
2009-12-08 |
Christian Urban |
changed names of attributes
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Manual regularization of a goal in FSet.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-08 |
Christian Urban |
added methods for the lifting_tac and the other tacs
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
make_inst3
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
trans2 replaced with equals_rsp_tac
|
changeset |
files
|
2009-12-08 |
Christian Urban |
corrected name of FSet in ROOT.ML
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Made fset work again to test all.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Finished the proof of ttt2 and found bug in regularize when trying ttt3.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Another lambda example theorem proved. Seems it starts working properly.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Removed pattern from quot_rel_rsp, since list_rel and all used introduced ones cannot be patterned
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Proper checked map_rsp.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Nitpick found a counterexample for one lemma.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
Added a 'rep_abs' in inj_repabs_trm of babs; and proved two lam examples.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
It also regularizes.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
inj_repabs also works.
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-08 |
Cezary Kaliszyk |
An example of working cleaning for lambda lifting. Still not sure why Babs helps.
|
changeset |
files
|
2009-12-08 |
Christian Urban |
tuned
|
changeset |
files
|
2009-12-08 |
Christian Urban |
the lift_tac produces a warning message if one of the three automatic proofs fails
|
changeset |
files
|
2009-12-08 |
Christian Urban |
added a thm list for ids
|
changeset |
files
|
2009-12-08 |
Christian Urban |
removed a fixme: map_info is now checked
|
changeset |
files
|
2009-12-07 |
Christian Urban |
tuning of the code
|
changeset |
files
|
2009-12-07 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-07 |
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 ===>
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
3 lambda examples in FSet. In the last one regularize_term fails.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
Handling of errors in lambda_prs_conv.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
babs_prs
|
changeset |
files
|
2009-12-07 |
Christian Urban |
clarified the function examples
|
changeset |
files
|
2009-12-07 |
Christian Urban |
first attempt to deal with Babs in regularise and cleaning (not yet working)
|
changeset |
files
|
2009-12-07 |
Christian Urban |
isabelle make tests all examples
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
make_inst for lambda_prs where the second quotient is not identity.
|
changeset |
files
|
2009-12-07 |
Christian Urban |
added "end" to each example theory
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
List moved after QuotMain
|
changeset |
files
|
2009-12-07 |
Christian Urban |
cleaning
|
changeset |
files
|
2009-12-07 |
Christian Urban |
final move
|
changeset |
files
|
2009-12-07 |
Christian Urban |
directory re-arrangement
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
inj_repabs_tac handles Babs now.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
Fix of regularize for babs and proof of babs_rsp.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
Using pair_prs; debugging the error in regularize of a lambda.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
QuotProd with product_quotient and a 3 respects and preserves lemmas.
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-07 |
Cezary Kaliszyk |
3 new example thms in MyInt; reveal problems with handling of lambdas; regularize fails with "Loose Bound".
|
changeset |
files
|
2009-12-07 |
Christian Urban |
simplified the regularize simproc
|
changeset |
files
|
2009-12-07 |
Christian Urban |
now simpler regularize_tac with added solver works
|
changeset |
files
|
2009-12-07 |
Christian Urban |
removed usage of HOL_basic_ss by using a slighly extended version of empty_ss
|
changeset |
files
|
2009-12-06 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-06 |
Christian Urban |
fixed examples
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Fix IntEx2 for equiv_list
|
changeset |
files
|
2009-12-06 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-06 |
Christian Urban |
working state again
|
changeset |
files
|
2009-12-06 |
Christian Urban |
added a theorem list for equivalence theorems
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Name changes.
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Solved all quotient goals.
|
changeset |
files
|
2009-12-06 |
Christian Urban |
updated Isabelle and deleted mono rules
|
changeset |
files
|
2009-12-06 |
Christian Urban |
more tuning of the code
|
changeset |
files
|
2009-12-06 |
Christian Urban |
puting code in separate sections
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Handle 'find_qt_asm' exception. Now all inj_repabs_goals should be solved automatically.
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-06 |
Cezary Kaliszyk |
Simpler definition code that works with any type maps.
|
changeset |
files
|
2009-12-06 |
Christian Urban |
working on lambda_prs with examples; polished code of clean_tac
|
changeset |
files
|
2009-12-06 |
Christian Urban |
renamed lambda_allex_prs
|
changeset |
files
|
2009-12-06 |
Christian Urban |
added more to IntEx2
|
changeset |
files
|
2009-12-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-05 |
Christian Urban |
added new example for Ints; regularise does not work in all instances
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Definitions folded first.
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Used symmetric definitions. Moved quotient_rsp to QuotMain.
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Proved foldl_rsp and ho_map_rsp
|
changeset |
files
|
2009-12-05 |
Christian Urban |
moved all_prs and ex_prs out from the conversion into the simplifier
|
changeset |
files
|
2009-12-05 |
Christian Urban |
further cleaning
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx.
|
changeset |
files
|
2009-12-05 |
Christian Urban |
simplified inj_repabs_trm
|
changeset |
files
|
2009-12-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-05 |
Christian Urban |
simpler version of clean_tac
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Handling of respects in the fast inj_repabs_tac; includes respects with quotient assumptions.
|
changeset |
files
|
2009-12-05 |
Cezary Kaliszyk |
Solutions to IntEx tests.
|
changeset |
files
|
2009-12-05 |
Christian Urban |
made some slight simplifications to the examples
|
changeset |
files
|
2009-12-05 |
Christian Urban |
added three examples to IntEx for testing ideas - regularisation and injection seem to be not quite right yet
|
changeset |
files
|
2009-12-04 |
Christian Urban |
tuned code
|
changeset |
files
|
2009-12-04 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-04 |
Christian Urban |
not yet quite functional treatment of constants
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Changed FOCUS to SUBGOAL in rep_abs_rsp_tac; another 20% speedup :)
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Changing FOCUS to CSUBGOAL (part 1)
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
abs_rep as ==
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Cleaning the Quotients file
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Minor renames and moving
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Cleaning/review of QuotScript.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
More cleaning
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
more name cleaning and removing
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Cleaning & Renaming coming from QuotList
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Cleaning in Quotients
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Even more name changes and cleaning
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
More code cleaning and name changes
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
merged
|
changeset |
files
|
2009-12-04 |
Christian Urban |
smaller theory footprint
|
changeset |
files
|
2009-12-04 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-04 |
Christian Urban |
merge
|
changeset |
files
|
2009-12-04 |
Christian Urban |
smaller theory footprint
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
More name changes
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Naming changes
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
code cleaning and renaming
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Removed previous inj_repabs_tac
|
changeset |
files
|
2009-12-04 |
Christian Urban |
some tuning
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
rep_abs_rsp_tac to replace the last use of instantiate_tac with matching and unification.
|
changeset |
files
|
2009-12-04 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-04 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Change equiv_trans2 to EQUALS_RSP, since we can prove it for any quotient type, not only for eqv relations.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
compose_tac instead of rtac to avoid unification; some code cleaning.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Got to about 5 seconds for the longest proof. APPLY_RSP_TAC' solves the quotient internally without instantiation resulting in a faster proof.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Using APPLY_RSP1; again a little bit faster.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Fixes after big merge.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
The big merge; probably non-functional.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Testing the new tactic everywhere
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
First version of the deterministic rep-abs-inj-tac.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Changing = to \<equiv> in case if we want to use simp.
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Even better: Completely got rid of the simps in both quotient_tac and inj_repabs_tac
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-04 |
Cezary Kaliszyk |
Made your version work again with LIST_REL_EQ.
|
changeset |
files
|
2009-12-03 |
Christian Urban |
the error occurs in APPLY_RSP_TAC where the wrong quotient (for LIST_REL) is applied
|
changeset |
files
|
2009-12-03 |
Christian Urban |
removed quot argument...not all examples work anymore
|
changeset |
files
|
2009-12-03 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-03 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-03 |
Christian Urban |
first version of internalised quotient theorems; added FIXME-TODO
|
changeset |
files
|
2009-12-03 |
Christian Urban |
further dead code
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Reintroduced varifyT; we still need it for permutation definition.
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Updated the examples
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Fixed previous mistake
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
defs used automatically by clean_tac
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Added qoutient_consts dest for getting all the constant definitions in the cleaning step.
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Added the definition to quotient constant data.
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
removing unused code
|
changeset |
files
|
2009-12-03 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-03 |
Christian Urban |
deleted some dead code
|
changeset |
files
|
2009-12-03 |
Cezary Kaliszyk |
Included all_prs and ex_prs in the lambda_prs conversion.
|
changeset |
files
|
2009-12-03 |
Christian Urban |
further simplification
|
changeset |
files
|
2009-12-03 |
Christian Urban |
simplified lambda_prs_conv
|
changeset |
files
|
2009-12-02 |
Christian Urban |
deleted now obsolete argument rty everywhere
|
changeset |
files
|
2009-12-02 |
Christian Urban |
deleted tests at the beginning of QuotMain
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Experiments with OPTION_map
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
More experiments with higher order quotients and theorems with non-lifted constants.
|
changeset |
files
|
2009-12-02 |
Christian Urban |
merged
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Lifting to 2 different types :)
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
New APPLY_RSP which finally does automatic partial lifting :). Doesn't support same relation yet.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Fixed unlam for non-abstractions and updated list_induct_part proof.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Removed the use of 'rty' from APPLY_RSP, finally LF proofs go automatically.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
The conversion approach works.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Trying a conversion based approach.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
A bit of progress; but the object-logic vs meta-logic distinction is troublesome.
|
changeset |
files
|
2009-12-02 |
Cezary Kaliszyk |
Added tactic for dealing with QUOT_TRUE and introducing QUOT_TRUE.
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
back in working state
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
clean
|
changeset |
files
|
2009-12-01 |
Christian Urban |
fixed previous commit
|
changeset |
files
|
2009-12-01 |
Christian Urban |
fixed problems with FOCUS
|
changeset |
files
|
2009-12-01 |
Christian Urban |
added a make_inst test
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
Transformation of QUOT_TRUE assumption by any given function
|
changeset |
files
|
2009-12-01 |
Christian Urban |
QUOT_TRUE joke
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
Removed last HOL_ss
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
more cleaning
|
changeset |
files
|
2009-12-01 |
Cezary Kaliszyk |
Cleaning 'aps'.
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-30 |
Christian Urban |
cleaned inj_regabs_trm
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
clean_tac rewrites the definitions the other way
|
changeset |
files
|
2009-11-30 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-30 |
Christian Urban |
added facilities to get all stored quotient data (equiv thms etc)
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
More code cleaning
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
Code cleaning.
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
Commented clean-tac
|
changeset |
files
|
2009-11-30 |
Cezary Kaliszyk |
Added another induction to LFex
|
changeset |
files
|
2009-11-29 |
Christian Urban |
tried to improve the inj_repabs_trm function but left the new part commented out
|
changeset |
files
|
2009-11-29 |
Christian Urban |
added a new version of QuotMain to experiment with qids
|
changeset |
files
|
2009-11-29 |
Christian Urban |
started functions for qid-insertion and fixed a bug in regularise
|
changeset |
files
|
2009-11-29 |
Cezary Kaliszyk |
Removed unnecessary HOL_ss which proved one of the subgoals.
|
changeset |
files
|
2009-11-29 |
Cezary Kaliszyk |
Added 'TRY' to refl in clean_tac to get as far as possible. Removed unnecessary [quot_rsp] in FSet. Added necessary [quot_rsp] and one lifted thm in LamEx.
|
changeset |
files
|
2009-11-29 |
Christian Urban |
introduced a global list of respectfulness lemmas; the attribute is [quot_rsp]
|
changeset |
files
|
2009-11-29 |
Christian Urban |
tuned
|
changeset |
files
|
2009-11-28 |
Christian Urban |
improved pattern matching inside the inj_repabs_tacs
|
changeset |
files
|
2009-11-28 |
Christian Urban |
selective debugging of the inj_repabs_tac (at the moment for step 3 and 4 debugging information is printed)
|
changeset |
files
|
2009-11-28 |
Christian Urban |
removed old inj_repabs_tac; kept only the one with (selective) debugging information
|
changeset |
files
|
2009-11-28 |
Christian Urban |
renamed r_mk_comb_tac to inj_repabs_tac
|
changeset |
files
|
2009-11-28 |
Christian Urban |
tuning
|
changeset |
files
|
2009-11-28 |
Christian Urban |
tuned comments
|
changeset |
files
|
2009-11-28 |
Christian Urban |
renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Manually finished LF induction.
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Moved fast instantiation to QuotMain
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
LFex proof a bit further.
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Looking at repabs proof in LF.
|
changeset |
files
|
2009-11-28 |
Christian Urban |
further proper merge
|
changeset |
files
|
2009-11-28 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-28 |
Christian Urban |
more simplification
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Merged and tested that all works.
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Finished and tested the new regularize
|
changeset |
files
|
2009-11-28 |
Christian Urban |
more tuning of the repabs-tactics
|
changeset |
files
|
2009-11-28 |
Christian Urban |
fixed examples in IntEx and FSet
|
changeset |
files
|
2009-11-28 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-28 |
Christian Urban |
fixed previous commit
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Cleaned all lemmas about regularisation of Ball and Bex and moved in one place. Second Ball simprox.
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Merged comment
|
changeset |
files
|
2009-11-28 |
Cezary Kaliszyk |
Integrated Stefan's tactic and changed substs to simps with empty context.
|
changeset |
files
|
2009-11-28 |
Christian Urban |
some slight tuning of the apply-tactic
|
changeset |
files
|
2009-11-28 |
Christian Urban |
annotated a proof with all steps and simplified LAMBDA_RES_TAC
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
The magical code from Stefan, will need to be integrated in the Simproc.
|
changeset |
files
|
2009-11-27 |
Christian Urban |
replaced FIRST' (map rtac list) with resolve_tac list
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Simplifying arguments; got rid of trans2_thm.
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Cleaning of LFex. Lambda_prs fails to unify in 2 places.
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Recommit
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
More cleaning in QuotMain, identity handling.
|
changeset |
files
|
2009-11-27 |
Cezary Kaliszyk |
Minor cleaning
|
changeset |
files
|
2009-11-27 |
Christian Urban |
tuned
|
changeset |
files
|
2009-11-27 |
Christian Urban |
some tuning
|
changeset |
files
|
2009-11-27 |
Christian Urban |
simplified gen_frees_tac and properly named abstracted variables
|
changeset |
files
|
2009-11-27 |
Christian Urban |
removed CHANGED'
|
changeset |
files
|
2009-11-27 |
Christian Urban |
introduced a separate lemma for id_simps
|
changeset |
files
|
2009-11-27 |
Christian Urban |
renamed inj_REPABS to inj_repabs_trm
|
changeset |
files
|
2009-11-27 |
Christian Urban |
tuned comments and moved slightly some code
|
changeset |
files
|
2009-11-27 |
Christian Urban |
deleted obsolete qenv code
|
changeset |
files
|
2009-11-27 |
Christian Urban |
renamed REGULARIZE to be regularize
|
changeset |
files
|
2009-11-26 |
Christian Urban |
more tuning
|
changeset |
files
|
2009-11-26 |
Christian Urban |
deleted get_fun_old and stuff
|
changeset |
files
|
2009-11-26 |
Christian Urban |
recommited changes of comments
|
changeset |
files
|
2009-11-26 |
Cezary Kaliszyk |
Merge Again
|
changeset |
files
|
2009-11-26 |
Cezary Kaliszyk |
Merged
|
changeset |
files
|
2009-11-26 |
Christian Urban |
tuned comments
|
changeset |
files
|
2009-11-26 |
Christian Urban |
some diagnostic code for r_mk_comb
|
changeset |
files
|
2009-11-26 |
Christian Urban |
introduced a new property for Ball and ===> on the left
|
changeset |
files
|
2009-11-26 |
Christian Urban |
fixed QuotList
|
changeset |
files
|
2009-11-26 |
Christian Urban |
changed left-res
|
changeset |
files
|
2009-11-26 |
Cezary Kaliszyk |
Manually regularized akind_aty_atrm.induct
|
changeset |
files
|
2009-11-26 |
Cezary Kaliszyk |
Playing with Monos in LFex.
|
changeset |
files
|
2009-11-26 |
Cezary Kaliszyk |
Fixed FSet after merge.
|
changeset |
files
|
2009-11-26 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-26 |
Christian Urban |
test with monos
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
applic_prs
|
changeset |
files
|
2009-11-25 |
Christian Urban |
polishing
|
changeset |
files
|
2009-11-25 |
Christian Urban |
reordered the code
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
Moved exception handling to QuotMain and cleaned FSet.
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
Finished manual lifting of list_induct_part :)
|
changeset |
files
|
2009-11-25 |
Christian Urban |
comments tuning and slight reordering
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
More moving from QuotMain to UnusedQuotMain
|
changeset |
files
|
2009-11-25 |
Christian Urban |
deleted some obsolete diagnostic code
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
Removed unused things from QuotMain.
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
All examples work again.
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
cleaning in MyInt
|
changeset |
files
|
2009-11-25 |
Cezary Kaliszyk |
lambda_prs and cleaning the existing examples.
|
changeset |
files
|
2009-11-25 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-25 |
Christian Urban |
fixed the problem with generalising variables; at the moment it is quite a hack
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Ho-matching failures...
|
changeset |
files
|
2009-11-24 |
Christian Urban |
changed unification to matching
|
changeset |
files
|
2009-11-24 |
Christian Urban |
unification
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Lambda & SOLVED' for new quotient_tac
|
changeset |
files
|
2009-11-24 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Conversion
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
The non-working procedure_tac.
|
changeset |
files
|
2009-11-24 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-24 |
Christian Urban |
use error instead of raising our own exception
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Fixes to the tactic after quotient_tac changed.
|
changeset |
files
|
2009-11-24 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-24 |
Christian Urban |
added a prepare_tac
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
TRY' for clean_tac
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Moved cleaning to QuotMain
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
New cleaning tactic
|
changeset |
files
|
2009-11-24 |
Christian Urban |
explicit phases for the cleaning
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Separate regularize_tac
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
Another theorem for which the new regularize differs from old one, so the goal is not proved. But it seems, that the new one is better.
|
changeset |
files
|
2009-11-24 |
Cezary Kaliszyk |
More fixes for inj_REPABS
|
changeset |
files
|
2009-11-24 |
Christian Urban |
addded a tactic, which sets up the three goals of the `algorithm'
|
changeset |
files
|
2009-11-23 |
Christian Urban |
fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
|
changeset |
files
|
2009-11-23 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-23 |
Christian Urban |
tuned some comments
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Another not-typechecking regularized term.
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
domain_type in regularizing equality
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
More theorems lifted in the goal-directed way.
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Finished temporary goal-directed lift_theorem wrapper.
|
changeset |
files
|
2009-11-23 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-23 |
Christian Urban |
a version of inj_REPABS (needs to be looked at again later)
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for atomize
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
lift_thm with a goal.
|
changeset |
files
|
2009-11-23 |
Christian Urban |
slight change in code layout
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for new code
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Removing dead code
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Move atomize_goal to QuotMain
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Removed second implementation of Regularize/Inject from FSet.
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Moved new repabs_inj code to QuotMain
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
New repabs behaves the same way as old one.
|
changeset |
files
|
2009-11-23 |
Christian Urban |
code review with Cezary
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
The other branch does not seem to work...
|
changeset |
files
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for recent changes.
|
changeset |
files
|
2009-11-22 |
Christian Urban |
updated to Isabelle 22nd November
|
changeset |
files
|
2009-11-21 |
Christian Urban |
a little tuning of comments
|
changeset |
files
|
2009-11-21 |
Christian Urban |
slight tuning
|
changeset |
files
|
2009-11-21 |
Christian Urban |
some debugging code, but cannot find the place where the cprems_of exception is raised
|
changeset |
files
|
2009-11-21 |
Christian Urban |
tried to prove the repabs_inj lemma, but failed for the moment
|
changeset |
files
|
2009-11-21 |
Christian Urban |
my first version of repabs injection
|
changeset |
files
|
2009-11-21 |
Christian Urban |
tuned
|
changeset |
files
|
2009-11-21 |
Christian Urban |
tunded
|
changeset |
files
|
2009-11-21 |
Christian Urban |
tuned
|
changeset |
files
|
2009-11-21 |
Christian Urban |
flagged qenv-stuff as obsolete
|
changeset |
files
|
2009-11-21 |
Christian Urban |
simplified get_fun so that it uses directly rty and qty, instead of qenv
|
changeset |
files
|
2009-11-20 |
Christian Urban |
started regularize of rtrm/qtrm version; looks quite promising
|
changeset |
files
|
2009-11-19 |
Christian Urban |
updated to new Isabelle
|
changeset |
files
|
2009-11-18 |
Christian Urban |
fixed the storage of qconst definitions
|
changeset |
files
|
2009-11-13 |
Cezary Kaliszyk |
Still don't know how to do the proof automatically.
|
changeset |
files
|
2009-11-13 |
Christian Urban |
added some tracing information to all phases of lifting to the function lift_thm
|
changeset |
files
|
2009-11-12 |
Cezary Kaliszyk |
merge of the merge?
|
changeset |
files
|
2009-11-12 |
Cezary Kaliszyk |
merged
|
changeset |
files
|
2009-11-12 |
Christian Urban |
added a FIXME commment
|
changeset |
files
|
2009-11-12 |
Christian Urban |
looking up data in quot_info works now (needs qualified string)
|
changeset |
files
|
2009-11-12 |
Christian Urban |
changed the quotdata to be a symtab table (needs fixing)
|
changeset |
files
|
2009-11-12 |
Christian Urban |
added a container for quotient constants (does not work yet though)
|
changeset |
files
|
2009-11-11 |
Cezary Kaliszyk |
Lifting towards goal and manually finished the proof.
|
changeset |
files
|
2009-11-11 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-11 |
Cezary Kaliszyk |
Modifications while preparing the goal-directed version.
|
changeset |
files
|
2009-11-11 |
Christian Urban |
updated to new Theory_Data and to new Isabelle
|
changeset |
files
|
2009-11-11 |
Cezary Kaliszyk |
Removed 'Toplevel.program' for polyml 5.3
|
changeset |
files
|
2009-11-10 |
Cezary Kaliszyk |
Atomizing a "goal" theorems.
|
changeset |
files
|
2009-11-10 |
Cezary Kaliszyk |
More code cleaning and commenting
|
changeset |
files
|
2009-11-09 |
Cezary Kaliszyk |
Minor cleaning and removing of some 'handle _'.
|
changeset |
files
|
2009-11-09 |
Cezary Kaliszyk |
Cleaning and commenting
|
changeset |
files
|
2009-11-09 |
Cezary Kaliszyk |
Fixes for the other get_fun implementation.
|
changeset |
files
|
2009-11-06 |
Christian Urban |
permutation lifting works now also
|
changeset |
files
|
2009-11-06 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-06 |
Christian Urban |
updated to new Isabelle version and added a new example file
|
changeset |
files
|
2009-11-06 |
Cezary Kaliszyk |
Minor changes
|
changeset |
files
|
2009-11-06 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-06 |
Cezary Kaliszyk |
fold_rsp
|
changeset |
files
|
2009-11-06 |
Christian Urban |
tuned the code in quotient and quotient_def
|
changeset |
files
|
2009-11-05 |
Cezary Kaliszyk |
More functionality for lifting list.cases and list.recs.
|
changeset |
files
|
2009-11-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-05 |
Christian Urban |
removed typing information from get_fun in quotient_def; *potentially* dangerous
|
changeset |
files
|
2009-11-05 |
Cezary Kaliszyk |
Remaining fixes for polymorphic types. map_append now lifts properly with 'a list and 'b list.
|
changeset |
files
|
2009-11-05 |
Christian Urban |
removed Simplifier.context
|
changeset |
files
|
2009-11-05 |
Christian Urban |
replaced check_term o parse_term by read_term
|
changeset |
files
|
2009-11-05 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-05 |
Cezary Kaliszyk |
Infrastructure for polymorphic types
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Two new tests for get_fun. Second one fails.
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Type instantiation in regularize
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Description of regularize
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Experiments with lifting partially applied constants.
|
changeset |
files
|
2009-11-04 |
Christian Urban |
more tuning
|
changeset |
files
|
2009-11-04 |
Christian Urban |
slightly tuned
|
changeset |
files
|
2009-11-04 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-04 |
Christian Urban |
separated the quotient_def into a separate file
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Experiments in Int
|
changeset |
files
|
2009-11-04 |
Christian Urban |
fixed definition of PLUS
|
changeset |
files
|
2009-11-04 |
Christian Urban |
simplified the quotient_def code
|
changeset |
files
|
2009-11-04 |
Cezary Kaliszyk |
Lifting 'fold1.simps(2)' and some cleaning.
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
Playing with alpha_refl.
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
Alpha.induct now lifts automatically.
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
applic_prs
|
changeset |
files
|
2009-11-03 |
Christian Urban |
simplified the quotient_def code; type of the defined constant must now be given; for-part eliminated
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
Automatic FORALL_PRS. 'list.induct' lifts automatically. Faster ALLEX_RSP
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-11-03 |
Cezary Kaliszyk |
Preparing infrastructure for general FORALL_PRS
|
changeset |
files
|
2009-11-02 |
Christian Urban |
split quotient.ML into two files
|
changeset |
files
|
2009-11-02 |
Christian Urban |
slightly saner way of parsing the quotient_def
|
changeset |
files
|
2009-11-02 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-02 |
Christian Urban |
changed Type.typ_match to Sign.typ_match
|
changeset |
files
|
2009-11-02 |
Cezary Kaliszyk |
Fixes after optimization and preparing for a general FORALL_PRS
|
changeset |
files
|
2009-11-02 |
Cezary Kaliszyk |
Optimization
|
changeset |
files
|
2009-11-02 |
Cezary Kaliszyk |
Map does not fully work yet.
|
changeset |
files
|
2009-11-02 |
Cezary Kaliszyk |
Fixed quotdata_lookup.
|
changeset |
files
|
2009-11-02 |
Christian Urban |
fixed problem with maps_update
|
changeset |
files
|
2009-11-02 |
Christian Urban |
merged
|
changeset |
files
|
2009-11-02 |
Christian Urban |
fixed the problem with types in map
|
changeset |
files
|
2009-10-31 |
Cezary Kaliszyk |
Automatic computation of application preservation and manually finished "alpha.induct". Slow...
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Regularize for equalities and a better tactic. "alpha.cases" now lifts.
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Regularization
|
changeset |
files
|
2009-10-30 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-30 |
Christian Urban |
added some facts about fresh and support of lam
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Finally merged the code of the versions of regularize and tested examples.
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Lemmas about fv.
|
changeset |
files
|
2009-10-30 |
Christian Urban |
changed the order of rfv and reformulated a3 with rfv
|
changeset |
files
|
2009-10-30 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-30 |
Christian Urban |
not sure what changed here
|
changeset |
files
|
2009-10-30 |
Christian Urban |
added fv-function
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
The proper real_alpha
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Finding applications and duplicates filtered out in abstractions
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Cleaning also in Lam
|
changeset |
files
|
2009-10-30 |
Cezary Kaliszyk |
Cleaning of the interface to lift.
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
Tried manually lifting real_alpha
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
More tests in Lam
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
Cleaning of 'map id' and 'prod_fun id id' in lower_defs.
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
Using subst for identity definition.
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
Lifting of the 3 lemmas in LamEx
|
changeset |
files
|
2009-10-29 |
Cezary Kaliszyk |
Fixed wrong CARD definition and removed the "Does not work anymore" comment.
|
changeset |
files
|
2009-10-29 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-28 |
Christian Urban |
updated some definitions; had to give sometimes different names; somewhere I introduced a bug, since not everything is working anymore (needs fixing!)
|
changeset |
files
|
2009-10-28 |
Christian Urban |
ported all constant definitions to new scheme
|
changeset |
files
|
2009-10-28 |
Christian Urban |
fixed the definition of alpha; this *breaks* some of the experiments
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
disambiguate ===> syntax
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
More cleaning in Lam code
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
cleaned FSet
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Some cleaning
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Cleaning the unnecessary theorems in 'IntEx'.
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Fix also in the general procedure.
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
merge
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Fixes
|
changeset |
files
|
2009-10-28 |
Christian Urban |
updated all definitions
|
changeset |
files
|
2009-10-28 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-28 |
Christian Urban |
added infrastructure for defining lifted constants
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
First experiments with Lambda
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Fixed mistake in const generation, will postpone this.
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
More finshed proofs and cleaning
|
changeset |
files
|
2009-10-28 |
Cezary Kaliszyk |
Proof of append_rsp
|
changeset |
files
|
2009-10-28 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-28 |
Christian Urban |
added a function for matching types
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Manual conversion of equality to equivalence allows lifting append_assoc.
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Simplfied interface to repabs_injection.
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
map_append lifted automatically.
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Manually lifted Map_Append.
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Merged
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
|
changeset |
files
|
2009-10-27 |
Christian Urban |
tuned
|
changeset |
files
|
2009-10-27 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-27 |
Christian Urban |
added equiv-thm to the quot_info
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Simplifying FSet with new functions.
|
changeset |
files
|
2009-10-27 |
Christian Urban |
added an example about lambda-terms
|
changeset |
files
|
2009-10-27 |
Christian Urban |
made quotients compatiple with Nominal; updated keyword file
|
changeset |
files
|
2009-10-27 |
Christian Urban |
merged
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Completely cleaned Int.
|
changeset |
files
|
2009-10-27 |
Cezary Kaliszyk |
Further reordering in Int code.
|
changeset |
files
|
2009-10-26 |
Cezary Kaliszyk |
Simplifying Int.
|
changeset |
files
|
2009-10-26 |
Cezary Kaliszyk |
Merge
|
changeset |
files
|