src/HOL/Matrix_LP/ComputeHOL.thy
changeset 55414 eab03e9cee8a
parent 55413 a8e96847523c
child 59582 0fbed69ff081
--- a/src/HOL/Matrix_LP/ComputeHOL.thy	Wed Feb 12 08:35:56 2014 +0100
+++ b/src/HOL/Matrix_LP/ComputeHOL.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -50,9 +50,9 @@
 lemma compute_snd: "snd (x,y) = y" by simp
 lemma compute_pair_eq: "((a, b) = (c, d)) = (a = c \<and> b = d)" by auto
 
-lemma prod_case_simp: "prod_case f (x,y) = f x y" by simp
+lemma case_prod_simp: "case_prod f (x,y) = f x y" by simp
 
-lemmas compute_pair = compute_fst compute_snd compute_pair_eq prod_case_simp
+lemmas compute_pair = compute_fst compute_snd compute_pair_eq case_prod_simp
 
 (*** compute_option ***)