Skip to content

Commit

Permalink
feat(Order/Group): a nontrivial densely linear ordered group isn't cy…
Browse files Browse the repository at this point in the history
…clic (#15547)
  • Loading branch information
urkud authored and bjoernkjoshanssen committed Sep 9, 2024
1 parent 669c659 commit aaa7119
Showing 1 changed file with 23 additions and 0 deletions.
23 changes: 23 additions & 0 deletions Mathlib/Algebra/Order/Group/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -102,4 +102,27 @@ lemma zpow_left_inj (hn : n ≠ 0) : a ^ n = b ^ n ↔ a = b := (zpow_left_injec
`zsmul_lt_zsmul_iff'`."]
lemma zpow_eq_zpow_iff' (hn : n ≠ 0) : a ^ n = b ^ n ↔ a = b := zpow_left_inj hn

variable (α) in
/-- A nontrivial densely linear ordered commutative group can't be a cyclic group. -/
@[to_additive
"A nontrivial densely linear ordered additive commutative group can't be a cyclic group."]
theorem not_isCyclic_of_denselyOrdered [DenselyOrdered α] [Nontrivial α] : ¬IsCyclic α := by
intro h
rcases exists_zpow_surjective α with ⟨a, ha⟩
rcases lt_trichotomy a 1 with hlt | rfl | hlt
· rcases exists_between hlt with ⟨b, hab, hb⟩
rcases ha b with ⟨k, rfl⟩
suffices 0 < k ∧ k < 1 by omega
rw [← one_lt_inv'] at hlt
simp_rw [← zpow_lt_zpow_iff hlt]
simp_all
· rcases exists_ne (1 : α) with ⟨b, hb⟩
simpa [hb.symm] using ha b
· rcases exists_between hlt with ⟨b, hb, hba⟩
rcases ha b with ⟨k, rfl⟩
suffices 0 < k ∧ k < 1 by omega
simp_rw [← zpow_lt_zpow_iff hlt]
simp_all

end LinearOrderedCommGroup

0 comments on commit aaa7119

Please sign in to comment.