src/HOL/BNF_Def.thy
changeset 55414 eab03e9cee8a
parent 55163 a740f312d9e4
child 55642 63beb38e9258
--- a/src/HOL/BNF_Def.thy	Wed Feb 12 08:35:56 2014 +0100
+++ b/src/HOL/BNF_Def.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -118,9 +118,9 @@
 lemma predicate2_eqD: "A = B \<Longrightarrow> A a b \<longleftrightarrow> B a b"
 by metis
 
-lemma sum_case_o_inj:
-"sum_case f g \<circ> Inl = f"
-"sum_case f g \<circ> Inr = g"
+lemma case_sum_o_inj:
+"case_sum f g \<circ> Inl = f"
+"case_sum f g \<circ> Inr = g"
 by auto
 
 lemma card_order_csum_cone_cexp_def: