Skip to content

Commit

Permalink
fix(linear_algebra/dimension): fix build
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Mar 23, 2019
1 parent 0d92ca1 commit 84ed310
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/linear_algebra/dimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -84,7 +84,7 @@ have (span α s).subtype '' ((span α s).subtype ⁻¹' s) = s :=
image_preimage_eq_of_subset $ by rw [← linear_map.range_coe, range_subtype]; exact subset_span,
begin
rw [← (is_basis_span hs).mk_eq_dim],
calc cardinal.mk ↥((submodule.subtype (span α s)) ⁻¹' s) =
calc cardinal.mk ↥((submodule.subtype (span α s) : span α s →ₗ[α] β) ⁻¹' s) =
cardinal.mk ↥((submodule.subtype (span α s)) '' ((submodule.subtype (span α s)) ⁻¹' s)) :
(cardinal.mk_eq_of_injective subtype.val_injective).symm
... = cardinal.mk ↥s : by rw this
Expand Down

0 comments on commit 84ed310

Please sign in to comment.