From 8833cdf99d3128466d85eb88aeb8e340e07e937c Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Sat, 18 Aug 2018 23:27:25 +0200 Subject: Reorganize methods --- ex/Methods.thy | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'ex/Methods.thy') diff --git a/ex/Methods.thy b/ex/Methods.thy index 415fbc3..c78af14 100644 --- a/ex/Methods.thy +++ b/ex/Methods.thy @@ -14,7 +14,7 @@ text "Wellformedness results, metatheorems written into the object theory using lemma assumes "A : U(i)" "B: A \ U(i)" "\x. x : A \ C x: B x \ U(i)" shows "\x:A. \y:B x. \z:C x y. \w:A. x =\<^sub>A w : U(i)" -by (simple lems: assms) +by (routine lems: assms) lemma @@ -38,7 +38,7 @@ text "Typechecking and constructing inhabitants:" \ \Correctly determines the type of the pair\ schematic_goal "\A: U(i); B: U(i); a : A; b : B\ \ : ?A" -by simple +by routine \ \Finds pair (too easy).\ schematic_goal "\A: U(i); B: U(i); a : A; b : B\ \ ?x : A \ B" @@ -56,19 +56,19 @@ lemma assumes "A: U(i)" "a: A" shows "(\<^bold>\x. )`a \ " proof compute - show "\x. x: A \ : A \ \" by simple -qed (simple lems: assms) + show "\x. x: A \ : A \ \" by routine +qed (routine lems: assms) lemma assumes "A: U(i)" "B: A \ U(i)" "a: A" "b: B(a)" shows "(\<^bold>\x y. )`a`b \ " proof compute - show "\x. x: A \ \<^bold>\y. : \y:B(x). \x:A. B(x)" by (simple lems: assms) + show "\x. x: A \ \<^bold>\y. : \y:B(x). \x:A. B(x)" by (routine lems: assms) show "(\<^bold>\b. )`b \ " proof compute - show "\b. b: B(a) \ : \x:A. B(x)" by (simple lems: assms) + show "\b. b: B(a) \ : \x:A. B(x)" by (routine lems: assms) qed fact qed fact -- cgit v1.2.3