src/HOL/Probability/Helly_Selection.thy
changeset 66453 cc19f7ca2ed6
parent 66447 a1f5c5c26fa6
child 67399 eab6ce8368fa
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     6 section \<open>Helly's selection theorem\<close>
     6 section \<open>Helly's selection theorem\<close>
     7 
     7 
     8 text \<open>The set of bounded, monotone, right continuous functions is sequentially compact\<close>
     8 text \<open>The set of bounded, monotone, right continuous functions is sequentially compact\<close>
     9 
     9 
    10 theory Helly_Selection
    10 theory Helly_Selection
    11   imports "~~/src/HOL/Library/Diagonal_Subsequence" Weak_Convergence
    11   imports "HOL-Library.Diagonal_Subsequence" Weak_Convergence
    12 begin
    12 begin
    13 
    13 
    14 lemma minus_one_less: "x - 1 < (x::real)"
    14 lemma minus_one_less: "x - 1 < (x::real)"
    15   by simp
    15   by simp
    16 
    16