src/HOLCF/Cprod.thy
changeset 35922 bfa52a972745
parent 35900 aa5dfb03eb1e
child 35926 e6aec5d665f0
--- a/src/HOLCF/Cprod.thy	Mon Mar 22 22:43:21 2010 -0700
+++ b/src/HOLCF/Cprod.thy	Mon Mar 22 22:55:26 2010 -0700
@@ -34,11 +34,11 @@
 
 definition
   csnd :: "('a * 'b) \<rightarrow> 'b" where
-  "csnd = (\<Lambda> p. snd p)"      
+  "csnd = (\<Lambda> p. snd p)"
 
 definition
   csplit :: "('a \<rightarrow> 'b \<rightarrow> 'c) \<rightarrow> ('a * 'b) \<rightarrow> 'c" where
-  "csplit = (\<Lambda> f p. f\<cdot>(cfst\<cdot>p)\<cdot>(csnd\<cdot>p))"
+  "csplit = (\<Lambda> f p. f\<cdot>(fst p)\<cdot>(snd p))"
 
 syntax
   "_ctuple" :: "['a, args] \<Rightarrow> 'a * 'b"  ("(1<_,/ _>)")
@@ -146,13 +146,13 @@
 by (simp add: csplit_def)
 
 lemma csplit2 [simp]: "csplit\<cdot>f\<cdot><x,y> = f\<cdot>x\<cdot>y"
-by (simp add: csplit_def)
+by (simp add: csplit_def cpair_def)
 
 lemma csplit3 [simp]: "csplit\<cdot>cpair\<cdot>z = z"
-by (simp add: csplit_def cpair_cfst_csnd)
+by (simp add: csplit_def cpair_def)
 
 lemma csplit_Pair [simp]: "csplit\<cdot>f\<cdot>(x, y) = f\<cdot>x\<cdot>y"
-by (simp add: csplit_def cfst_def csnd_def)
+by (simp add: csplit_def)
 
 lemmas Cprod_rews = cfst_cpair csnd_cpair csplit2