src/HOL/Real/HahnBanach/Bounds.thy
changeset 16417 9bc16273c2d4
parent 14653 0848ab6fe5fc
child 19736 d8d0f8f51d69
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     3     Author:     Gertrud Bauer, TU Munich
     3     Author:     Gertrud Bauer, TU Munich
     4 *)
     4 *)
     5 
     5 
     6 header {* Bounds *}
     6 header {* Bounds *}
     7 
     7 
     8 theory Bounds = Main + Real:
     8 theory Bounds imports Main Real begin
     9 
     9 
    10 locale lub =
    10 locale lub =
    11   fixes A and x
    11   fixes A and x
    12   assumes least [intro?]: "(\<And>a. a \<in> A \<Longrightarrow> a \<le> b) \<Longrightarrow> x \<le> b"
    12   assumes least [intro?]: "(\<And>a. a \<in> A \<Longrightarrow> a \<le> b) \<Longrightarrow> x \<le> b"
    13     and upper [intro?]: "a \<in> A \<Longrightarrow> a \<le> x"
    13     and upper [intro?]: "a \<in> A \<Longrightarrow> a \<le> x"