src/HOL/Library/Extended_Real.thy
changeset 54863 82acc20ded73
parent 54416 7fb88ed6ff3c
child 55913 c1409c103b77
equal deleted inserted replaced
54862:c65e5cbdbc97 54863:82acc20ded73
  1620       proof (cases "\<forall>i. f i = 0")
  1620       proof (cases "\<forall>i. f i = 0")
  1621         case True
  1621         case True
  1622         then have "range f = {0}"
  1622         then have "range f = {0}"
  1623           by auto
  1623           by auto
  1624         with True show "c * SUPR UNIV f \<le> y"
  1624         with True show "c * SUPR UNIV f \<le> y"
  1625           using * by (auto simp: SUP_def min_max.sup_absorb1)
  1625           using * by (auto simp: SUP_def max.absorb1)
  1626       next
  1626       next
  1627         case False
  1627         case False
  1628         then obtain i where "f i \<noteq> 0"
  1628         then obtain i where "f i \<noteq> 0"
  1629           by auto
  1629           by auto
  1630         with *[of i] `c = \<infinity>` `0 \<le> f i` show ?thesis
  1630         with *[of i] `c = \<infinity>` `0 \<le> f i` show ?thesis
  1777   then show "Sup ((\<lambda>x. a + x) ` A) \<le> a + Sup A" .
  1777   then show "Sup ((\<lambda>x. a + x) ` A) \<le> a + Sup A" .
  1778   show "a + Sup A \<le> Sup ((\<lambda>x. a + x) ` A)"
  1778   show "a + Sup A \<le> Sup ((\<lambda>x. a + x) ` A)"
  1779   proof (cases a)
  1779   proof (cases a)
  1780     case PInf with `A \<noteq> {}`
  1780     case PInf with `A \<noteq> {}`
  1781     show ?thesis
  1781     show ?thesis
  1782       by (auto simp: image_constant min_max.sup_absorb1)
  1782       by (auto simp: image_constant max.absorb1)
  1783   next
  1783   next
  1784     case (real r)
  1784     case (real r)
  1785     then have **: "op + (- a) ` op + a ` A = A"
  1785     then have **: "op + (- a) ` op + a ` A = A"
  1786       by (auto simp: image_iff ac_simps zero_ereal_def[symmetric])
  1786       by (auto simp: image_iff ac_simps zero_ereal_def[symmetric])
  1787     from *[of "-a" "(\<lambda>x. a + x) ` A"] real show ?thesis
  1787     from *[of "-a" "(\<lambda>x. a + x) ` A"] real show ?thesis