From c2eea7696bdfb5f0045d60ee28d39c361c038455 Mon Sep 17 00:00:00 2001 From: Burkhart Wolff Date: Wed, 3 Apr 2024 16:15:29 +0200 Subject: [PATCH] ... --- .../technical_report/technical_report.thy | 37 +++++++++++++++---- 1 file changed, 30 insertions(+), 7 deletions(-) diff --git a/Isabelle_DOF/ontologies/technical_report/technical_report.thy b/Isabelle_DOF/ontologies/technical_report/technical_report.thy index 51104cc..c6a64a8 100644 --- a/Isabelle_DOF/ontologies/technical_report/technical_report.thy +++ b/Isabelle_DOF/ontologies/technical_report/technical_report.thy @@ -78,8 +78,8 @@ doc_class report = \background\\<^sup>* ~~ \technical || example \\<^sup>+ ~~ \conclusion\\<^sup>+ ~~ - \index\\<^sup>* ~~ - bibliography)" + bibliography ~~ + \index\ ~~ \annex\\<^sup>* )" ML\ML_Syntax.print_string\ ML\ML_Syntax.atomic\ @@ -149,14 +149,37 @@ lemma seq_cancel : "Lang (a ~~ b) \ Lang (a ~~ c) = (Lang (b) \ Lang ( c) = (Lang (a) \ Lang (c))" sorry + + +lemma opt_star_incl:"Lang (opt a) \ Lang (Star a)" by (simp add: opt_def subset_iff) +lemma rep1_star_incl:"Lang (rep1 a) \ Lang (Star a)" + unfolding rep1_def + apply(subst L_Star) + apply(subst L_Conc) + by force + + +lemma regexp_unit_right : "Lang (a) = Lang (a ~~ One) " by simp +lemma regexp_unit_left : "Lang (a) = Lang (One ~~ a) " by simp + +lemma regexp_seq_mono : + "Lang(a) \ Lang (a') \ Lang(b) \ Lang (b') \ Lang(a ~~ b) \ Lang(a' ~~ b')" + by auto + +lemma seq_d1 : "Lang (opt b ~~ a) \ Lang ( 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\ +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 + +text\Not a terribly deep theorem, but an interesting property of consistency between +ontologies - so, a lemma that shouldn't break if the involved ontologies were changed: +the structural language of articles should be included in the structural language of reports, +that is to say, reports should just have a richer structure than ordinary papers: \ + +theorem articles_sub_reports: \(Lang article_monitor) \ Lang report_monitor\ unfolding article_monitor_def report_monitor_def apply(simp only: seq_cancel seq_d1 seq_d2 seq_d3) - oops + done end