Skip to content

Commit

Permalink
feat(analysis/special_functions/trigonometric/angle): induction_on (#…
Browse files Browse the repository at this point in the history
…11886)

Add `real.angle.induction_on`, for use in deducing results for
`real.angle` from those for `ℝ`.
  • Loading branch information
jsm28 committed Feb 7, 2022
1 parent 26179cc commit 98ef84e
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/analysis/special_functions/trigonometric/angle.lean
Expand Up @@ -36,6 +36,12 @@ def coe_hom : ℝ →+ angle := quotient_add_group.mk' _

@[simp] lemma coe_coe_hom : (coe_hom : ℝ → angle) = coe := rfl

/-- An induction principle to deduce results for `angle` from those for `ℝ`, used with
`induction θ using real.angle.induction_on`. -/
@[elab_as_eliminator]
protected lemma induction_on {p : angle → Prop} (θ : angle) (h : ∀ x : ℝ, p x) : p θ :=
quotient.induction_on' θ h

@[simp] lemma coe_zero : ↑(0 : ℝ) = (0 : angle) := rfl
@[simp] lemma coe_add (x y : ℝ) : ↑(x + y : ℝ) = (↑x + ↑y : angle) := rfl
@[simp] lemma coe_neg (x : ℝ) : ↑(-x : ℝ) = -(↑x : angle) := rfl
Expand Down

0 comments on commit 98ef84e

Please sign in to comment.