Skip to content

Commit

Permalink
chore(algebra/group_power): move inv_one from group_power to field (#…
Browse files Browse the repository at this point in the history
…1495)

* chore(algebra/group_power): move inv_one from group_power to field

*  fix
  • Loading branch information
ChrisHughes24 authored and mergify[bot] committed Sep 27, 2019
1 parent 74f09d0 commit e0c204e
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 2 additions & 0 deletions src/algebra/field.lean
Expand Up @@ -19,6 +19,8 @@ instance division_ring.to_domain [s : division_ring α] : domain α :=
division_ring.mul_ne_zero (mt or.inl hn) (mt or.inr hn) h
..s }

@[simp] theorem inv_one [division_ring α] : (1⁻¹ : α) = 1 := by rw [inv_eq_one_div, one_div_one]

@[simp] theorem inv_inv' [discrete_field α] (x : α) : x⁻¹⁻¹ = x :=
if h : x = 0
then by rw [h, inv_zero, inv_zero]
Expand Down
2 changes: 0 additions & 2 deletions src/algebra/group_power.lean
Expand Up @@ -17,8 +17,6 @@ import data.int.basic data.list.basic
universes u v
variable {α : Type u}

@[simp] theorem inv_one [division_ring α] : (1⁻¹ : α) = 1 := by rw [inv_eq_one_div, one_div_one]

/-- The power operation in a monoid. `a^n = a*a*...*a` n times. -/
def monoid.pow [monoid α] (a : α) : ℕ → α
| 0 := 1
Expand Down

0 comments on commit e0c204e

Please sign in to comment.