Skip to content

Commit

Permalink
chore(Data/Finset/PiInduction): remove porting note about `clear_valu…
Browse files Browse the repository at this point in the history
…e` (#12100)

This tactic now exists.
  • Loading branch information
grunweg committed Apr 12, 2024
1 parent 72721e3 commit cd0e7a0
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Data/Finset/PiInduction.lean
Expand Up @@ -49,8 +49,7 @@ theorem induction_on_pi_of_choice (r : ∀ i, α i → Finset (α i) → Prop)
· rcases sigma_nonempty.1 hne with ⟨i, -, hi⟩
rcases H_ex i (f i) hi with ⟨x, x_mem, hr⟩
set g := update f i ((f i).erase x) with hg
-- Porting note: this tactic does not exist yet
-- clear_value g
clear_value g
have hx' : x ∉ g i := by
rw [hg, update_same]
apply not_mem_erase
Expand Down

0 comments on commit cd0e7a0

Please sign in to comment.