Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-480
+480
+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.
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
more name cleaning and removing
2009-12-04, by Cezary Kaliszyk
More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList
2009-12-04, by Cezary Kaliszyk
Cleaning & Renaming coming from QuotList
2009-12-04, by Cezary Kaliszyk
Cleaning in Quotients
2009-12-04, by Cezary Kaliszyk
Even more name changes and cleaning
2009-12-04, by Cezary Kaliszyk
More code cleaning and name changes
2009-12-04, by Cezary Kaliszyk
merge
2009-12-04, by Cezary Kaliszyk
merged
2009-12-04, by Cezary Kaliszyk
smaller theory footprint
2009-12-04, by Christian Urban
merged
2009-12-04, by Christian Urban
merge
2009-12-04, by Christian Urban
smaller theory footprint
2009-12-04, by Christian Urban
More name changes
2009-12-04, by Cezary Kaliszyk
Naming changes
2009-12-04, by Cezary Kaliszyk
code cleaning and renaming
2009-12-04, by Cezary Kaliszyk
merge
2009-12-04, by Cezary Kaliszyk
Removed previous inj_repabs_tac
2009-12-04, by Cezary Kaliszyk
some tuning
2009-12-04, by Christian Urban
merge
2009-12-04, by Cezary Kaliszyk
rep_abs_rsp_tac to replace the last use of instantiate_tac with matching and unification.
2009-12-04, by Cezary Kaliszyk
merged
2009-12-04, by Christian Urban
merged
2009-12-04, by Christian Urban
Change equiv_trans2 to EQUALS_RSP, since we can prove it for any quotient type, not only for eqv relations.
2009-12-04, by Cezary Kaliszyk
compose_tac instead of rtac to avoid unification; some code cleaning.
2009-12-04, by 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.
2009-12-04, by Cezary Kaliszyk
Using APPLY_RSP1; again a little bit faster.
2009-12-04, by Cezary Kaliszyk
Fixes after big merge.
2009-12-04, by Cezary Kaliszyk
The big merge; probably non-functional.
2009-12-04, by Cezary Kaliszyk
Testing the new tactic everywhere
2009-12-04, by Cezary Kaliszyk
First version of the deterministic rep-abs-inj-tac.
2009-12-04, by Cezary Kaliszyk
Changing = to \<equiv> in case if we want to use simp.
2009-12-04, by Cezary Kaliszyk
Even better: Completely got rid of the simps in both quotient_tac and inj_repabs_tac
2009-12-04, by Cezary Kaliszyk
merge
2009-12-04, by Cezary Kaliszyk
Made your version work again with LIST_REL_EQ.
2009-12-04, by Cezary Kaliszyk
the error occurs in APPLY_RSP_TAC where the wrong quotient (for LIST_REL) is applied
2009-12-03, by Christian Urban
removed quot argument...not all examples work anymore
2009-12-03, by Christian Urban
merged
2009-12-03, by Christian Urban
merged
2009-12-03, by Christian Urban
first version of internalised quotient theorems; added FIXME-TODO
2009-12-03, by Christian Urban
further dead code
2009-12-03, by Christian Urban
Reintroduced varifyT; we still need it for permutation definition.
2009-12-03, by Cezary Kaliszyk
Updated the examples
2009-12-03, by Cezary Kaliszyk
Fixed previous mistake
2009-12-03, by Cezary Kaliszyk
defs used automatically by clean_tac
2009-12-03, by Cezary Kaliszyk
Added qoutient_consts dest for getting all the constant definitions in the cleaning step.
2009-12-03, by Cezary Kaliszyk
Added the definition to quotient constant data.
2009-12-03, by Cezary Kaliszyk
removing unused code
2009-12-03, by Cezary Kaliszyk
merged
2009-12-03, by Christian Urban
deleted some dead code
2009-12-03, by Christian Urban
Included all_prs and ex_prs in the lambda_prs conversion.
2009-12-03, by Cezary Kaliszyk
further simplification
2009-12-03, by Christian Urban
simplified lambda_prs_conv
2009-12-03, by Christian Urban
deleted now obsolete argument rty everywhere
2009-12-02, by Christian Urban
deleted tests at the beginning of QuotMain
2009-12-02, by Christian Urban
Experiments with OPTION_map
2009-12-02, by Cezary Kaliszyk
merge
2009-12-02, by Cezary Kaliszyk
More experiments with higher order quotients and theorems with non-lifted constants.
2009-12-02, by Cezary Kaliszyk
merged
2009-12-02, by Christian Urban
Lifting to 2 different types :)
2009-12-02, by Cezary Kaliszyk
New APPLY_RSP which finally does automatic partial lifting :). Doesn't support same relation yet.
2009-12-02, by Cezary Kaliszyk
Fixed unlam for non-abstractions and updated list_induct_part proof.
2009-12-02, by Cezary Kaliszyk
Removed the use of 'rty' from APPLY_RSP, finally LF proofs go automatically.
2009-12-02, by Cezary Kaliszyk
The conversion approach works.
2009-12-02, by Cezary Kaliszyk
Trying a conversion based approach.
2009-12-02, by Cezary Kaliszyk
A bit of progress; but the object-logic vs meta-logic distinction is troublesome.
2009-12-02, by Cezary Kaliszyk
Added tactic for dealing with QUOT_TRUE and introducing QUOT_TRUE.
2009-12-02, by Cezary Kaliszyk
back in working state
2009-12-01, by Cezary Kaliszyk
clean
2009-12-01, by Cezary Kaliszyk
fixed previous commit
2009-12-01, by Christian Urban
fixed problems with FOCUS
2009-12-01, by Christian Urban
added a make_inst test
2009-12-01, by Christian Urban
Transformation of QUOT_TRUE assumption by any given function
2009-12-01, by Cezary Kaliszyk
QUOT_TRUE joke
2009-12-01, by Christian Urban
Removed last HOL_ss
2009-12-01, by Cezary Kaliszyk
more cleaning
2009-12-01, by Cezary Kaliszyk
Cleaning 'aps'.
2009-12-01, by Cezary Kaliszyk
merge
2009-11-30, by Cezary Kaliszyk
cleaned inj_regabs_trm
2009-11-30, by Christian Urban
merge
2009-11-30, by Cezary Kaliszyk
clean_tac rewrites the definitions the other way
2009-11-30, by Cezary Kaliszyk
merged
2009-11-30, by Christian Urban
added facilities to get all stored quotient data (equiv thms etc)
2009-11-30, by Christian Urban
More code cleaning
2009-11-30, by Cezary Kaliszyk
Code cleaning.
2009-11-30, by Cezary Kaliszyk
Commented clean-tac
2009-11-30, by Cezary Kaliszyk
Added another induction to LFex
2009-11-30, by Cezary Kaliszyk
tried to improve the inj_repabs_trm function but left the new part commented out
2009-11-29, by Christian Urban
added a new version of QuotMain to experiment with qids
2009-11-29, by Christian Urban
started functions for qid-insertion and fixed a bug in regularise
2009-11-29, by Christian Urban
Removed unnecessary HOL_ss which proved one of the subgoals.
2009-11-29, by 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.
2009-11-29, by Cezary Kaliszyk
introduced a global list of respectfulness lemmas; the attribute is [quot_rsp]
2009-11-29, by Christian Urban
tuned
2009-11-29, by Christian Urban
improved pattern matching inside the inj_repabs_tacs
2009-11-28, by Christian Urban
selective debugging of the inj_repabs_tac (at the moment for step 3 and 4 debugging information is printed)
2009-11-28, by Christian Urban
removed old inj_repabs_tac; kept only the one with (selective) debugging information
2009-11-28, by Christian Urban
renamed r_mk_comb_tac to inj_repabs_tac
2009-11-28, by Christian Urban
tuning
2009-11-28, by Christian Urban
tuned comments
2009-11-28, by Christian Urban
renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names
2009-11-28, by Christian Urban
Manually finished LF induction.
2009-11-28, by Cezary Kaliszyk
Moved fast instantiation to QuotMain
2009-11-28, by Cezary Kaliszyk
LFex proof a bit further.
2009-11-28, by Cezary Kaliszyk
merge
2009-11-28, by Cezary Kaliszyk
Looking at repabs proof in LF.
2009-11-28, by Cezary Kaliszyk
further proper merge
2009-11-28, by Christian Urban
merged
2009-11-28, by Christian Urban
more simplification
2009-11-28, by Christian Urban
Merged and tested that all works.
2009-11-28, by Cezary Kaliszyk
Finished and tested the new regularize
2009-11-28, by Cezary Kaliszyk
more tuning of the repabs-tactics
2009-11-28, by Christian Urban
fixed examples in IntEx and FSet
2009-11-28, by Christian Urban
merged
2009-11-28, by Christian Urban
fixed previous commit
2009-11-28, by Christian Urban
Cleaned all lemmas about regularisation of Ball and Bex and moved in one place. Second Ball simprox.
2009-11-28, by Cezary Kaliszyk
Merged comment
2009-11-28, by Cezary Kaliszyk
Integrated Stefan's tactic and changed substs to simps with empty context.
2009-11-28, by Cezary Kaliszyk
some slight tuning of the apply-tactic
2009-11-28, by Christian Urban
annotated a proof with all steps and simplified LAMBDA_RES_TAC
2009-11-28, by Christian Urban
Merge
2009-11-27, by Cezary Kaliszyk
The magical code from Stefan, will need to be integrated in the Simproc.
2009-11-27, by Cezary Kaliszyk
replaced FIRST' (map rtac list) with resolve_tac list
2009-11-27, by Christian Urban
Simplifying arguments; got rid of trans2_thm.
2009-11-27, by Cezary Kaliszyk
Cleaning of LFex. Lambda_prs fails to unify in 2 places.
2009-11-27, by Cezary Kaliszyk
Recommit
2009-11-27, by Cezary Kaliszyk
Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
2009-11-27, by Cezary Kaliszyk
More cleaning in QuotMain, identity handling.
2009-11-27, by Cezary Kaliszyk
Minor cleaning
2009-11-27, by Cezary Kaliszyk
tuned
2009-11-27, by Christian Urban
some tuning
2009-11-27, by Christian Urban
simplified gen_frees_tac and properly named abstracted variables
2009-11-27, by Christian Urban
removed CHANGED'
2009-11-27, by Christian Urban
introduced a separate lemma for id_simps
2009-11-27, by Christian Urban
renamed inj_REPABS to inj_repabs_trm
2009-11-27, by Christian Urban
tuned comments and moved slightly some code
2009-11-27, by Christian Urban
deleted obsolete qenv code
2009-11-27, by Christian Urban
renamed REGULARIZE to be regularize
2009-11-27, by Christian Urban
more tuning
2009-11-26, by Christian Urban
deleted get_fun_old and stuff
2009-11-26, by Christian Urban
recommited changes of comments
2009-11-26, by Christian Urban
Merge Again
2009-11-26, by Cezary Kaliszyk
Merged
2009-11-26, by Cezary Kaliszyk
tuned comments
2009-11-26, by Christian Urban
some diagnostic code for r_mk_comb
2009-11-26, by Christian Urban
introduced a new property for Ball and ===> on the left
2009-11-26, by Christian Urban
fixed QuotList
2009-11-26, by Christian Urban
changed left-res
2009-11-26, by Christian Urban
Manually regularized akind_aty_atrm.induct
2009-11-26, by Cezary Kaliszyk
Playing with Monos in LFex.
2009-11-26, by Cezary Kaliszyk
Fixed FSet after merge.
2009-11-26, by Cezary Kaliszyk
merged
2009-11-26, by Christian Urban
test with monos
2009-11-26, by Christian Urban
applic_prs
2009-11-25, by Cezary Kaliszyk
polishing
2009-11-25, by Christian Urban
reordered the code
2009-11-25, by Christian Urban
Moved exception handling to QuotMain and cleaned FSet.
2009-11-25, by Cezary Kaliszyk
Merge
2009-11-25, by Cezary Kaliszyk
Finished manual lifting of list_induct_part :)
2009-11-25, by Cezary Kaliszyk
comments tuning and slight reordering
2009-11-25, by Christian Urban
Merge
2009-11-25, by Cezary Kaliszyk
More moving from QuotMain to UnusedQuotMain
2009-11-25, by Cezary Kaliszyk
deleted some obsolete diagnostic code
2009-11-25, by Christian Urban
Removed unused things from QuotMain.
2009-11-25, by Cezary Kaliszyk
All examples work again.
2009-11-25, by Cezary Kaliszyk
cleaning in MyInt
2009-11-25, by Cezary Kaliszyk
lambda_prs and cleaning the existing examples.
2009-11-25, by Cezary Kaliszyk
merged
2009-11-25, by Christian Urban
fixed the problem with generalising variables; at the moment it is quite a hack
2009-11-25, by Christian Urban
Ho-matching failures...
2009-11-24, by Cezary Kaliszyk
changed unification to matching
2009-11-24, by Christian Urban
unification
2009-11-24, by Christian Urban
Lambda & SOLVED' for new quotient_tac
2009-11-24, by Cezary Kaliszyk
merged
2009-11-24, by Christian Urban
Conversion
2009-11-24, by Cezary Kaliszyk
The non-working procedure_tac.
2009-11-24, by Cezary Kaliszyk
merged
2009-11-24, by Christian Urban
use error instead of raising our own exception
2009-11-24, by Christian Urban
Fixes to the tactic after quotient_tac changed.
2009-11-24, by Cezary Kaliszyk
merged
2009-11-24, by Christian Urban
added a prepare_tac
2009-11-24, by Christian Urban
TRY' for clean_tac
2009-11-24, by Cezary Kaliszyk
Moved cleaning to QuotMain
2009-11-24, by Cezary Kaliszyk
New cleaning tactic
2009-11-24, by Cezary Kaliszyk
explicit phases for the cleaning
2009-11-24, by Christian Urban
Separate regularize_tac
2009-11-24, by 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.
2009-11-24, by Cezary Kaliszyk
More fixes for inj_REPABS
2009-11-24, by Cezary Kaliszyk
addded a tactic, which sets up the three goals of the `algorithm'
2009-11-24, by Christian Urban
fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
2009-11-23, by Christian Urban
merged
2009-11-23, by Christian Urban
tuned some comments
2009-11-23, by Christian Urban
Another not-typechecking regularized term.
2009-11-23, by Cezary Kaliszyk
domain_type in regularizing equality
2009-11-23, by Cezary Kaliszyk
More theorems lifted in the goal-directed way.
2009-11-23, by Cezary Kaliszyk
Finished temporary goal-directed lift_theorem wrapper.
2009-11-23, by Cezary Kaliszyk
merged
2009-11-23, by Christian Urban
a version of inj_REPABS (needs to be looked at again later)
2009-11-23, by Christian Urban
Fixes for atomize
2009-11-23, by Cezary Kaliszyk
merge
2009-11-23, by Cezary Kaliszyk
lift_thm with a goal.
2009-11-23, by Cezary Kaliszyk
slight change in code layout
2009-11-23, by Christian Urban
Fixes for new code
2009-11-23, by Cezary Kaliszyk
Removing dead code
2009-11-23, by Cezary Kaliszyk
Move atomize_goal to QuotMain
2009-11-23, by Cezary Kaliszyk
Removed second implementation of Regularize/Inject from FSet.
2009-11-23, by Cezary Kaliszyk
Moved new repabs_inj code to QuotMain
2009-11-23, by Cezary Kaliszyk
New repabs behaves the same way as old one.
2009-11-23, by Cezary Kaliszyk
code review with Cezary
2009-11-23, by Christian Urban
The other branch does not seem to work...
2009-11-23, by Cezary Kaliszyk
Fixes for recent changes.
2009-11-23, by Cezary Kaliszyk
updated to Isabelle 22nd November
2009-11-22, by Christian Urban
a little tuning of comments
2009-11-22, by Christian Urban
slight tuning
2009-11-21, by Christian Urban
some debugging code, but cannot find the place where the cprems_of exception is raised
2009-11-21, by Christian Urban
tried to prove the repabs_inj lemma, but failed for the moment
2009-11-21, by Christian Urban
my first version of repabs injection
2009-11-21, by Christian Urban
tuned
2009-11-21, by Christian Urban
tunded
2009-11-21, by Christian Urban
tuned
2009-11-21, by Christian Urban
flagged qenv-stuff as obsolete
2009-11-21, by Christian Urban
simplified get_fun so that it uses directly rty and qty, instead of qenv
2009-11-21, by Christian Urban
started regularize of rtrm/qtrm version; looks quite promising
2009-11-20, by Christian Urban
updated to new Isabelle
2009-11-19, by Christian Urban
fixed the storage of qconst definitions
2009-11-18, by Christian Urban
Still don't know how to do the proof automatically.
2009-11-13, by Cezary Kaliszyk
added some tracing information to all phases of lifting to the function lift_thm
2009-11-13, by Christian Urban
merge of the merge?
2009-11-12, by Cezary Kaliszyk
merged
2009-11-12, by Cezary Kaliszyk
added a FIXME commment
2009-11-12, by Christian Urban
looking up data in quot_info works now (needs qualified string)
2009-11-12, by Christian Urban
changed the quotdata to be a symtab table (needs fixing)
2009-11-12, by Christian Urban
added a container for quotient constants (does not work yet though)
2009-11-12, by Christian Urban
Lifting towards goal and manually finished the proof.
2009-11-11, by Cezary Kaliszyk
merge
2009-11-11, by Cezary Kaliszyk
less
more
|
(0)
-480
+480
+1000
tip