Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Mar 18, 2024
1 parent c318688 commit 70c816d
Show file tree
Hide file tree
Showing 5 changed files with 4 additions and 84 deletions.
1 change: 0 additions & 1 deletion Std.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,6 @@ import Std.Tactic.OpenPrivate
import Std.Tactic.PermuteGoals
import Std.Tactic.PrintDependents
import Std.Tactic.PrintPrefix
import Std.Tactic.Relation.Rfl
import Std.Tactic.SeqFocus
import Std.Tactic.SqueezeScope
import Std.Tactic.Unreachable
Expand Down
3 changes: 2 additions & 1 deletion Std/Data/List/Perm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,9 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura, Jeremy Avigad, Mario Carneiro
-/
import Std.Tactic.Alias
import Std.Tactic.Relation.Rfl
import Std.Data.List.Init.Attach
import Std.Data.List.Pairwise
-- Adaptation note: nightly-2024-03-18. We should be able to remove this after nightly-2024-03-19.
import Lean.Elab.Tactic.Rfl

/-!
# List Permutations
Expand Down
3 changes: 0 additions & 3 deletions Std/Logic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -32,9 +32,6 @@ end Classical

theorem heq_iff_eq : HEq a b ↔ a = b := ⟨eq_of_heq, heq_of_eq⟩

theorem proof_irrel_heq {p q : Prop} (hp : p) (hq : q) : HEq hp hq := by
cases propext (iff_of_true hp hq); rfl

@[simp] theorem eq_rec_constant {α : Sort _} {a a' : α} {β : Sort _} (y : β) (h : a = a') :
(@Eq.rec α a (fun α _ => β) y a' h) = y := by cases h; rfl

Expand Down
78 changes: 0 additions & 78 deletions Std/Tactic/Relation/Rfl.lean

This file was deleted.

3 changes: 2 additions & 1 deletion test/rfl.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
import Std.Tactic.Relation.Rfl
import Lean.Elab.Tactic.Rfl
-- Adaptation note: we should be able to remove this import after nightly-2024-03-19

set_option linter.missingDocs false

Expand Down

0 comments on commit 70c816d

Please sign in to comment.