Skip to content

Commit

Permalink
unsimp, protect
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies authored Oct 28, 2024
1 parent cfb3a94 commit 6f3cca4
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Data/Real/EReal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -132,11 +132,11 @@ protected def rec {C : EReal → Sort*} (h_bot : C ⊥) (h_real : ∀ a : ℝ, C
| (a : ℝ) => h_real a
| ⊤ => h_top

@[simp] lemma «forall» {p : EReal → Prop} : (∀ r, p r) ↔ p ⊥ ∧ p ⊤ ∧ ∀ r : ℝ, p r where
protected lemma «forall» {p : EReal → Prop} : (∀ r, p r) ↔ p ⊥ ∧ p ⊤ ∧ ∀ r : ℝ, p r where
mp h := ⟨h _, h _, fun _ ↦ h _⟩
mpr h := EReal.rec h.1 h.2.2 h.2.1

@[simp] lemma «exists» {p : EReal → Prop} : (∃ r, p r) ↔ p ⊥ ∨ p ⊤ ∨ ∃ r : ℝ, p r where
protected lemma «exists» {p : EReal → Prop} : (∃ r, p r) ↔ p ⊥ ∨ p ⊤ ∨ ∃ r : ℝ, p r where
mp := by rintro ⟨r, hr⟩; cases r <;> aesop
mpr := by rintro (h | h | ⟨r, hr⟩) <;> exact ⟨_, ‹_›⟩

Expand Down

0 comments on commit 6f3cca4

Please sign in to comment.