src/HOL/Record.thy
changeset 54147 97a8ff4e4ac9
parent 51112 da97167e03f7
child 55066 4e5ddf3162ac
--- a/src/HOL/Record.thy	Fri Oct 18 10:35:57 2013 +0200
+++ b/src/HOL/Record.thy	Fri Oct 18 10:43:20 2013 +0200
@@ -399,7 +399,7 @@
 lemma refl_conj_eq: "Q = R \<Longrightarrow> P \<and> Q \<longleftrightarrow> P \<and> R"
   by simp
 
-lemma iso_tuple_UNIV_I [no_atp]: "x \<in> UNIV \<equiv> True"
+lemma iso_tuple_UNIV_I: "x \<in> UNIV \<equiv> True"
   by simp
 
 lemma iso_tuple_True_simp: "(True \<Longrightarrow> PROP P) \<equiv> PROP P"