QuotScript.thy
changeset 166 3300260b63a1
parent 162 20f0b148cfe2
child 171 13aab4c59096
--- a/QuotScript.thy	Fri Oct 23 18:20:06 2009 +0200
+++ b/QuotScript.thy	Sat Oct 24 08:09:09 2009 +0200
@@ -498,6 +498,9 @@
   shows "!f. All f = Ball (Respects R) ((absf ---> id) f)"
   sorry
 
+lemma ho_all_prs: "op = ===> op = ===> op = All All"
+  apply (auto)
+  done
 
 end