From 9ffa5ed2a972db4ae6274a7852de37945a32ab0e Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Tue, 3 Jul 2018 17:06:58 +0200 Subject: Rewrote methods: wellformed now two lines, uses named theorems. New, more powerful derive method. Used these to rewrite proofs. --- EqualProps.thy | 48 ++++++++++++++++++------------------------------ 1 file changed, 18 insertions(+), 30 deletions(-) (limited to 'EqualProps.thy') diff --git a/EqualProps.thy b/EqualProps.thy index b691133..10d3b17 100644 --- a/EqualProps.thy +++ b/EqualProps.thy @@ -18,6 +18,7 @@ section \Symmetry / Path inverse\ definition inv :: "[Term, Term, Term] \ Term" ("(1inv[_,/ _,/ _])") where "inv[A,x,y] \ \<^bold>\p:x =\<^sub>A y. indEqual[A] (\x y _. y =\<^sub>A x) (\x. refl(x)) x y p" + lemma inv_type: assumes "p : x =\<^sub>A y" shows "inv[A,x,y]`p : y =\<^sub>A x" @@ -64,45 +65,32 @@ section \Transitivity / Path composition\ text "``Raw'' composition function, of type \\x,y:A. x =\<^sub>A y \ (\z:A. y =\<^sub>A z \ x =\<^sub>A z)\." definition rcompose :: "Term \ Term" ("(1rcompose[_])") - where "rcompose[A] \ \<^bold>\x:A. \<^bold>\y:A. \<^bold>\p:x =\<^sub>A y. indEqual[A] + where "rcompose[A] \ \<^bold>\x:A. \<^bold>\y:A. \<^bold>\p:(x =\<^sub>A y). indEqual[A] (\x y _. \z:A. y =\<^sub>A z \ x =\<^sub>A z) - (\x. \<^bold>\z:A. \<^bold>\p:x =\<^sub>A z. indEqual[A](\x z _. x =\<^sub>A z) (\x. refl(x)) x z p) + (\x. \<^bold>\z:A. \<^bold>\p:(x =\<^sub>A z). indEqual[A](\x z _. x =\<^sub>A z) (\x. refl(x)) x z p) x y p" text "``Natural'' composition function abbreviation, effectively equivalent to a function of type \\x,y,z:A. x =\<^sub>A y \ y =\<^sub>A z \ x =\<^sub>A z\." abbreviation compose :: "[Term, Term, Term, Term] \ Term" ("(1compose[_,/ _,/ _,/ _])") - where "compose[A,x,y,z] \ \<^bold>\p:x =\<^sub>A y. \<^bold>\q:y =\<^sub>A z. rcompose[A]`x`y`p`z`q" + where "compose[A,x,y,z] \ \<^bold>\p:(x =\<^sub>A y). \<^bold>\q:(y =\<^sub>A z). rcompose[A]`x`y`p`z`q" + + +lemma compose_type: + assumes "p : x =\<^sub>A y" and "q : y =\<^sub>A z" + shows "compose[A,x,y,z]`p`q : x =\<^sub>A z" + +sorry lemma compose_comp: assumes "a : A" shows "compose[A,a,a,a]`refl(a)`refl(a) \ refl(a)" -proof (unfold rcompose_def) - have "compose[A,a,a,a]`refl(a) \ \<^bold>\q:a =\<^sub>A a. rcompose[A]`a`a`refl(a)`a`q" - proof standard+ (*TODO: Set up the Simplifier to handle this proof at some point.*) - fix p q assume "p : a =\<^sub>A a" and "q : a =\<^sub>A a" - then show "rcompose[A]`a`a`p`a`q : a =\<^sub>A a" - proof (unfold rcompose_def) - have "(\<^bold>\x:A. \<^bold>\y:A. \<^bold>\p:x =\<^sub>A y. (indEqual[A] - (\x y _. \z:A. y =[A] z \ x =[A] z) - (\x. \<^bold>\z:A. \<^bold>\q:x =\<^sub>A z. (indEqual[A] (\x z _. x =\<^sub>A z) refl x z q)) - x y p))`a`a`p`a`q \ ..." (*Okay really need to set up the Simplifier...*) -oops - -text "The above proof is a good candidate for proof automation; in particular we would like the system to be able to automatically find the conditions of the \using\ clause in the proof. -This would likely involve something like: - 1. Recognizing that there is a function application that can be simplified. - 2. Noting that the obstruction to applying \Prod_comp\ is the requirement that \refl(a) : a =\<^sub>A a\. - 3. Obtaining such a condition, using the known fact \a : A\ and the introduction rule \Equal_intro\." - -lemmas Equal_simps [simp] = inv_comp compose_comp - -section \Pretty printing\ - -abbreviation inv_pretty :: "[Term, Term, Term, Term] \ Term" ("(1_\<^sup>-\<^sup>1[_, _, _])" 500) - where "p\<^sup>-\<^sup>1[A,x,y] \ inv[A,x,y]`p" - -abbreviation compose_pretty :: "[Term, Term, Term, Term, Term, Term] \ Term" ("(1_ \[_, _, _, _]/ _)") - where "p \[A,x,y,z] q \ compose[A,x,y,z]`p`q" \ No newline at end of file +sorry \ \Long and tedious proof if the Simplifier is not set up.\ + + +lemmas Equal_simps [intro] = inv_comp compose_comp + + +end \ No newline at end of file -- cgit v1.2.3