From 20f163eba9b30684a4d39c25eb48d872efe692cf Mon Sep 17 00:00:00 2001 From: Burkhart Wolff Date: Wed, 3 Apr 2024 15:01:25 +0200 Subject: [PATCH] experiments --- .../technical_report/technical_report.thy | 20 +++++++++++++++---- 1 file changed, 16 insertions(+), 4 deletions(-) diff --git a/Isabelle_DOF/ontologies/technical_report/technical_report.thy b/Isabelle_DOF/ontologies/technical_report/technical_report.thy index 5f8bc61..51104cc 100644 --- a/Isabelle_DOF/ontologies/technical_report/technical_report.thy +++ b/Isabelle_DOF/ontologies/technical_report/technical_report.thy @@ -75,7 +75,8 @@ doc_class report = abstract ~~ \table_of_contents\ ~~ \introduction\\<^sup>+ ~~ - \technical || figure \\<^sup>+ ~~ + \background\\<^sup>* ~~ + \technical || example \\<^sup>+ ~~ \conclusion\\<^sup>+ ~~ \index\\<^sup>* ~~ bibliography)" @@ -138,12 +139,23 @@ notation Times (infixr "~~" 60) notation Atom ("\_\" 65) -lemma seq_cancel : "Lang (a ~~ b) \ Lang (a ~~ c) = (Lang (b) \ Lang (c))" sorry +lemma seq_cancel : "Lang (a ~~ b) \ Lang (a ~~ c) = (Lang (b) \ Lang (c))" + apply auto + thm subsetCE + apply(drule_tac c=x in subsetCE) + prefer 3 apply assumption + find_theorems subset_eq elim + prefer 2 + sledgehammer + + sorry lemma seq_d1 : "Lang (opt b ~~ a) \ Lang ( c) = (Lang (a) \ Lang (c))" sorry -lemma seq_d2 : "Lang (a) \ Lang (opt b ~~ c) = (Lang (a) \ Lang (c))" sorry +lemma seq_d2 : "Lang (rep1 b ~~ a) \ Lang ( c) = (Lang (a) \ Lang (c))" sorry +lemma seq_d3 : "Lang (a) \ Lang (opt b ~~ c) = (Lang (a) \ Lang (c))" sorry +lemma seq_d4 : "Lang (a) \ Lang (Star b ~~ c) = (Lang (a) \ Lang (c))" sorry lemma \(Lang article_monitor) \ Lang report_monitor\ unfolding article_monitor_def report_monitor_def - apply(simp only: seq_cancel seq_d1 seq_d2) + apply(simp only: seq_cancel seq_d1 seq_d2 seq_d3) oops