Zulip Chat Archive

Stream: general

Topic: dsimp killing notations


Patrick Massot (Nov 03 2021 at 15:25):

In

import measure_theory.integral.interval_integral

open topological_space

variables {E : Type*} [normed_group E] [normed_space  E]
          [complete_space E] [second_countable_topology E]
          [measurable_space E] [borel_space E]

example (f :   E) (a b : ) :  t in a..b, f t = 0 :=
begin
  dsimp, -- new goal is: interval_integral f a b measure_theory.measure_space.volume
  sorry
end

Does anyone understand why dsimp is killing the notation?

Floris van Doorn (Nov 03 2021 at 15:27):

Probably because it reduces λ t, f t to f.

Patrick Massot (Nov 03 2021 at 15:32):

This sounds plausible indeed. Do you see any way to prevent that?

Patrick Massot (Nov 03 2021 at 15:35):

Maybe we should add something like

notation `∫_` a `..` b `, ` f ` ∂` μ:70 := interval_integral f a b μ
notation `∫_` a `..` b `, ` f:70 := interval_integral f a b measure_theory.measure_space.volume

Kyle Miller (Nov 03 2021 at 16:17):

Does dsimp { beta := ff } prevent it?

Kyle Miller (Nov 03 2021 at 16:18):

It doesn't prevent it.

Kyle Miller (Nov 03 2021 at 16:19):

Oh, I should have paid more attention to Floris's reduction: dsimp {eta := ff} prevents it.


Last updated: Dec 20 2023 at 11:08 UTC