src/HOL/Transfer.thy
changeset 63092 a949b2a5f51d
parent 62324 ae44f16dcea5
child 63343 fb5d8a50c641
--- a/src/HOL/Transfer.thy	Fri May 13 20:22:02 2016 +0200
+++ b/src/HOL/Transfer.thy	Fri May 13 20:24:10 2016 +0200
@@ -510,7 +510,7 @@
   "right_total A \<Longrightarrow> ((A ===> A ===> op=) ===> implies) reflp reflp"
   "bi_total A \<Longrightarrow> ((A ===> A ===> rev_implies) ===> rev_implies) reflp reflp"
   "bi_total A \<Longrightarrow> ((A ===> A ===> op=) ===> rev_implies) reflp reflp"
-using assms unfolding reflp_def[abs_def] rev_implies_def bi_total_def right_total_def rel_fun_def
+unfolding reflp_def[abs_def] rev_implies_def bi_total_def right_total_def rel_fun_def
 by fast+
 
 lemma right_unique_transfer [transfer_rule]: