src/HOL/Imperative_HOL/ex/Linked_Lists.thy
changeset 55414 eab03e9cee8a
parent 53108 d84c8de81edf
child 55584 a879f14b6f95
--- a/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Wed Feb 12 08:35:56 2014 +0100
+++ b/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -692,7 +692,7 @@
 
 
 
-lemma sum_distrib: "sum_case fl fr (case x of Empty \<Rightarrow> y | Node v n \<Rightarrow> (z v n)) = (case x of Empty \<Rightarrow> sum_case fl fr y | Node v n \<Rightarrow> sum_case fl fr (z v n))"
+lemma sum_distrib: "case_sum fl fr (case x of Empty \<Rightarrow> y | Node v n \<Rightarrow> (z v n)) = (case x of Empty \<Rightarrow> case_sum fl fr y | Node v n \<Rightarrow> case_sum fl fr (z v n))"
 by (cases x) auto
 
 subsection {* Induction refinement by applying the abstraction function to our induct rule *}