src/HOL/Modules.thy
changeset 68074 8d50467f7555
parent 68073 fad29d2a17a5
child 68189 6163c90694ef
--- a/src/HOL/Modules.thy	Thu May 03 15:07:14 2018 +0200
+++ b/src/HOL/Modules.thy	Thu May 03 16:17:44 2018 +0200
@@ -186,7 +186,7 @@
 lemma span_zero: "0 \<in> span S"
   by (auto simp: span_explicit intro!: exI[of _ "{}"])
 
-lemma span_UNIV: "span UNIV = UNIV"
+lemma span_UNIV[simp]: "span UNIV = UNIV"
   by (auto intro: span_base)
 
 lemma span_add: "x \<in> span S \<Longrightarrow> y \<in> span S \<Longrightarrow> x + y \<in> span S"