src/HOL/Orderings.thy
changeset 54857 5c05f7c5f8ae
parent 54147 97a8ff4e4ac9
child 54860 69b3e46d8fbe
equal deleted inserted replaced
54856:356b4c0a2061 54857:5c05f7c5f8ae
  1153 end
  1153 end
  1154 
  1154 
  1155 lemma min_absorb1: "x \<le> y \<Longrightarrow> min x y = x"
  1155 lemma min_absorb1: "x \<le> y \<Longrightarrow> min x y = x"
  1156 by (simp add: min_def)
  1156 by (simp add: min_def)
  1157 
  1157 
  1158 lemma max_absorb2: "x \<le> y ==> max x y = y"
  1158 lemma max_absorb2: "x \<le> y \<Longrightarrow> max x y = y"
  1159 by (simp add: max_def)
  1159 by (simp add: max_def)
  1160 
  1160 
  1161 lemma min_absorb2: "(y\<Colon>'a\<Colon>order) \<le> x \<Longrightarrow> min x y = y"
  1161 lemma min_absorb2: "(y\<Colon>'a\<Colon>order) \<le> x \<Longrightarrow> min x y = y"
  1162 by (simp add:min_def)
  1162 by (simp add:min_def)
  1163 
  1163