@@ -3,7 +3,7 @@ Copyright (c) 2014 Robert Lewis. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Robert Lewis, Leonardo de Moura, Mario Carneiro, Floris van Doorn
5
5
! This file was ported from Lean 3 source module algebra.order.field.basic
6
- ! leanprover-community/mathlib commit 5a82b0671532663333e205f422124a98bdfe673f
6
+ ! leanprover-community/mathlib commit acb3d204d4ee883eb686f45d486a2a6811a01329
7
7
! Please do not edit these lines, except to modify the commit id
8
8
! if you have ported upstream changes.
9
9
-/
@@ -581,7 +581,7 @@ theorem StrictMono.div_const {β : Type _} [Preorder β] {f : β → α} (hf : S
581
581
#align strict_mono.div_const StrictMono.div_const
582
582
583
583
-- see Note [lower instance priority]
584
- instance (priority := 100 ) LinearOrderedField .toDenselyOrdered : DenselyOrdered α where
584
+ instance (priority := 100 ) LinearOrderedSemiField .toDenselyOrdered : DenselyOrdered α where
585
585
dense a₁ a₂ h :=
586
586
⟨(a₁ + a₂) / 2 ,
587
587
calc
@@ -592,7 +592,7 @@ instance (priority := 100) LinearOrderedField.toDenselyOrdered : DenselyOrdered
592
592
(a₁ + a₂) / 2 < (a₂ + a₂) / 2 := div_lt_div_of_lt zero_lt_two (add_lt_add_right h _)
593
593
_ = a₂ := add_self_div_two a₂
594
594
⟩
595
- #align linear_ordered_field.to_densely_ordered LinearOrderedField .toDenselyOrdered
595
+ #align linear_ordered_field.to_densely_ordered LinearOrderedSemiField .toDenselyOrdered
596
596
597
597
theorem min_div_div_right {c : α} (hc : 0 ≤ c) (a b : α) : min (a / c) (b / c) = min a b / c :=
598
598
Eq.symm <| Monotone.map_min fun _ _ => div_le_div_of_le hc
@@ -997,11 +997,4 @@ theorem abs_div (a b : α) : |a / b| = |a| / |b| :=
997
997
theorem abs_one_div (a : α) : |1 / a| = 1 / |a| := by rw [abs_div, abs_one]
998
998
#align abs_one_div abs_one_div
999
999
1000
- theorem pow_minus_two_nonneg : 0 ≤ a ^ (-2 : ℤ) := by
1001
- simp only [inv_nonneg, zpow_neg]
1002
- change 0 ≤ a ^ ((2 : ℕ) : ℤ)
1003
- rw [zpow_ofNat]
1004
- apply sq_nonneg
1005
- #align pow_minus_two_nonneg pow_minus_two_nonneg
1006
-
1007
1000
end
0 commit comments