changeset 77138 | c8597292cd41 |
parent 69895 | 6b03a8cf092d |
--- a/src/HOL/Library/Product_Order.thy Mon Jan 30 10:15:01 2023 +0100 +++ b/src/HOL/Library/Product_Order.thy Mon Jan 30 15:24:17 2023 +0000 @@ -35,6 +35,9 @@ lemma Pair_le [simp]: "(a, b) \<le> (c, d) \<longleftrightarrow> a \<le> c \<and> b \<le> d" unfolding less_eq_prod_def by simp +lemma atLeastAtMost_prod_eq: "{a..b} = {fst a..fst b} \<times> {snd a..snd b}" + by (auto simp: less_eq_prod_def) + instance prod :: (preorder, preorder) preorder proof fix x y z :: "'a \<times> 'b"