Skip to content

Commit 75a10f1

Browse files
committed
Shorten apply-style proofs in Scenes
1 parent 9607eda commit 75a10f1

File tree

1 file changed

+2
-10
lines changed

1 file changed

+2
-10
lines changed

Scenes.thy

Lines changed: 2 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -60,22 +60,14 @@ lemma equiv_region: "equiv UNIV (region X)"
6060
done
6161

6262
lemma equiv_coregion: "equiv UNIV (coregion X)"
63-
apply (transfer)
64-
apply (rule equivI)
65-
apply (rule refl_onI)
66-
apply (auto)
67-
apply (rule symI)
68-
apply (auto)
69-
apply (rule transI)
70-
apply (auto)
71-
done
63+
by (transfer) (auto intro!: equivI refl_onI symI transI)
7264

7365
lemma region_coregion_Id:
7466
"idem_scene X \<Longrightarrow> region X \<inter> coregion X = Id"
7567
by (transfer, auto, metis idem_overrider.ovr_idem)
7668

7769
lemma state_eq_iff: "idem_scene S \<Longrightarrow> x = y \<longleftrightarrow> (x, y) \<in> region S \<and> (x, y) \<in> coregion S"
78-
by (metis IntE IntI pair_in_Id_conv region_coregion_Id)
70+
using region_coregion_Id by auto
7971

8072
lift_definition scene_override :: "'a \<Rightarrow> 'a \<Rightarrow> ('a scene) \<Rightarrow> 'a" ("_ \<oplus>\<^sub>S _ on _" [95,0,96] 95)
8173
is "\<lambda> s\<^sub>1 s\<^sub>2 F. F s\<^sub>1 s\<^sub>2" .

0 commit comments

Comments
 (0)