wenzelm [Wed, 07 May 2008 12:38:55 +0200] rev 26840
added logic-specific sessions;
berghofe [Wed, 07 May 2008 10:59:54 +0200] rev 26839
Updated.
berghofe [Wed, 07 May 2008 10:59:53 +0200] rev 26838
Instantiated rule increasing_chain_adm_lemma in proof of flatstream_adm_lemma
to avoid problems with HO unification.
berghofe [Wed, 07 May 2008 10:59:52 +0200] rev 26837
Replaced instance declarations for sets by instance declarations for bool.
Together with the instance declarations for fun from Ffun, this subsumes the
old instance declarations for sets.
berghofe [Wed, 07 May 2008 10:59:51 +0200] rev 26836
Adm now imports Ffun rather than Cont, because SetPcpo, which imports Adm,
needs functions (since sets are now just functions).
berghofe [Wed, 07 May 2008 10:59:50 +0200] rev 26835
Lookup and union operations on terms are now modulo eta conversion.
berghofe [Wed, 07 May 2008 10:59:49 +0200] rev 26834
Terms returned by decomp are now eta-contracted.
berghofe [Wed, 07 May 2008 10:59:48 +0200] rev 26833
Added function for computing instantiation for the subst rule, which is used
in vars_gen_hyp_subst_tac and blast_hyp_subst_tac to avoid problems with
HO unification.
berghofe [Wed, 07 May 2008 10:59:47 +0200] rev 26832
eq_assumption now uses aeconv instead of aconv.
berghofe [Wed, 07 May 2008 10:59:46 +0200] rev 26831
- Removed function eta_contract_atom, which did not quite work
- Corrected and simplified function aeconv
berghofe [Wed, 07 May 2008 10:59:45 +0200] rev 26830
Replaced Pattern.eta_contract_atom by Envir.eta_contract.
berghofe [Wed, 07 May 2008 10:59:44 +0200] rev 26829
Removed instantiation for set.
berghofe [Wed, 07 May 2008 10:59:43 +0200] rev 26828
Explicitely applied ext in proof of tnd.
berghofe [Wed, 07 May 2008 10:59:42 +0200] rev 26827
Deleted subset_antisym in a few proofs, because it is
accidentally applied to predicates as well.
berghofe [Wed, 07 May 2008 10:59:41 +0200] rev 26826
- Tuned imports
- Replaced blast by simp in proof of Stable_final_E_NOT_empty, since blast looped
because of the new encoding of sets.
berghofe [Wed, 07 May 2008 10:59:40 +0200] rev 26825
Manually applied subset_antisym in proof of Compl_fixedpoint, because it is
accidentally applied to predicates as well.
berghofe [Wed, 07 May 2008 10:59:39 +0200] rev 26824
Replaced blast by fast in proof of INT_Un_Compl_subset, since blast looped
because of the new encoding of sets.
berghofe [Wed, 07 May 2008 10:59:38 +0200] rev 26823
Functions get_branching_types and get_arities now use fold instead of foldl/r.
berghofe [Wed, 07 May 2008 10:59:37 +0200] rev 26822
Temporarily disabled invocations of new code generator that do no
longer work due to the encoding of sets as predicates
berghofe [Wed, 07 May 2008 10:59:36 +0200] rev 26821
Replaced instance "set :: (plus) plus" by "fun :: (type, type) plus"
berghofe [Wed, 07 May 2008 10:59:35 +0200] rev 26820
- Deleted arity proofs for set
- Produce specific instances of theorems insert_eqvt, set_eqvt and perm_set_eq
berghofe [Wed, 07 May 2008 10:59:34 +0200] rev 26819
Replaced union_empty2 by Un_empty_right.
berghofe [Wed, 07 May 2008 10:59:33 +0200] rev 26818
Instantiated rule expand_fun_eq in proof of set_of_eq_empty_iff, to avoid that
it gets applied to sets as well.
berghofe [Wed, 07 May 2008 10:59:32 +0200] rev 26817
Deleted instance "set :: ({heap, finite}) heap"
berghofe [Wed, 07 May 2008 10:59:29 +0200] rev 26816
- Declared subset_eq as code lemma
- Deleted types_code declaration for sets
berghofe [Wed, 07 May 2008 10:59:27 +0200] rev 26815
Deleted instantiation "set :: (enum) enum"
berghofe [Wed, 07 May 2008 10:59:24 +0200] rev 26814
Replaced + and * on sets by \<oplus> and \<otimes>, to avoid clash with
definitions of + and * on functions.
berghofe [Wed, 07 May 2008 10:59:23 +0200] rev 26813
Rephrased calculational proofs to avoid problems with HO unification
berghofe [Wed, 07 May 2008 10:59:22 +0200] rev 26812
Rephrased forward proofs to avoid problems with HO unification
berghofe [Wed, 07 May 2008 10:59:21 +0200] rev 26811
Rephrased proof of ann_hoare_case_analysis, to avoid problems with HO unification