aboutsummaryrefslogtreecommitdiff
path: root/ProdProps.thy
diff options
context:
space:
mode:
authorJosh Chen2018-08-18 14:34:08 +0200
committerJosh Chen2018-08-18 14:34:08 +0200
commit41f13f91d023e497d9b35e7a958a961aa0c7a5e5 (patch)
tree848fc34e93a7e248a87cc419fe9f5d870334b4d7 /ProdProps.thy
parentcf7b0d7b3a10a65c2d382faad909bfb83b194fc7 (diff)
Misc formatting
Diffstat (limited to '')
-rw-r--r--ProdProps.thy1
1 files changed, 0 insertions, 1 deletions
diff --git a/ProdProps.thy b/ProdProps.thy
index 7071b39..adadb29 100644
--- a/ProdProps.thy
+++ b/ProdProps.thy
@@ -21,7 +21,6 @@ text "
lemma compose_assoc:
assumes "A: U(i)" and "f: A \<rightarrow> B" "g: B \<rightarrow> C" "h: \<Prod>x:C. D(x)"
shows "(h \<circ> g) \<circ> f \<equiv> h \<circ> (g \<circ> f)"
-
proof (subst (0 1 2 3) compose_def)
show "\<^bold>\<lambda>x. (\<^bold>\<lambda>y. h`(g`y))`(f`x) \<equiv> \<^bold>\<lambda>x. h`((\<^bold>\<lambda>y. g`(f`y))`x)"
proof (subst Prod_eq)