src/HOL/HOLCF/LowerPD.thy
changeset 61169 4de9ff3ea29a
parent 58880 0baae4311a9f
child 61998 b66d2ca1f907
--- a/src/HOL/HOLCF/LowerPD.thy	Sun Sep 13 22:25:21 2015 +0200
+++ b/src/HOL/HOLCF/LowerPD.thy	Sun Sep 13 22:56:52 2015 +0200
@@ -407,14 +407,14 @@
 by (simp add: lower_map_def lower_bind_bind)
 
 lemma ep_pair_lower_map: "ep_pair e p \<Longrightarrow> ep_pair (lower_map\<cdot>e) (lower_map\<cdot>p)"
-apply default
+apply standard
 apply (induct_tac x rule: lower_pd_induct, simp_all add: ep_pair.e_inverse)
 apply (induct_tac y rule: lower_pd_induct)
 apply (simp_all add: ep_pair.e_p_below monofun_cfun del: lower_plus_below_iff)
 done
 
 lemma deflation_lower_map: "deflation d \<Longrightarrow> deflation (lower_map\<cdot>d)"
-apply default
+apply standard
 apply (induct_tac x rule: lower_pd_induct, simp_all add: deflation.idem)
 apply (induct_tac x rule: lower_pd_induct)
 apply (simp_all add: deflation.below monofun_cfun del: lower_plus_below_iff)