src/HOLCF/HOLCF.thy
changeset 40002 c5b5f7a3a3b1
parent 39974 b525988432e9
child 40011 b974cf829099
--- a/src/HOLCF/HOLCF.thy	Mon Oct 11 16:24:44 2010 -0700
+++ b/src/HOLCF/HOLCF.thy	Mon Oct 11 21:35:31 2010 -0700
@@ -15,7 +15,16 @@
 
 ML {* path_add "~~/src/HOLCF/Library" *}
 
-text {* Legacy theorem names *}
+text {* Legacy theorem names deprecated after Isabelle2009-2: *}
+
+lemmas expand_fun_below = fun_below_iff
+lemmas below_fun_ext = fun_belowI
+lemmas expand_cfun_eq = cfun_eq_iff
+lemmas ext_cfun = cfun_eqI
+lemmas expand_cfun_below = cfun_below_iff
+lemmas below_cfun_ext = cfun_belowI
+
+text {* Older legacy theorem names: *}
 
 lemmas sq_ord_less_eq_trans = below_eq_trans
 lemmas sq_ord_eq_less_trans = eq_below_trans