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