src/HOL/Probability/Stopping_Time.thy
changeset 67226 ec32cdaab97b
parent 66453 cc19f7ca2ed6
child 69313 b021008c5397
equal deleted inserted replaced
67225:cb34f5f49a08 67226:ec32cdaab97b
     1 (* Author: Johannes Hölzl <hoelzl@in.tum.de> *)
     1 (* Author: Johannes Hölzl <hoelzl@in.tum.de> *)
     2 
     2 
     3 section {* Stopping times *}
     3 section \<open>Stopping times\<close>
     4 
     4 
     5 theory Stopping_Time
     5 theory Stopping_Time
     6   imports "HOL-Analysis.Analysis"
     6   imports "HOL-Analysis.Analysis"
     7 begin
     7 begin
     8 
     8