doc-src/Locales/Locales/Examples.thy
changeset 46855 f72a2bedd7a9
parent 37206 7f2a6f3143ad
equal deleted inserted replaced
46854:940dbfd43dc4 46855:f72a2bedd7a9
   191 
   191 
   192   This style of working is illustrated in the block below, where
   192   This style of working is illustrated in the block below, where
   193   notions of infimum and supremum for partial orders are introduced,
   193   notions of infimum and supremum for partial orders are introduced,
   194   together with theorems about their uniqueness.  *}
   194   together with theorems about their uniqueness.  *}
   195 
   195 
   196   context partial_order begin
   196   context partial_order
       
   197   begin
   197 
   198 
   198   definition
   199   definition
   199     is_inf where "is_inf x y i =
   200     is_inf where "is_inf x y i =
   200       (i \<sqsubseteq> x \<and> i \<sqsubseteq> y \<and> (\<forall>z. z \<sqsubseteq> x \<and> z \<sqsubseteq> y \<longrightarrow> z \<sqsubseteq> i))"
   201       (i \<sqsubseteq> x \<and> i \<sqsubseteq> y \<and> (\<forall>z. z \<sqsubseteq> x \<and> z \<sqsubseteq> y \<longrightarrow> z \<sqsubseteq> i))"
   201 
   202