From 41f13f91d023e497d9b35e7a958a961aa0c7a5e5 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Sat, 18 Aug 2018 14:34:08 +0200 Subject: Misc formatting --- ProdProps.thy | 1 - 1 file changed, 1 deletion(-) (limited to 'ProdProps.thy') 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 \ B" "g: B \ C" "h: \x:C. D(x)" shows "(h \ g) \ f \ h \ (g \ f)" - proof (subst (0 1 2 3) compose_def) show "\<^bold>\x. (\<^bold>\y. h`(g`y))`(f`x) \ \<^bold>\x. h`((\<^bold>\y. g`(f`y))`x)" proof (subst Prod_eq) -- cgit v1.2.3