src/HOL/Conditionally_Complete_Lattices.thy
changeset 69593 3dda49e08b9d
parent 69275 9bbd5497befd
child 69611 42cc3609fedf
equal deleted inserted replaced
69592:a80d8ec6c998 69593:3dda49e08b9d
   168 end
   168 end
   169 
   169 
   170 
   170 
   171 text \<open>
   171 text \<open>
   172 
   172 
   173 To avoid name classes with the @{class complete_lattice}-class we prefix @{const Sup} and
   173 To avoid name classes with the \<^class>\<open>complete_lattice\<close>-class we prefix \<^const>\<open>Sup\<close> and
   174 @{const Inf} in theorem names with c.
   174 \<^const>\<open>Inf\<close> in theorem names with c.
   175 
   175 
   176 \<close>
   176 \<close>
   177 
   177 
   178 class conditionally_complete_lattice = lattice + Sup + Inf +
   178 class conditionally_complete_lattice = lattice + Sup + Inf +
   179   assumes cInf_lower: "x \<in> X \<Longrightarrow> bdd_below X \<Longrightarrow> Inf X \<le> x"
   179   assumes cInf_lower: "x \<in> X \<Longrightarrow> bdd_below X \<Longrightarrow> Inf X \<le> x"