# HG changeset patch # User huffman # Date 1288995328 25200 # Node ID adb22dbb5242d2b93ebe0ca53b6642c5114533a3 # Parent a26503ac7c877c8befa8c940139b56ba3d995f52 (infixl "<<" 55) -> (infix "<<" 50) diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/ConvexPD.thy --- a/src/HOLCF/ConvexPD.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/ConvexPD.thy Fri Nov 05 15:15:28 2010 -0700 @@ -33,7 +33,7 @@ unfolding convex_le_def by (fast intro: PDPlus_upper_mono PDPlus_lower_mono) lemma convex_le_PDUnit_PDUnit_iff [simp]: - "(PDUnit a \\ PDUnit b) = a \ b" + "(PDUnit a \\ PDUnit b) = (a \ b)" unfolding convex_le_def upper_le_def lower_le_def Rep_PDUnit by fast lemma convex_le_PDUnit_lemma1: diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/Library/Sum_Cpo.thy --- a/src/HOLCF/Library/Sum_Cpo.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/Library/Sum_Cpo.thy Fri Nov 05 15:15:28 2010 -0700 @@ -21,10 +21,10 @@ instance .. end -lemma Inl_below_Inl [simp]: "Inl x \ Inl y = x \ y" +lemma Inl_below_Inl [simp]: "Inl x \ Inl y \ x \ y" unfolding below_sum_def by simp -lemma Inr_below_Inr [simp]: "Inr x \ Inr y = x \ y" +lemma Inr_below_Inr [simp]: "Inr x \ Inr y \ x \ y" unfolding below_sum_def by simp lemma Inl_below_Inr [simp]: "\ Inl x \ Inr y" diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/LowerPD.thy --- a/src/HOLCF/LowerPD.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/LowerPD.thy Fri Nov 05 15:15:28 2010 -0700 @@ -43,7 +43,7 @@ unfolding lower_le_def Rep_PDPlus by fast lemma lower_le_PDUnit_PDUnit_iff [simp]: - "(PDUnit a \\ PDUnit b) = a \ b" + "(PDUnit a \\ PDUnit b) = (a \ b)" unfolding lower_le_def Rep_PDUnit by fast lemma lower_le_PDUnit_PDPlus_iff: diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/Porder.thy --- a/src/HOLCF/Porder.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/Porder.thy Fri Nov 05 15:15:28 2010 -0700 @@ -15,10 +15,10 @@ begin notation - below (infixl "<<" 55) + below (infix "<<" 50) notation (xsymbols) - below (infixl "\" 55) + below (infix "\" 50) lemma below_eq_trans: "\a \ b; b = c\ \ a \ c" by (rule subst) @@ -62,7 +62,7 @@ subsection {* Upper bounds *} -definition is_ub :: "'a set \ 'a \ bool" (infixl "<|" 55) where +definition is_ub :: "'a set \ 'a \ bool" (infix "<|" 55) where "S <| x \ (\y\S. y \ x)" lemma is_ubI: "(\x. x \ S \ x \ u) \ S <| u" @@ -94,7 +94,7 @@ subsection {* Least upper bounds *} -definition is_lub :: "'a set \ 'a \ bool" (infixl "<<|" 55) where +definition is_lub :: "'a set \ 'a \ bool" (infix "<<|" 55) where "S <<| x \ S <| x \ (\u. S <| u \ x \ u)" definition lub :: "'a set \ 'a" where diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/Sprod.thy --- a/src/HOLCF/Sprod.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/Sprod.thy Fri Nov 05 15:15:28 2010 -0700 @@ -151,18 +151,18 @@ lemma spair_sfst_ssnd: "(:sfst\p, ssnd\p:) = p" by (cases p, simp_all) -lemma below_sprod: "x \ y = (sfst\x \ sfst\y \ ssnd\x \ ssnd\y)" +lemma below_sprod: "(x \ y) = (sfst\x \ sfst\y \ ssnd\x \ ssnd\y)" by (simp add: Rep_sprod_simps sfst_def ssnd_def cont_Rep_sprod) lemma eq_sprod: "(x = y) = (sfst\x = sfst\y \ ssnd\x = ssnd\y)" by (auto simp add: po_eq_conv below_sprod) -lemma sfst_below_iff: "sfst\x \ y = x \ (:y, ssnd\x:)" +lemma sfst_below_iff: "sfst\x \ y \ x \ (:y, ssnd\x:)" apply (cases "x = \", simp, cases "y = \", simp) apply (simp add: below_sprod) done -lemma ssnd_below_iff: "ssnd\x \ y = x \ (:sfst\x, y:)" +lemma ssnd_below_iff: "ssnd\x \ y \ x \ (:sfst\x, y:)" apply (cases "x = \", simp, cases "y = \", simp) apply (simp add: below_sprod) done diff -r a26503ac7c87 -r adb22dbb5242 src/HOLCF/UpperPD.thy --- a/src/HOLCF/UpperPD.thy Wed Nov 03 17:22:25 2010 -0700 +++ b/src/HOLCF/UpperPD.thy Fri Nov 05 15:15:28 2010 -0700 @@ -42,7 +42,7 @@ unfolding upper_le_def Rep_PDPlus by fast lemma upper_le_PDUnit_PDUnit_iff [simp]: - "(PDUnit a \\ PDUnit b) = a \ b" + "(PDUnit a \\ PDUnit b) = (a \ b)" unfolding upper_le_def Rep_PDUnit by fast lemma upper_le_PDPlus_PDUnit_iff: