src/HOL/Multivariate_Analysis/Linear_Algebra.thy
changeset 60307 75e1aa7a450e
parent 60303 00c06f1315d0
child 60420 884f54e01427
equal deleted inserted replaced
60306:6b7c64ab8bd2 60307:75e1aa7a450e
  1655   "\<exists>B. (B :: ('a::euclidean_space) set) \<subseteq> V \<and> independent B \<and> V \<subseteq> span B \<and> (card B = dim V)"
  1655   "\<exists>B. (B :: ('a::euclidean_space) set) \<subseteq> V \<and> independent B \<and> V \<subseteq> span B \<and> (card B = dim V)"
  1656   unfolding dim_def some_eq_ex[of "\<lambda>n. \<exists>B. B \<subseteq> V \<and> independent B \<and> V \<subseteq> span B \<and> (card B = n)"]
  1656   unfolding dim_def some_eq_ex[of "\<lambda>n. \<exists>B. B \<subseteq> V \<and> independent B \<and> V \<subseteq> span B \<and> (card B = n)"]
  1657   using maximal_independent_subset[of V] independent_bound
  1657   using maximal_independent_subset[of V] independent_bound
  1658   by auto
  1658   by auto
  1659 
  1659 
       
  1660 corollary dim_le_card:
       
  1661   fixes s :: "'a::euclidean_space set"
       
  1662   shows "finite s \<Longrightarrow> dim s \<le> card s"
       
  1663 by (metis basis_exists card_mono)
       
  1664 
  1660 text {* Consequences of independence or spanning for cardinality. *}
  1665 text {* Consequences of independence or spanning for cardinality. *}
  1661 
  1666 
  1662 lemma independent_card_le_dim:
  1667 lemma independent_card_le_dim:
  1663   fixes B :: "'a::euclidean_space set"
  1668   fixes B :: "'a::euclidean_space set"
  1664   assumes "B \<subseteq> V"
  1669   assumes "B \<subseteq> V"