# HG changeset patch # User haftmann # Date 1310925317 -7200 # Node ID 771014555553d94e5d47af05811f923523154f41 # Parent 8a50dc70cbff81818387d8b20cb972bf2ab88768 generalized INT_anti_mono diff -r 8a50dc70cbff -r 771014555553 src/HOL/Complete_Lattice.thy --- a/src/HOL/Complete_Lattice.thy Sun Jul 17 19:48:02 2011 +0200 +++ b/src/HOL/Complete_Lattice.thy Sun Jul 17 19:55:17 2011 +0200 @@ -533,8 +533,6 @@ "u \ A \ (\x\A. insert a (B x)) = insert a (\x\A. B x)" by blast --- {* continue generalization from here *} - lemma (in complete_lattice) INF_constant: "(\y\A. c) = (if A = {} then \ else c)" by (simp add: INF_empty) @@ -572,14 +570,14 @@ by (fact INF_bool_eq) lemma (in complete_lattice) INF_anti_mono: - "B \ A \ (\x. x \ A \ f x \ g x) \ (\x\A. f x) \ (\x\A. g x)" + "B \ A \ (\x. x \ A \ f x \ g x) \ (\x\B. f x) \ (\x\B. g x)" -- {* The last inclusion is POSITIVE! *} - by (blast dest: subsetD) + by (blast intro: INF_mono dest: subsetD) lemma INT_anti_mono: - "B \ A \ (\x. x \ A \ f x \ g x) \ (\x\A. f x) \ (\x\A. g x)" + "B \ A \ (\x. x \ A \ f x \ g x) \ (\x\B. f x) \ (\x\B. g x)" -- {* The last inclusion is POSITIVE! *} - by (blast dest: subsetD) + by (fact INF_anti_mono) lemma Pow_INT_eq: "Pow (\x\A. B x) = (\x\A. Pow (B x))" by blast