recovered metis proof after 115965966e15 (Odd clash of type variables!?);
authorwenzelm
Sun, 21 Dec 2014 15:59:19 +0100
changeset 59166 4e43651235b2
parent 59165 115965966e15
child 59167 c484992c813a
recovered metis proof after 115965966e15 (Odd clash of type variables!?);
src/HOL/Cardinals/Cardinal_Order_Relation.thy
--- a/src/HOL/Cardinals/Cardinal_Order_Relation.thy	Sun Dec 21 15:03:45 2014 +0100
+++ b/src/HOL/Cardinals/Cardinal_Order_Relation.thy	Sun Dec 21 15:59:19 2014 +0100
@@ -1550,9 +1550,11 @@
 lemma Pfunc_mono[simp]:
 assumes "A1 \<subseteq> A2" and "B1 \<subseteq> B2"
 shows "Pfunc A B1 \<subseteq> Pfunc A B2"
-using assms in_mono unfolding Pfunc_def apply safe
-apply(case_tac "x a", auto)
-by (metis in_mono option.simps(5))
+using assms unfolding Pfunc_def
+apply safe
+apply (case_tac "x a", auto)
+apply (metis in_mono option.simps(5))
+done
 
 lemma card_of_Func_UNIV_UNIV:
 "|Func (UNIV::'a set) (UNIV::'b set)| =o |UNIV::('a \<Rightarrow> 'b) set|"