Wed, 07 May 2008 10:59:37 +0200 Temporarily disabled invocations of new code generator that do no
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
Wed, 07 May 2008 10:59:36 +0200 Replaced instance "set :: (plus) plus" by "fun :: (type, type) plus"
berghofe [Wed, 07 May 2008 10:59:36 +0200] rev 26821
Replaced instance "set :: (plus) plus" by "fun :: (type, type) plus"
Wed, 07 May 2008 10:59:35 +0200 - Deleted arity proofs for set
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
Wed, 07 May 2008 10:59:34 +0200 Replaced union_empty2 by Un_empty_right.
berghofe [Wed, 07 May 2008 10:59:34 +0200] rev 26819
Replaced union_empty2 by Un_empty_right.
Wed, 07 May 2008 10:59:33 +0200 Instantiated rule expand_fun_eq in proof of set_of_eq_empty_iff, to avoid that
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.
Wed, 07 May 2008 10:59:32 +0200 Deleted instance "set :: ({heap, finite}) heap"
berghofe [Wed, 07 May 2008 10:59:32 +0200] rev 26817
Deleted instance "set :: ({heap, finite}) heap"
Wed, 07 May 2008 10:59:29 +0200 - Declared subset_eq as code lemma
berghofe [Wed, 07 May 2008 10:59:29 +0200] rev 26816
- Declared subset_eq as code lemma - Deleted types_code declaration for sets
Wed, 07 May 2008 10:59:27 +0200 Deleted instantiation "set :: (enum) enum"
berghofe [Wed, 07 May 2008 10:59:27 +0200] rev 26815
Deleted instantiation "set :: (enum) enum"
Wed, 07 May 2008 10:59:24 +0200 Replaced + and * on sets by \<oplus> and \<otimes>, to avoid clash with
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.
Wed, 07 May 2008 10:59:23 +0200 Rephrased calculational proofs to avoid problems with HO unification
berghofe [Wed, 07 May 2008 10:59:23 +0200] rev 26813
Rephrased calculational proofs to avoid problems with HO unification
Wed, 07 May 2008 10:59:22 +0200 Rephrased forward 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
Wed, 07 May 2008 10:59:21 +0200 Rephrased proof of ann_hoare_case_analysis, 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
Wed, 07 May 2008 10:59:20 +0200 Locally deleted some definitions that were applied too eagerly because
berghofe [Wed, 07 May 2008 10:59:20 +0200] rev 26810
Locally deleted some definitions that were applied too eagerly because of eta-expansion
Wed, 07 May 2008 10:59:19 +0200 - Instantiated parts_insert_substD to avoid problems with HO unification
berghofe [Wed, 07 May 2008 10:59:19 +0200] rev 26809
- Instantiated parts_insert_substD to avoid problems with HO unification - Replaced auto by fastsimp in proof of parts_invKey, since auto looped because of the new encoding of sets
Wed, 07 May 2008 10:59:18 +0200 Instantiated parts_insert_substD to avoid problems with HO unification
berghofe [Wed, 07 May 2008 10:59:18 +0200] rev 26808
Instantiated parts_insert_substD to avoid problems with HO unification
Wed, 07 May 2008 10:59:02 +0200 Replaced blast by fast in proof of parts_singleton, since blast looped
berghofe [Wed, 07 May 2008 10:59:02 +0200] rev 26807
Replaced blast by fast in proof of parts_singleton, since blast looped because of the new encoding of sets.
Wed, 07 May 2008 10:57:19 +0200 Adapted to encoding of sets as predicates
berghofe [Wed, 07 May 2008 10:57:19 +0200] rev 26806
Adapted to encoding of sets as predicates
Wed, 07 May 2008 10:56:58 +0200 Replaced forward proofs of existential statements by backward proofs
berghofe [Wed, 07 May 2008 10:56:58 +0200] rev 26805
Replaced forward proofs of existential statements by backward proofs to avoid problems with HO unification
Wed, 07 May 2008 10:56:55 +0200 Adapted functions mk_setT and dest_setT to encoding of sets as predicates.
berghofe [Wed, 07 May 2008 10:56:55 +0200] rev 26804
Adapted functions mk_setT and dest_setT to encoding of sets as predicates.
Wed, 07 May 2008 10:56:52 +0200 - Explicitely passed pred_subset_eq and pred_equals_eq as an argument to the
berghofe [Wed, 07 May 2008 10:56:52 +0200] rev 26803
- Explicitely passed pred_subset_eq and pred_equals_eq as an argument to the to_set and to_pred attributes, because it is no longer applied automatically - Manually applied predicate1I in proof of accp_subset, because it is no longer part of the claset - Replaced psubset_def by less_le
Wed, 07 May 2008 10:56:50 +0200 Deleted instantiation "set :: (type) itself".
berghofe [Wed, 07 May 2008 10:56:50 +0200] rev 26802
Deleted instantiation "set :: (type) itself".
Wed, 07 May 2008 10:56:49 +0200 - Function dec in Trancl_Tac must eta-contract relation before calling
berghofe [Wed, 07 May 2008 10:56:49 +0200] rev 26801
- Function dec in Trancl_Tac must eta-contract relation before calling decr, since it is now a function and could therefore be in eta-expanded form - The trancl prover now does more eta-contraction itself, so eta-contraction is no longer necessary in Tranclp_tac.
Wed, 07 May 2008 10:56:43 +0200 - Now uses Orderings as parent theory
berghofe [Wed, 07 May 2008 10:56:43 +0200] rev 26800
- Now uses Orderings as parent theory - "'a set" is now just a type abbreviation for "'a => bool" - The instantiation "set :: (type) ord" and the definition of (p)subset is no longer needed, since it is subsumed by the order on functions and booleans. The derived theorems (p)subset_eq can be used as a replacement. - mem_Collect_eq and Collect_mem_eq can now be derived from the definitions of mem and Collect. - Replaced the instantiation "set :: (type) minus" by the two instantiations "fun :: (type, minus) minus" and "bool :: minus". The theorem set_diff_eq can be used as a replacement for the definition set_diff_def - Replaced the instantiation "set :: (type) uminus" by the two instantiations "fun :: (type, uminus) uminus" and "bool :: uminus". The theorem Compl_eq can be used as a replacement for the definition Compl_def. - Variable P in rule split_if must be instantiated manually in proof of split_if_mem2 due to problems with HO unification - Moved definition of dense linear orders and proofs about LEAST from Orderings to Set - Deleted code setup for sets
Wed, 07 May 2008 10:56:41 +0200 Deleted instance "set :: (type) power" and moved instance
berghofe [Wed, 07 May 2008 10:56:41 +0200] rev 26799
Deleted instance "set :: (type) power" and moved instance "fun :: (type, type) power" to the beginning of the theory
Wed, 07 May 2008 10:56:40 +0200 split_beta is now declared as monotonicity rule, to allow bounded
berghofe [Wed, 07 May 2008 10:56:40 +0200] rev 26798
split_beta is now declared as monotonicity rule, to allow bounded quantifiers in introduction rules of inductive predicates.
Wed, 07 May 2008 10:56:39 +0200 - Added mem_def and predicate1I in some of the proofs
berghofe [Wed, 07 May 2008 10:56:39 +0200] rev 26797
- Added mem_def and predicate1I in some of the proofs - pred_equals_eq and pred_subset_eq are no longer used in the conversion between sets and predicates, because sets and predicates can no longer be distinguished
Wed, 07 May 2008 10:56:38 +0200 - Now imports Code_Setup, rather than Set and Fun, since the theorems
berghofe [Wed, 07 May 2008 10:56:38 +0200] rev 26796
- Now imports Code_Setup, rather than Set and Fun, since the theorems about orderings are already needed in Set - Moved "Dense orders" section to Set, since it requires set notation. - The "Order on sets" section is no longer necessary, since it is subsumed by the order on functions and booleans. - Moved proofs of Least_mono and Least_equality to Set, since they require set notation. - In proof of "instance fun :: (type, order) order", use ext instead of expand_fun_eq, since the latter is not yet available. - predicate1I is no longer declared as introduction rule, since it interferes with subsetI
Wed, 07 May 2008 10:56:37 +0200 - Explicitely applied predicate1I in a few proofs, because it is no longer
berghofe [Wed, 07 May 2008 10:56:37 +0200] rev 26795
- Explicitely applied predicate1I in a few proofs, because it is no longer part of the claset - Explicitely passed pred_subset_eq and pred_equals_eq as an argument to the to_set attribute, because it is no longer applied automatically
Wed, 07 May 2008 10:56:36 +0200 - Now imports Fun rather than Orderings
berghofe [Wed, 07 May 2008 10:56:36 +0200] rev 26794
- Now imports Fun rather than Orderings - Moved "Set as lattice" section behind "Fun as lattice" section, since sets are just functions. - The instantiations instantiation set :: (type) distrib_lattice instantiation set :: (type) complete_lattice are no longer needed, and the former definitions inf_set_eq, sup_set_eq, Inf_set_def, and Sup_set_def can now be derived from abstract properties of sup, inf, etc.
Wed, 07 May 2008 10:56:35 +0200 Instantiated some rules to avoid problems with HO unification.
berghofe [Wed, 07 May 2008 10:56:35 +0200] rev 26793
Instantiated some rules to avoid problems with HO unification.
(0) -10000 -3000 -1000 -300 -100 -50 -30 +30 +50 +100 +300 +1000 +3000 +10000 +30000 tip