typo
authortraytel
Fri, 19 Sep 2014 10:40:56 +0200
changeset 58386 6999f55645ea
parent 58385 9cbef70cff8e
child 58387 bc35a30cf0f2
typo
src/HOL/Transfer.thy
--- a/src/HOL/Transfer.thy	Fri Sep 19 10:00:34 2014 +0200
+++ b/src/HOL/Transfer.thy	Fri Sep 19 10:40:56 2014 +0200
@@ -263,7 +263,7 @@
 lemma Domainp_iff: "Domainp T x \<longleftrightarrow> (\<exists>y. T x y)"
   by auto
 
-lemma Domaimp_refl[transfer_domain_rule]:
+lemma Domainp_refl[transfer_domain_rule]:
   "Domainp T = Domainp T" ..
 
 lemma Domainp_prod_fun_eq[relator_domain]: