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
|