Skip to content

Commit

Permalink
chore: generalise exists_eq_right_right (#353)
Browse files Browse the repository at this point in the history
  • Loading branch information
b-mehta authored Nov 8, 2023
1 parent 869c615 commit 87b0742
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Std/Logic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -482,10 +482,10 @@ theorem not_forall_of_exists_not {p : α → Prop} : (∃ x, ¬p x) → ¬∀ x,
@[simp] theorem exists_eq_or_imp : (∃ a, (a = a' ∨ q a) ∧ p a) ↔ p a' ∨ ∃ a, q a ∧ p a := by
simp only [or_and_right, exists_or, exists_eq_left]

@[simp] theorem exists_eq_right_right : (∃ (a : α), p a ∧ b ∧ a = a') ↔ p a' ∧ b := by
@[simp] theorem exists_eq_right_right : (∃ (a : α), p a ∧ q a ∧ a = a') ↔ p a' ∧ q a' := by
simp [← and_assoc]

@[simp] theorem exists_eq_right_right' : (∃ (a : α), p a ∧ b ∧ a' = a) ↔ p a' ∧ b := by
@[simp] theorem exists_eq_right_right' : (∃ (a : α), p a ∧ q a ∧ a' = a) ↔ p a' ∧ q a' := by
(conv in _=_ => rw [eq_comm]); simp

@[simp] theorem exists_prop : (∃ _h : a, b) ↔ a ∧ b :=
Expand Down

0 comments on commit 87b0742

Please sign in to comment.