We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
2 parents ffc8688 + 0b773e5 commit 87dc3e1Copy full SHA for 87dc3e1
BoogieLang/Util.thy
@@ -357,6 +357,14 @@ lemma max_min_disjoint:
357
using assms
358
by (metis Diff_Diff_Int Diff_eq_empty_iff List.finite_set Max_ge Min_le_iff disjoint_iff_not_equal inf.cobounded2 leD)
359
360
+lemma max_min_disjoint_2:
361
+ assumes "\<forall> a. a \<in> A \<longrightarrow> a \<le> a_max"
362
+ and "\<forall> b. b \<in> B \<longrightarrow> b_min \<le> (b :: vname)"
363
+ and "a_max < b_min"
364
+ shows "A \<inter> B = {}"
365
+ using assms
366
+ by fastforce
367
+
368
lemma dom_map_of_2:"dom (map_of R) = set (map fst R)"
369
by (simp add: Map.dom_map_of_conv_image_fst)
370
0 commit comments