aboutsummaryrefslogtreecommitdiff
path: root/ProdProps.thy
diff options
context:
space:
mode:
authorJosh Chen2018-08-18 23:27:25 +0200
committerJosh Chen2018-08-18 23:27:25 +0200
commit8833cdf99d3128466d85eb88aeb8e340e07e937c (patch)
tree87094caffe667540ac03cc05e9e1054c04a112d9 /ProdProps.thy
parente1be5f97bb2a42b3179bc24b118d69af137f8e5d (diff)
Reorganize methods
Diffstat (limited to '')
-rw-r--r--ProdProps.thy12
1 files changed, 6 insertions, 6 deletions
diff --git a/ProdProps.thy b/ProdProps.thy
index 3e51102..1af6ad3 100644
--- a/ProdProps.thy
+++ b/ProdProps.thy
@@ -29,10 +29,10 @@ proof (subst (0 1 2 3) compose_def)
proof compute
show "\<And>x. x: A \<Longrightarrow> h`(g`(f`x)) \<equiv> h`((\<^bold>\<lambda>y. g`(f`y))`x)"
proof compute
- show "\<And>x. x: A \<Longrightarrow> g`(f`x): C" by (simple lems: assms)
+ show "\<And>x. x: A \<Longrightarrow> g`(f`x): C" by (routine lems: assms)
qed
- show "\<And>x. x: B \<Longrightarrow> h`(g`x): D(g`x)" by (simple lems: assms)
- qed (simple lems: assms)
+ show "\<And>x. x: B \<Longrightarrow> h`(g`x): D(g`x)" by (routine lems: assms)
+ qed (routine lems: assms)
qed fact
qed
@@ -44,9 +44,9 @@ proof (subst compose_def, subst Prod_eq)
show "\<And>a. a: A \<Longrightarrow> (\<^bold>\<lambda>x. c(x))`((\<^bold>\<lambda>x. b(x))`a) \<equiv> (\<^bold>\<lambda>x. c (b x))`a"
proof compute
show "\<And>a. a: A \<Longrightarrow> c((\<^bold>\<lambda>x. b(x))`a) \<equiv> (\<^bold>\<lambda>x. c(b(x)))`a"
- by compute (simple lems: assms, compute?)+
- qed (simple lems: assms)
-qed (simple lems: assms)
+ by (derive lems: assms)
+ qed (routine lems: assms)
+qed (derive lems: assms)
end