@@ -32,22 +32,22 @@ instance {α : Type*} [Mul α] [Preorder α] [MulLeftStrictMono α] :
3232    PosMulStrictMono (WithZero α) where 
3333  mul_lt_mul_of_pos_left
3434  | (x : α), hx, 0 , (b : α), _ => by  simpa only [mul_zero] using WithZero.zero_lt_coe _
35-   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; exact mul_lt_mul_left' h x 
35+   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; gcongr 
3636
3737open  Function in 
3838instance  {α : Type*} [Mul α] [Preorder α] [MulRightStrictMono α] :
3939    MulPosStrictMono (WithZero α) where 
4040  mul_lt_mul_of_pos_right
4141  | (x : α), hx, 0 , (b : α), _ => by  simpa only [mul_zero] using WithZero.zero_lt_coe _
42-   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; exact mul_lt_mul_right' h x 
42+   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; gcongr 
4343
4444instance  {α : Type*} [Mul α] [Preorder α] [MulLeftMono α] :
4545    PosMulMono (WithZero α) where 
4646  mul_le_mul_of_nonneg_left
4747  | 0 , _, a, b, _ => by  simp
4848  | (x : α), _, 0 , _, _ => by  simp
4949  | (x : α), _, (a : α), 0 , h => by  simp at h
50-   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; exact mul_le_mul_left' h x 
50+   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; gcongr 
5151
5252-- This makes `lt_mul_of_le_of_one_lt'` work on `ℤᵐ⁰` 
5353open  Function in 
@@ -57,7 +57,7 @@ instance {α : Type*} [Mul α] [Preorder α] [MulRightMono α] :
5757  | 0 , _, a, b, _ => by  simp
5858  | (x : α), _, 0 , _, _ => by  simp
5959  | (x : α), _, (a : α), 0 , h => by  simp at h
60-   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; exact mul_le_mul_right' h x 
60+   | (x : α), hx, (a : α), (b : α), h => by  norm_cast at h ⊢; gcongr 
6161
6262section  Units
6363
0 commit comments