1998-08-20 |
paulson |
Must remove leD from simpset
|
changeset |
files
|
1998-08-20 |
paulson |
tidied
|
changeset |
files
|
1998-08-20 |
paulson |
Must remove less_imp_le from simpset
|
changeset |
files
|
1998-08-20 |
nipkow |
Added converse_rtranclE(2)
|
changeset |
files
|
1998-08-20 |
paulson |
Now qed_spec_mp respects locales, by calling ml_store_thm
|
changeset |
files
|
1998-08-19 |
wenzelm |
fixed param;
|
changeset |
files
|
1998-08-19 |
wenzelm |
assume: adjust_maxidx;
|
changeset |
files
|
1998-08-19 |
paulson |
new version, more resistant to PROOF FAILED. Now it distinguishes between
|
changeset |
files
|
1998-08-19 |
paulson |
The warning "Rewrite rule from different theory" is ALWAYS printed, even if
|
changeset |
files
|
1998-08-19 |
paulson |
new theorem zero_less_diff
|
changeset |
files
|
1998-08-19 |
paulson |
Misc changes
|
changeset |
files
|
1998-08-19 |
paulson |
Deleted obsolete declaration of PartE'
|
changeset |
files
|
1998-08-19 |
paulson |
Tidied, removing uses of less_imp_diff_positive
|
changeset |
files
|
1998-08-19 |
paulson |
tidied
|
changeset |
files
|
1998-08-19 |
paulson |
fixed overloading of "image"
|
changeset |
files
|
1998-08-19 |
paulson |
Overloading decl should assist Blast_tac
|
changeset |
files
|
1998-08-19 |
paulson |
less_imp_diff_positive is redundant with new simprule zero_less_diff
|
changeset |
files
|
1998-08-19 |
paulson |
Some new theorems. zero_less_diff replaces less_imp_diff_positive
|
changeset |
files
|
1998-08-18 |
paulson |
ZF.thy
|
changeset |
files
|
1998-08-18 |
paulson |
new theorem Un_Diff_Int
|
changeset |
files
|
1998-08-18 |
paulson |
added comment
|
changeset |
files
|
1998-08-18 |
paulson |
new theorem diff_Suc_less_diff
|
changeset |
files
|
1998-08-17 |
wenzelm |
added get_tthmss;
|
changeset |
files
|
1998-08-17 |
nipkow |
Mention RegExp2NA.
|
changeset |
files
|
1998-08-17 |
paulson |
expandshort
|
changeset |
files
|
1998-08-17 |
paulson |
Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
|
changeset |
files
|
1998-08-17 |
paulson |
Now allows "." in rule names, with special treatment for "be"
|
changeset |
files
|
1998-08-17 |
nipkow |
Direct translation RegExp -> NA!
|
changeset |
files
|
1998-08-17 |
nipkow |
Additions to Lex.
|
changeset |
files
|
1998-08-14 |
paulson |
got rid of some goal thy commands
|
changeset |
files
|
1998-08-14 |
paulson |
now trans_tac is part of the claset...
|
changeset |
files
|
1998-08-14 |
paulson |
Moved Un_subset_iff and Int_subset_iff from UNITY to equalities.ML
|
changeset |
files
|
1998-08-14 |
paulson |
expandshort
|
changeset |
files
|
1998-08-14 |
paulson |
Uses Goal instead of "goal...thy" to avoid theory problems
|
changeset |
files
|
1998-08-13 |
paulson |
even more tidying of Goal commands
|
changeset |
files
|
1998-08-13 |
paulson |
tidying
|
changeset |
files
|
1998-08-13 |
paulson |
Moved the definition of s_u (as s) into the locale
|
changeset |
files
|
1998-08-13 |
paulson |
Constrains, Stable, Invariant...more of the substitution axiom, but Union
|
changeset |
files
|
1998-08-13 |
paulson |
simpler SELECT_GOAL no longer inserts a dummy parameter
|
changeset |
files
|
1998-08-13 |
paulson |
Rule mk_triv_goal for making instances of triv_goal
|
changeset |
files
|
1998-08-13 |
paulson |
Blast_tac is faster
|
changeset |
files
|
1998-08-13 |
paulson |
stac now handles definitions as well as equalities
|
changeset |
files
|
1998-08-13 |
paulson |
stac
|
changeset |
files
|
1998-08-12 |
oheimb |
minor adaption for SML/NJ
|
changeset |
files
|
1998-08-12 |
oheimb |
added theorems Id_o, o_Id
|
changeset |
files
|
1998-08-12 |
oheimb |
cleanup for Fun.thy:
|
changeset |
files
|
1998-08-12 |
oheimb |
the splitter is now defined as a functor
|
changeset |
files
|
1998-08-12 |
oheimb |
renamed mk_meta_eq to meta_eq
|
changeset |
files
|
1998-08-12 |
oheimb |
removed superfluous o_apply
|
changeset |
files
|
1998-08-12 |
oheimb |
streamlined proofs with new hoare_conseq1, hoare_conseq2
|
changeset |
files
|
1998-08-12 |
oheimb |
defined map_upd by translation via fun_upd
|
changeset |
files
|
1998-08-12 |
oheimb |
added Eps_eq
|
changeset |
files
|
1998-08-12 |
oheimb |
removed use_thys implied by use_thy "Main"
|
changeset |
files
|
1998-08-12 |
oheimb |
repaired proof of chfindom_monofun2cont
|
changeset |
files
|
1998-08-12 |
oheimb |
added length_Suc_conv, finite_set
|
changeset |
files
|
1998-08-12 |
oheimb |
replaced idt by pttrn in @filter
|
changeset |
files
|
1998-08-12 |
oheimb |
replaced split_etas by split_eta_proc
|
changeset |
files
|
1998-08-12 |
oheimb |
added ospec
|
changeset |
files
|
1998-08-12 |
oheimb |
minor correction: n must not be used as free variable
|
changeset |
files
|
1998-08-12 |
slotosch |
eliminated fabs,fapp.
|
changeset |
files
|