From 8833cdf99d3128466d85eb88aeb8e340e07e937c Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Sat, 18 Aug 2018 23:27:25 +0200 Subject: Reorganize methods --- Proj.thy | 8 ++++---- 1 file changed, 4 insertions(+), 4 deletions(-) (limited to 'Proj.thy') diff --git a/Proj.thy b/Proj.thy index dffc127..a1c4c8f 100644 --- a/Proj.thy +++ b/Proj.thy @@ -24,9 +24,9 @@ unfolding fst_def by (derive lems: assms) lemma fst_comp: assumes "A: U(i)" and "B: A \ U(i)" and "a: A" and "b: B(a)" shows "fst() \ a" unfolding fst_def -proof +proof compute show "a: A" and "b: B(a)" by fact+ -qed (simple lems: assms)+ +qed (routine lems: assms)+ lemma snd_type: assumes "\x:A. B(x): U(i)" and "p: \x:A. B(x)" shows "snd(p): B(fst p)" @@ -46,11 +46,11 @@ qed fact lemma snd_comp: assumes "A: U(i)" and "B: A \ U(i)" and "a: A" and "b: B(a)" shows "snd() \ b" unfolding snd_def -proof +proof compute show "\x y. y: B(x) \ y: B(x)" . show "a: A" by fact show "b: B(a)" by fact -qed (simple lems: assms) +qed (routine lems: assms) text "Rule attribute declarations:" -- cgit v1.2.3