emphasized general nature of parameter
authorhaftmann
Tue, 13 Oct 2015 09:21:14 +0200
changeset 61423 9b6a0fb85fa3
parent 61422 0dfcd0fb4172
child 61424 c3658c18b7bc
emphasized general nature of parameter
src/HOL/BNF_Def.thy
--- a/src/HOL/BNF_Def.thy	Tue Oct 13 09:21:14 2015 +0200
+++ b/src/HOL/BNF_Def.thy	Tue Oct 13 09:21:14 2015 +0200
@@ -164,7 +164,7 @@
   by (subst (asm) surjective_pairing, unfold prod.case) (erule pick_middlep[THEN conjunct2])
 
 lemma csquare_fstOp_sndOp:
-  "csquare (Collect (split (P OO Q))) snd fst (fstOp P Q) (sndOp P Q)"
+  "csquare (Collect (f (P OO Q))) snd fst (fstOp P Q) (sndOp P Q)"
   unfolding csquare_def fstOp_def sndOp_def using pick_middlep by simp
 
 lemma snd_fst_flip: "snd xy = (fst \<circ> (%(x, y). (y, x))) xy"