Skip to content

Commit

Permalink
Fixed duplicated theorems after the forbidden "rebinds" changes
Browse files Browse the repository at this point in the history
  • Loading branch information
binghe authored and mn200 committed Sep 8, 2023
1 parent 705d331 commit 64b350e
Show file tree
Hide file tree
Showing 3 changed files with 12 additions and 14 deletions.
11 changes: 6 additions & 5 deletions src/probability/measureScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -5446,7 +5446,7 @@ val _ = reveal "C";

(*** measure_space Theorems ***)

Theorem measure_space_eq' : (* was: measure_space_measure_eq *)
Theorem measure_space_measure_eq :
!sp sts u v. measure_space (sp,sts,u) /\ (!s. s IN sts ==> u s = v s) ==>
measure_space (sp,sts,v)
Proof
Expand All @@ -5460,10 +5460,10 @@ Theorem measure_space_cong:
(measure_space (sp,sts,u) <=> measure_space (sp,sts,v))
Proof
rw[] >> eq_tac >> rw[]
>> dxrule_at_then (Pos $ el 1) irule measure_space_eq' >> simp[]
>> dxrule_at_then (Pos $ el 1) irule measure_space_measure_eq >> simp[]
QED

Theorem measure_space_add:
Theorem measure_space_add':
!a mu nu p. measure_space (space a,subsets a,mu) /\
measure_space (space a,subsets a,nu) /\
(!s. s IN subsets a ==> p s = mu s + nu s) ==>
Expand All @@ -5489,11 +5489,12 @@ Proof
measure_space (space a,subsets a,m)’ suffices_by (rw[] >>
last_x_assum $ drule_then assume_tac >> pop_assum $ drule_all_then assume_tac >> simp[]) >>
Induct_on ‘s’ >> rw[]
>- (fs[EXTREAL_SUM_IMAGE_EMPTY] >> irule measure_space_eq' \\
>- (fs[EXTREAL_SUM_IMAGE_EMPTY] >> irule measure_space_measure_eq \\
qexists_tac ‘K 0’ >> simp[] >> dxrule_then assume_tac measure_space_trivial >>
fs[sigma_finite_measure_space_def,K_DEF]) >>
last_x_assum $ qspecl_then [‘a’,‘f’,‘\t. EXTREAL_SUM_IMAGE (C f t) s’] assume_tac >> rfs[] >>
irule measure_space_add >> qexistsl_tac [‘f e’,‘(\t. EXTREAL_SUM_IMAGE (C f t) s)’] >>
irule measure_space_add' >>
qexistsl_tac [‘f e’,‘(\t. EXTREAL_SUM_IMAGE (C f t) s)’] >>
simp[] >> qx_gen_tac ‘t’ >> rw[] >>
qspecl_then [‘C f t’,‘s’,‘e’]
(fn th => assume_tac th >> rfs[DELETE_NON_ELEMENT_RWT] >> pop_assum irule) $
Expand Down
9 changes: 6 additions & 3 deletions src/probability/real_borelScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -1489,8 +1489,11 @@ Proof
>> FIRST_X_ASSUM MATCH_MP_TAC >> art []
QED

(* cf. borelTheory.in_borel_measurable_imp' for measure_space version *)
Theorem in_borel_measurable_open :
(* cf. borelTheory.in_borel_measurable_imp' for measure_space version
NOTE: theorem renamed due to name conflicts with HVG's work.
*)
Theorem in_borel_measurable_open_imp : (* was: in_borel_measurable_open *)
!a f. sigma_algebra a /\
(!s. open s ==> (PREIMAGE f s) INTER space a IN subsets a) ==>
f IN measurable a borel
Expand All @@ -1506,7 +1509,7 @@ Theorem in_borel_measurable_continuous_on : (* was: borel_measurable_continuous_
!f. f continuous_on UNIV ==> f IN measurable borel borel
Proof
rpt STRIP_TAC
>> MATCH_MP_TAC in_borel_measurable_open
>> MATCH_MP_TAC in_borel_measurable_open_imp
>> rw [sigma_algebra_borel]
>> Know `open {x | x IN UNIV /\ f x IN s}`
>- (MATCH_MP_TAC CONTINUOUS_OPEN_PREIMAGE (* key lemma *) \\
Expand Down
6 changes: 0 additions & 6 deletions src/real/analysis/integrationScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -18860,12 +18860,6 @@ val HAS_BOUNDED_VARIATION_ON_REFLECT_INTERVAL = store_thm ("HAS_BOUNDED_VARIATIO
REPEAT STRIP_TAC THEN MATCH_MP_TAC HAS_BOUNDED_VARIATION_ON_REFLECT THEN
ASM_REWRITE_TAC[REFLECT_INTERVAL]);

val VECTOR_VARIATION_REFLECT_INTERVAL = store_thm ("VECTOR_VARIATION_REFLECT_INTERVAL",
``!f:real->real a b.
vector_variation (interval[a,b]) (\x. f(-x)) =
vector_variation (interval[-b,-a]) f``,
REWRITE_TAC[VECTOR_VARIATION_REFLECT, REFLECT_INTERVAL]);

val HAS_BOUNDED_VARIATION_COMPOSE_DECREASING = store_thm ("HAS_BOUNDED_VARIATION_COMPOSE_DECREASING",
``!f g:real->real a b.
(!x y. x IN interval[a,b] /\ y IN interval[a,b] /\ x <= y
Expand Down

0 comments on commit 64b350e

Please sign in to comment.