File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -62,10 +62,10 @@ instance channel :: (type) embeddable
62
62
63
63
subsection \<open>Values\<close>
64
64
65
- typedef val = "UNIV :: V set" morphisms to_zfc_set from_zfc_set ..
65
+ typedef val = "UNIV :: V set" morphisms val_to_zfc_set val_from_zfc_set ..
66
66
67
67
instance val :: embeddable
68
- by standard ( meson to_zfc_set_inject inj_def )
68
+ by standard ( meson val_to_zfc_set_inject inj_def )
69
69
70
70
definition encode :: "'a::embeddable \<Rightarrow> val" where
71
71
[ simp ]: "encode = (SOME f. inj f)"
@@ -74,7 +74,7 @@ lemma encode_injectivity:
74
74
shows "inj encode"
75
75
proof -
76
76
have "\<exists>f :: 'a::embeddable \<Rightarrow> val. inj f"
77
- by ( meson ex_inj from_zfc_set_inject [ OF UNIV_I UNIV_I ] inj_def )
77
+ by ( meson ex_inj val_from_zfc_set_inject [ OF UNIV_I UNIV_I ] inj_def )
78
78
then show ?thesis
79
79
by ( auto intro : someI [ where P = inj ])
80
80
qed
You can’t perform that action at this time.
0 commit comments