src/HOL/Analysis/Linear_Algebra.thy
changeset 66641 ff2e0115fea4
parent 66503 7685861f337d
child 66804 3f9bb52082c4
equal deleted inserted replaced
66640:c61c957b0439 66641:ff2e0115fea4
   308   unfolding span_def by (rule hull_unique)
   308   unfolding span_def by (rule hull_unique)
   309 
   309 
   310 lemma span_minimal: "S \<subseteq> T \<Longrightarrow> subspace T \<Longrightarrow> span S \<subseteq> T"
   310 lemma span_minimal: "S \<subseteq> T \<Longrightarrow> subspace T \<Longrightarrow> span S \<subseteq> T"
   311   unfolding span_def by (rule hull_minimal)
   311   unfolding span_def by (rule hull_minimal)
   312 
   312 
   313 lemma span_UNIV: "span UNIV = UNIV"
   313 lemma span_UNIV [simp]: "span UNIV = UNIV"
   314   by (intro span_unique) auto
   314   by (intro span_unique) auto
   315 
   315 
   316 lemma (in real_vector) span_induct:
   316 lemma (in real_vector) span_induct:
   317   assumes x: "x \<in> span S"
   317   assumes x: "x \<in> span S"
   318     and P: "subspace (Collect P)"
   318     and P: "subspace (Collect P)"