2009-11-27 |
Christian Urban |
deleted obsolete qenv code
|
file |
diff |
annotate
|
2009-11-27 |
Christian Urban |
renamed REGULARIZE to be regularize
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
applic_prs
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
Removed unused things from QuotMain.
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
cleaning in MyInt
|
file |
diff |
annotate
|
2009-11-25 |
Christian Urban |
fixed the problem with generalising variables; at the moment it is quite a hack
|
file |
diff |
annotate
|
2009-11-24 |
Christian Urban |
added a prepare_tac
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
Moved cleaning to QuotMain
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
New cleaning tactic
|
file |
diff |
annotate
|
2009-11-24 |
Christian Urban |
explicit phases for the cleaning
|
file |
diff |
annotate
|
2009-11-24 |
Christian Urban |
addded a tactic, which sets up the three goals of the `algorithm'
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Finished temporary goal-directed lift_theorem wrapper.
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for atomize
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
lift_thm with a goal.
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for new code
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Moved new repabs_inj code to QuotMain
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
New repabs behaves the same way as old one.
|
file |
diff |
annotate
|
2009-11-23 |
Christian Urban |
code review with Cezary
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
a little tuning of comments
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
some debugging code, but cannot find the place where the cprems_of exception is raised
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
tried to prove the repabs_inj lemma, but failed for the moment
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
my first version of repabs injection
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
tunded
|
file |
diff |
annotate
|
2009-11-21 |
Christian Urban |
simplified get_fun so that it uses directly rty and qty, instead of qenv
|
file |
diff |
annotate
|
2009-11-20 |
Christian Urban |
started regularize of rtrm/qtrm version; looks quite promising
|
file |
diff |
annotate
|
2009-11-19 |
Christian Urban |
updated to new Isabelle
|
file |
diff |
annotate
|
2009-11-18 |
Christian Urban |
fixed the storage of qconst definitions
|
file |
diff |
annotate
|
2009-11-12 |
Christian Urban |
looking up data in quot_info works now (needs qualified string)
|
file |
diff |
annotate
|
2009-11-12 |
Christian Urban |
added a container for quotient constants (does not work yet though)
|
file |
diff |
annotate
|
2009-11-11 |
Christian Urban |
updated to new Theory_Data and to new Isabelle
|
file |
diff |
annotate
|
2009-11-11 |
Cezary Kaliszyk |
Removed 'Toplevel.program' for polyml 5.3
|
file |
diff |
annotate
|
2009-11-05 |
Christian Urban |
removed typing information from get_fun in quotient_def; *potentially* dangerous
|
file |
diff |
annotate
|
2009-11-05 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-11-04 |
Cezary Kaliszyk |
Experiments with lifting partially applied constants.
|
file |
diff |
annotate
|
2009-11-04 |
Cezary Kaliszyk |
Experiments in Int
|
file |
diff |
annotate
|
2009-11-04 |
Christian Urban |
fixed definition of PLUS
|
file |
diff |
annotate
|
2009-11-04 |
Christian Urban |
simplified the quotient_def code
|
file |
diff |
annotate
|
2009-11-03 |
Christian Urban |
simplified the quotient_def code; type of the defined constant must now be given; for-part eliminated
|
file |
diff |
annotate
|
2009-11-02 |
Christian Urban |
slightly saner way of parsing the quotient_def
|
file |
diff |
annotate
|
2009-11-02 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-11-02 |
Christian Urban |
changed Type.typ_match to Sign.typ_match
|
file |
diff |
annotate
|
2009-11-02 |
Cezary Kaliszyk |
Fixes after optimization and preparing for a general FORALL_PRS
|
file |
diff |
annotate
|
2009-10-30 |
Cezary Kaliszyk |
Cleaning of the interface to lift.
|
file |
diff |
annotate
|
2009-10-28 |
Cezary Kaliszyk |
disambiguate ===> syntax
|
file |
diff |
annotate
|
2009-10-28 |
Cezary Kaliszyk |
Cleaning the unnecessary theorems in 'IntEx'.
|
file |
diff |
annotate
|
2009-10-28 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2009-10-28 |
Cezary Kaliszyk |
Fixes
|
file |
diff |
annotate
|
2009-10-28 |
Christian Urban |
updated all definitions
|
file |
diff |
annotate
|
2009-10-28 |
Christian Urban |
added infrastructure for defining lifted constants
|
file |
diff |
annotate
|
2009-10-27 |
Cezary Kaliszyk |
Simplfied interface to repabs_injection.
|
file |
diff |
annotate
|
2009-10-27 |
Cezary Kaliszyk |
Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
|
file |
diff |
annotate
|
2009-10-27 |
Christian Urban |
made quotients compatiple with Nominal; updated keyword file
|
file |
diff |
annotate
|
2009-10-27 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-10-27 |
Cezary Kaliszyk |
Completely cleaned Int.
|
file |
diff |
annotate
|
2009-10-27 |
Cezary Kaliszyk |
Further reordering in Int code.
|
file |
diff |
annotate
|
2009-10-26 |
Cezary Kaliszyk |
Simplifying Int.
|
file |
diff |
annotate
|
2009-10-26 |
Cezary Kaliszyk |
Merge
|
file |
diff |
annotate
|
2009-10-26 |
Cezary Kaliszyk |
Simplifying Int and Working on map
|
file |
diff |
annotate
|
2009-10-26 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-10-26 |
Cezary Kaliszyk |
Simplifying code in int
|
file |
diff |
annotate
|
2009-10-26 |
Cezary Kaliszyk |
Symmetry of integer addition
|
file |
diff |
annotate
|
2009-10-24 |
Christian Urban |
added "print_quotients" command to th ekeyword file
|
file |
diff |
annotate
|
2009-10-24 |
Christian Urban |
added another example file about integers (see HOL/Int.thy)
|
file |
diff |
annotate
|