equal
deleted
inserted
replaced
449 lemma Always_Diff_Un_eq: "[| F \<in> Always(A) |] ==> (F \<in> Always(C-A \<union> B)) \<longleftrightarrow> (F \<in> Always(B))" |
449 lemma Always_Diff_Un_eq: "[| F \<in> Always(A) |] ==> (F \<in> Always(C-A \<union> B)) \<longleftrightarrow> (F \<in> Always(B))" |
450 by (auto simp add: Always_eq_includes_reachable) |
450 by (auto simp add: Always_eq_includes_reachable) |
451 |
451 |
452 (*Delete the nearest invariance assumption (which will be the second one |
452 (*Delete the nearest invariance assumption (which will be the second one |
453 used by Always_Int_I) *) |
453 used by Always_Int_I) *) |
454 lemmas Always_thin = thin_rl [of "F \<in> Always(A)"] |
454 lemmas Always_thin = thin_rl [of "F \<in> Always(A)"] for F A |
455 |
455 |
456 (*To allow expansion of the program's definition when appropriate*) |
456 (*To allow expansion of the program's definition when appropriate*) |
457 named_theorems program "program definitions" |
457 named_theorems program "program definitions" |
458 |
458 |
459 ML |
459 ML |