Zulip Chat Archive

Stream: mathlib4

Topic: simpa


Patrick Massot (Apr 27 2023 at 15:53):

I'm sure this has been discussed before, but did we loose simpa as an abbreviation of simpa using this on purpose?

Patrick Massot (Apr 28 2023 at 15:29):

After some more investigation, simpa indeed does something with this, but not the expected thing (expected based on Lean 3 behavior). In Lean 3:

import logic.basic
import tactic.simpa

example (P : Prop) (h : ¬ ¬ P) : P :=
begin
  have : ¬ ¬ P := h,
  simpa,
end

works but in Lean 4,

import Mathlib.Logic.Basic
import Std.Tactic.Simpa

example (P : Prop) (h : ¬ ¬ P) : P := by
  have : ¬ ¬ P := h
  simpa

doesn't, you need to do

import Mathlib.Logic.Basic
import Std.Tactic.Simpa

example (P : Prop) (h : ¬ ¬ P) : P := by
  have : ¬ ¬ P := h
  simp at this
  assumption

@Mario Carneiro

Mario Carneiro (Apr 28 2023 at 15:47):

fixed on master

Patrick Massot (Apr 28 2023 at 15:58):

Thanks!


Last updated: Dec 20 2023 at 11:08 UTC