src/HOL/Orderings.thy
changeset 82690 cccbfa567117
parent 82593 88043331f166
child 82695 d93ead9ac6df
equal deleted inserted replaced
82689:817f97d8cd26 82690:cccbfa567117
  1390   { fix m assume m: "m < ?x"
  1390   { fix m assume m: "m < ?x"
  1391     from not_less_Least[OF m] have "\<not> P m" . }
  1391     from not_less_Least[OF m] have "\<not> P m" . }
  1392   with LeastI_ex[OF H] show ?rhs by blast
  1392   with LeastI_ex[OF H] show ?rhs by blast
  1393 qed
  1393 qed
  1394 
  1394 
       
  1395 lemma exists_least_iff': 
       
  1396   shows "(\<exists>n. P n) \<longleftrightarrow> P (Least P) \<and> (\<forall>m < (Least P). \<not> P m)"
       
  1397   using LeastI_ex not_less_Least by auto
       
  1398 
  1395 end
  1399 end
  1396 
  1400 
  1397 
  1401 
  1398 subsection \<open>Order on \<^typ>\<open>bool\<close>\<close>
  1402 subsection \<open>Order on \<^typ>\<open>bool\<close>\<close>
  1399 
  1403