src/HOL/Probability/Projective_Limit.thy
changeset 63885 a6cd18af8bf9
parent 63626 44ce6b524ff3
child 63918 6bf55e6e0b75
equal deleted inserted replaced
63884:d588f684ccaf 63885:a6cd18af8bf9
   453 end
   453 end
   454 
   454 
   455 hide_const (open) PiF
   455 hide_const (open) PiF
   456 hide_const (open) Pi\<^sub>F
   456 hide_const (open) Pi\<^sub>F
   457 hide_const (open) Pi'
   457 hide_const (open) Pi'
   458 hide_const (open) Abs_finmap
       
   459 hide_const (open) Rep_finmap
       
   460 hide_const (open) finmap_of
   458 hide_const (open) finmap_of
   461 hide_const (open) proj
   459 hide_const (open) proj
   462 hide_const (open) domain
   460 hide_const (open) domain
   463 hide_const (open) basis_finmap
   461 hide_const (open) basis_finmap
   464 
   462 
   475 
   473 
   476 locale polish_product_prob_space =
   474 locale polish_product_prob_space =
   477   product_prob_space "\<lambda>_. borel::('a::polish_space) measure" I for I::"'i set"
   475   product_prob_space "\<lambda>_. borel::('a::polish_space) measure" I for I::"'i set"
   478 
   476 
   479 sublocale polish_product_prob_space \<subseteq> P: polish_projective I "\<lambda>J. PiM J (\<lambda>_. borel::('a) measure)"
   477 sublocale polish_product_prob_space \<subseteq> P: polish_projective I "\<lambda>J. PiM J (\<lambda>_. borel::('a) measure)"
   480 proof qed
   478   ..
   481 
   479 
   482 lemma (in polish_product_prob_space) limP_eq_PiM: "lim = PiM I (\<lambda>_. borel)"
   480 lemma (in polish_product_prob_space) limP_eq_PiM: "lim = PiM I (\<lambda>_. borel)"
   483   by (rule PiM_eq) (auto simp: emeasure_PiM emeasure_lim_emb)
   481   by (rule PiM_eq) (auto simp: emeasure_PiM emeasure_lim_emb)
   484 
   482 
   485 end
   483 end