File tree Expand file tree Collapse file tree 1 file changed +2
-10
lines changed Expand file tree Collapse file tree 1 file changed +2
-10
lines changed Original file line number Diff line number Diff line change @@ -60,22 +60,14 @@ lemma equiv_region: "equiv UNIV (region X)"
60
60
done
61
61
62
62
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 )
72
64
73
65
lemma region_coregion_Id :
74
66
"idem_scene X \<Longrightarrow> region X \<inter> coregion X = Id"
75
67
by ( transfer , auto , metis idem_overrider.ovr_idem )
76
68
77
69
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
79
71
80
72
lift_definition scene_override :: "'a \<Rightarrow> 'a \<Rightarrow> ('a scene) \<Rightarrow> 'a" ( "_ \<oplus>\<^sub>S _ on _" [ 95 , 0 , 96 ] 95 )
81
73
is "\<lambda> s\<^sub>1 s\<^sub>2 F. F s\<^sub>1 s\<^sub>2" .
You can’t perform that action at this time.
0 commit comments