@@ -111,7 +111,7 @@ variable (Q) {g}
111
111
theorem LinearMap.lTensor_surjective (hg : Function.Surjective g) :
112
112
Function.Surjective (lTensor Q g) := by
113
113
intro z
114
- induction z using TensorProduct.induction_on with
114
+ induction z with
115
115
| zero => exact ⟨0 , map_zero _⟩
116
116
| tmul q p =>
117
117
obtain ⟨n, rfl⟩ := hg p
@@ -136,7 +136,7 @@ theorem LinearMap.lTensor_range :
136
136
theorem LinearMap.rTensor_surjective (hg : Function.Surjective g) :
137
137
Function.Surjective (rTensor Q g) := by
138
138
intro z
139
- induction z using TensorProduct.induction_on with
139
+ induction z with
140
140
| zero => exact ⟨0 , map_zero _⟩
141
141
| tmul p q =>
142
142
obtain ⟨n, rfl⟩ := hg p
@@ -532,12 +532,12 @@ lemma Ideal.map_includeLeft_eq (I : Ideal A) :
532
532
use x + y
533
533
simp only [map_add]
534
534
· rintro a x ⟨x, hx, rfl⟩
535
- induction a using TensorProduct.induction_on with
535
+ induction a with
536
536
| zero =>
537
537
use 0
538
538
simp only [map_zero, smul_eq_mul, zero_mul]
539
539
| tmul a b =>
540
- induction x using TensorProduct.induction_on with
540
+ induction x with
541
541
| zero =>
542
542
use 0
543
543
simp only [map_zero, smul_eq_mul, mul_zero]
@@ -557,7 +557,7 @@ lemma Ideal.map_includeLeft_eq (I : Ideal A) :
557
557
simp only [map_add, ha', add_smul, hb']
558
558
559
559
· rintro x ⟨y, rfl⟩
560
- induction y using TensorProduct.induction_on with
560
+ induction y with
561
561
| zero =>
562
562
rw [map_zero]
563
563
apply zero_mem
@@ -600,12 +600,12 @@ lemma Ideal.map_includeRight_eq (I : Ideal B) :
600
600
use x + y
601
601
simp only [map_add]
602
602
· rintro a x ⟨x, hx, rfl⟩
603
- induction a using TensorProduct.induction_on with
603
+ induction a with
604
604
| zero =>
605
605
use 0
606
606
simp only [map_zero, smul_eq_mul, zero_mul]
607
607
| tmul a b =>
608
- induction x using TensorProduct.induction_on with
608
+ induction x with
609
609
| zero =>
610
610
use 0
611
611
simp only [map_zero, smul_eq_mul, mul_zero]
@@ -625,7 +625,7 @@ lemma Ideal.map_includeRight_eq (I : Ideal B) :
625
625
simp only [map_add, ha', add_smul, hb']
626
626
627
627
· rintro x ⟨y, rfl⟩
628
- induction y using TensorProduct.induction_on with
628
+ induction y with
629
629
| zero =>
630
630
rw [map_zero]
631
631
apply zero_mem
0 commit comments