src/HOL/Library/Product_Vector.thy
changeset 61915 e9812a95d108
parent 60679 ade12ef2773c
child 61969 e01015e49041
--- a/src/HOL/Library/Product_Vector.thy	Tue Dec 22 15:39:01 2015 +0100
+++ b/src/HOL/Library/Product_Vector.thy	Tue Dec 22 21:58:27 2015 +0100
@@ -449,6 +449,10 @@
   using snd_add snd_scaleR
   by (rule bounded_linear_intro [where K=1], simp add: norm_prod_def)
 
+lemmas bounded_linear_fst_comp = bounded_linear_fst[THEN bounded_linear_compose]
+
+lemmas bounded_linear_snd_comp = bounded_linear_snd[THEN bounded_linear_compose]
+
 lemma bounded_linear_Pair:
   assumes f: "bounded_linear f"
   assumes g: "bounded_linear g"