src/HOL/Hahn_Banach/Bounds.thy
changeset 58744 c434e37f290e
parent 54263 c4159fe6fa46
child 58745 5d452cf4bce7
equal deleted inserted replaced
58743:c07a59140fee 58744:c434e37f290e
     1 (*  Title:      HOL/Hahn_Banach/Bounds.thy
     1 (*  Title:      HOL/Hahn_Banach/Bounds.thy
     2     Author:     Gertrud Bauer, TU Munich
     2     Author:     Gertrud Bauer, TU Munich
     3 *)
     3 *)
     4 
     4 
     5 header {* Bounds *}
     5 header \<open>Bounds\<close>
     6 
     6 
     7 theory Bounds
     7 theory Bounds
     8 imports Main "~~/src/HOL/Library/ContNotDenum"
     8 imports Main "~~/src/HOL/Library/ContNotDenum"
     9 begin
     9 begin
    10 
    10 
    26   shows "\<Squnion>A = (x::'a::order)"
    26   shows "\<Squnion>A = (x::'a::order)"
    27 proof -
    27 proof -
    28   interpret lub A x by fact
    28   interpret lub A x by fact
    29   show ?thesis
    29   show ?thesis
    30   proof (unfold the_lub_def)
    30   proof (unfold the_lub_def)
    31     from `lub A x` show "The (lub A) = x"
    31     from \<open>lub A x\<close> show "The (lub A) = x"
    32     proof
    32     proof
    33       fix x' assume lub': "lub A x'"
    33       fix x' assume lub': "lub A x'"
    34       show "x' = x"
    34       show "x' = x"
    35       proof (rule order_antisym)
    35       proof (rule order_antisym)
    36         from lub' show "x' \<le> x"
    36         from lub' show "x' \<le> x"