Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2019-12-12 09:05 69e861e9

View on Github →

feat(measure_theory/bochner_integration): connecting the Bochner integral with the integral on ennreal-valued functions (#1790)

  • shorter proof
  • feat(measure_theory/bochner_integration): connecting the Bochner integral with the integral on ennreal This PR proves that ∫ f = ∫ f⁺ - ∫ f⁻, with the first integral sign being the Bochner integral of a real-valued function f : α → ℝ, and second and third integral sign being the integral on ennreal-valued functions. See integral_eq_lintegral_max_sub_lintegral_min. I feel that most of the basic properties of the Bochner integral are proved. Please let me know if you think something else is needed.
  • various things :
  • add guides for typeclass inference;
  • add norm_cast tags;
  • prove some corollaries;
  • add doc strings;
  • other fixes
  • Update bochner_integration.lean
  • add some doc strings
  • Fix doc strings
  • Update bochner_integration.lean
  • Update bochner_integration.lean
  • fix doc strings
  • Update bochner_integration.lean
  • Use dot notation
  • use dot notation
  • Update Meas.lean

Estimated changes

added def borel
added theorem borel_comap
added theorem borel_eq_generate_Iio
added theorem borel_eq_generate_Ioi
added theorem borel_eq_subtype
added theorem borel_induced
added theorem borel_prod
added theorem borel_prod_le
added theorem ennreal.measurable.add
added theorem ennreal.measurable.mul
added theorem ennreal.measurable.sub
deleted theorem ennreal.measurable_add
deleted theorem ennreal.measurable_mul
deleted theorem ennreal.measurable_sub
added theorem is_measurable_Ico
added theorem is_measurable_Iio
added theorem is_measurable_Ioo
added theorem is_measurable_ball
added theorem is_measurable_closure
added theorem is_measurable_interior
added theorem is_measurable_le
added theorem measurable.add
added theorem measurable.infi
added theorem measurable.infi_Prop
added theorem measurable.is_glb
added theorem measurable.is_lub
added theorem measurable.max
added theorem measurable.min
added theorem measurable.mul
added theorem measurable.neg
added theorem measurable.sub
added theorem measurable.supr
added theorem measurable.supr_Prop
added theorem measurable_finset_sum
added theorem measurable_neg_iff
deleted theorem measure_theory.borel_prod
added theorem nnreal.measurable.add
added theorem nnreal.measurable.mul
added theorem nnreal.measurable.sub
deleted theorem nnreal.measurable_add
deleted theorem nnreal.measurable_mul
deleted theorem nnreal.measurable_sub
modified theorem measure_theory.l1.coe_add
modified theorem measure_theory.l1.coe_neg
modified theorem measure_theory.l1.coe_smul
modified theorem measure_theory.l1.coe_sub
modified theorem measure_theory.l1.coe_zero
added theorem measurable.fst
added theorem measurable.prod_mk
added theorem measurable.snd
added theorem measurable.subtype_mk
added theorem measurable.subtype_val
deleted theorem measurable_fst
deleted theorem measurable_prod_mk
deleted theorem measurable_snd
deleted theorem measurable_subtype_mk
deleted theorem measurable_subtype_val