src/HOL/Import/HOL4Compat.thy
changeset 44690 b6d8b11ed399
parent 41550 efa734d9b221
child 44740 a2940bc24bad
equal deleted inserted replaced
44681:49ef76b4a634 44690:b6d8b11ed399
   419   assume allx: "ALL x. P x \<longrightarrow> 0 < x"
   419   assume allx: "ALL x. P x \<longrightarrow> 0 < x"
   420   assume px: "P x"
   420   assume px: "P x"
   421   assume allx': "ALL x. P x \<longrightarrow> x < z"
   421   assume allx': "ALL x. P x \<longrightarrow> x < z"
   422   have "EX s. ALL y. (EX x : Collect P. y < x) = (y < s)"
   422   have "EX s. ALL y. (EX x : Collect P. y < x) = (y < s)"
   423   proof (rule posreal_complete)
   423   proof (rule posreal_complete)
   424     show "ALL x : Collect P. 0 < x"
       
   425     proof safe
       
   426       fix x
       
   427       assume P: "P x"
       
   428       from allx
       
   429       have "P x \<longrightarrow> 0 < x"
       
   430         ..
       
   431       with P show "0 < x" by simp
       
   432     qed
       
   433   next
       
   434     from px
   424     from px
   435     show "EX x. x : Collect P"
   425     show "EX x. x : Collect P"
   436       by auto
   426       by auto
   437   next
   427   next
   438     from allx'
   428     from allx'