We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
adjoin.range_algebraMap_subset
1 parent 9f5b327 commit ac69319Copy full SHA for ac69319
Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean
@@ -303,11 +303,8 @@ theorem adjoin_eq_range_algebraMap_adjoin :
303
theorem adjoin.algebraMap_mem (x : F) : algebraMap F E x ∈ adjoin F S :=
304
IntermediateField.algebraMap_mem (adjoin F S) x
305
306
-theorem adjoin.range_algebraMap_subset : Set.range (algebraMap F E) ⊆ adjoin F S := by
307
- intro x hx
308
- obtain ⟨f, hf⟩ := hx
309
- rw [← hf]
310
- exact adjoin.algebraMap_mem F S f
+theorem adjoin.range_algebraMap_subset : Set.range (algebraMap F E) ⊆ adjoin F S :=
+ set_range_subset (adjoin F S)
311
312
instance adjoin.fieldCoe : CoeTC F (adjoin F S) where
313
coe x := ⟨algebraMap F E x, adjoin.algebraMap_mem F S x⟩
0 commit comments