Skip to content

Commit 4ef6095

Browse files
urkuddagurtomas
authored andcommitted
chore(Logic/Basic): drop 3 long-deprecated theorems (#14157)
1 parent 9d54b6e commit 4ef6095

File tree

1 file changed

+3
-13
lines changed

1 file changed

+3
-13
lines changed

Mathlib/Logic/Basic.lean

+3-13
Original file line numberDiff line numberDiff line change
@@ -353,19 +353,9 @@ alias Iff.or := or_congr
353353
alias ⟨Or.rotate, _⟩ := or_rotate
354354
#align or.rotate Or.rotate
355355

356-
@[deprecated Or.imp (since := "2022-10-24")]
357-
theorem or_of_or_of_imp_of_imp {a b c d : Prop} (h₁ : a ∨ b) (h₂ : a → c) (h₃ : b → d) :
358-
c ∨ d :=
359-
Or.imp h₂ h₃ h₁
360-
#align or_of_or_of_imp_of_imp or_of_or_of_imp_of_imp
361-
362-
@[deprecated Or.imp_left (since := "2022-10-24")]
363-
theorem or_of_or_of_imp_left {a c b : Prop} (h₁ : a ∨ c) (h : a → b) : b ∨ c := Or.imp_left h h₁
364-
#align or_of_or_of_imp_left or_of_or_of_imp_left
365-
366-
@[deprecated Or.imp_right (since := "2022-10-24")]
367-
theorem or_of_or_of_imp_right {c a b : Prop} (h₁ : c ∨ a) (h : a → b) : c ∨ b := Or.imp_right h h₁
368-
#align or_of_or_of_imp_right or_of_or_of_imp_right
356+
#align or_of_or_of_imp_of_imp Or.imp
357+
#align or_of_or_of_imp_left Or.imp_left
358+
#align or_of_or_of_imp_right Or.imp_right
369359

370360
theorem Or.elim3 {c d : Prop} (h : a ∨ b ∨ c) (ha : a → d) (hb : b → d) (hc : c → d) : d :=
371361
Or.elim h ha fun h₂ ↦ Or.elim h₂ hb hc

0 commit comments

Comments
 (0)