2008-05-08 |
wenzelm |
misc tuning;
|
changeset |
files
|
2008-05-08 |
urbanc |
slight tuning of the 1st paragraph
|
changeset |
files
|
2008-05-08 |
wenzelm |
unused;
|
changeset |
files
|
2008-05-08 |
wenzelm |
converted HOL specific elements;
|
changeset |
files
|
2008-05-08 |
wenzelm |
added rail setup for verblbrace, verbrbrace;
|
changeset |
files
|
2008-05-08 |
urbanc |
added at_set_avoiding lemmas
|
changeset |
files
|
2008-05-07 |
wenzelm |
removed obsolete conversion guide -- converted only section on tactics;
|
changeset |
files
|
2008-05-07 |
wenzelm |
converted ZF specific elements;
|
changeset |
files
|
2008-05-07 |
wenzelm |
enabled ThyOutput.source option by default;
|
changeset |
files
|
2008-05-07 |
wenzelm |
output_entity: ignore ThyOutput.source option;
|
changeset |
files
|
2008-05-07 |
wenzelm |
updated generated file;
|
changeset |
files
|
2008-05-07 |
wenzelm |
converted HOLCF specific elements;
|
changeset |
files
|
2008-05-07 |
wenzelm |
added logic-specific sessions;
|
changeset |
files
|
2008-05-07 |
berghofe |
Updated.
|
changeset |
files
|
2008-05-07 |
berghofe |
Instantiated rule increasing_chain_adm_lemma in proof of flatstream_adm_lemma
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced instance declarations for sets by instance declarations for bool.
|
changeset |
files
|
2008-05-07 |
berghofe |
Adm now imports Ffun rather than Cont, because SetPcpo, which imports Adm,
|
changeset |
files
|
2008-05-07 |
berghofe |
Lookup and union operations on terms are now modulo eta conversion.
|
changeset |
files
|
2008-05-07 |
berghofe |
Terms returned by decomp are now eta-contracted.
|
changeset |
files
|
2008-05-07 |
berghofe |
Added function for computing instantiation for the subst rule, which is used
|
changeset |
files
|
2008-05-07 |
berghofe |
eq_assumption now uses aeconv instead of aconv.
|
changeset |
files
|
2008-05-07 |
berghofe |
- Removed function eta_contract_atom, which did not quite work
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced Pattern.eta_contract_atom by Envir.eta_contract.
|
changeset |
files
|
2008-05-07 |
berghofe |
Removed instantiation for set.
|
changeset |
files
|
2008-05-07 |
berghofe |
Explicitely applied ext in proof of tnd.
|
changeset |
files
|
2008-05-07 |
berghofe |
Deleted subset_antisym in a few proofs, because it is
|
changeset |
files
|
2008-05-07 |
berghofe |
- Tuned imports
|
changeset |
files
|
2008-05-07 |
berghofe |
Manually applied subset_antisym in proof of Compl_fixedpoint, because it is
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced blast by fast in proof of INT_Un_Compl_subset, since blast looped
|
changeset |
files
|
2008-05-07 |
berghofe |
Functions get_branching_types and get_arities now use fold instead of foldl/r.
|
changeset |
files
|
2008-05-07 |
berghofe |
Temporarily disabled invocations of new code generator that do no
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced instance "set :: (plus) plus" by "fun :: (type, type) plus"
|
changeset |
files
|
2008-05-07 |
berghofe |
- Deleted arity proofs for set
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced union_empty2 by Un_empty_right.
|
changeset |
files
|
2008-05-07 |
berghofe |
Instantiated rule expand_fun_eq in proof of set_of_eq_empty_iff, to avoid that
|
changeset |
files
|
2008-05-07 |
berghofe |
Deleted instance "set :: ({heap, finite}) heap"
|
changeset |
files
|
2008-05-07 |
berghofe |
- Declared subset_eq as code lemma
|
changeset |
files
|
2008-05-07 |
berghofe |
Deleted instantiation "set :: (enum) enum"
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced + and * on sets by \<oplus> and \<otimes>, to avoid clash with
|
changeset |
files
|
2008-05-07 |
berghofe |
Rephrased calculational proofs to avoid problems with HO unification
|
changeset |
files
|
2008-05-07 |
berghofe |
Rephrased forward proofs to avoid problems with HO unification
|
changeset |
files
|
2008-05-07 |
berghofe |
Rephrased proof of ann_hoare_case_analysis, to avoid problems with HO unification
|
changeset |
files
|
2008-05-07 |
berghofe |
Locally deleted some definitions that were applied too eagerly because
|
changeset |
files
|
2008-05-07 |
berghofe |
- Instantiated parts_insert_substD to avoid problems with HO unification
|
changeset |
files
|
2008-05-07 |
berghofe |
Instantiated parts_insert_substD to avoid problems with HO unification
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced blast by fast in proof of parts_singleton, since blast looped
|
changeset |
files
|
2008-05-07 |
berghofe |
Adapted to encoding of sets as predicates
|
changeset |
files
|
2008-05-07 |
berghofe |
Replaced forward proofs of existential statements by backward proofs
|
changeset |
files
|
2008-05-07 |
berghofe |
Adapted functions mk_setT and dest_setT to encoding of sets as predicates.
|
changeset |
files
|
2008-05-07 |
berghofe |
- Explicitely passed pred_subset_eq and pred_equals_eq as an argument to the
|
changeset |
files
|
2008-05-07 |
berghofe |
Deleted instantiation "set :: (type) itself".
|
changeset |
files
|
2008-05-07 |
berghofe |
- Function dec in Trancl_Tac must eta-contract relation before calling
|
changeset |
files
|
2008-05-07 |
berghofe |
- Now uses Orderings as parent theory
|
changeset |
files
|
2008-05-07 |
berghofe |
Deleted instance "set :: (type) power" and moved instance
|
changeset |
files
|
2008-05-07 |
berghofe |
split_beta is now declared as monotonicity rule, to allow bounded
|
changeset |
files
|
2008-05-07 |
berghofe |
- Added mem_def and predicate1I in some of the proofs
|
changeset |
files
|
2008-05-07 |
berghofe |
- Now imports Code_Setup, rather than Set and Fun, since the theorems
|
changeset |
files
|
2008-05-07 |
berghofe |
- Explicitely applied predicate1I in a few proofs, because it is no longer
|
changeset |
files
|
2008-05-07 |
berghofe |
- Now imports Fun rather than Orderings
|
changeset |
files
|
2008-05-07 |
berghofe |
Instantiated some rules to avoid problems with HO unification.
|
changeset |
files
|