8000 Merge `master` into `enhancement/untyped-synchronous-channels` · input-output-hk/thorn-calculus@02e9785 · GitHub
[go: up one dir, main page]

Skip to content

Commit 02e9785

Browse files
committed
Merge master into enhancement/untyped-synchronous-channels
2 parents 92fb2bd + a9d7a1f commit 02e9785

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Thorn_Calculus-Foundations.thy

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -62,10 +62,10 @@ instance channel :: (type) embeddable
6262

6363
subsection \<open>Values\<close>
6464

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 ..
6666

6767
instance val :: embeddable
68-
by standard (meson to_zfc_set_inject inj_def)
68+
by standard (meson val_to_zfc_set_inject inj_def)
6969

7070
definition encode :: "'a::embeddable \<Rightarrow> val" where
7171
[simp]: "encode = (SOME f. inj f)"
@@ -74,7 +74,7 @@ lemma encode_injectivity:
7474
shows "inj encode"
7575
proof -
7676
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)
7878
then show ?thesis
7979
by (auto intro: someI [where P = inj])
8080
qed

0 commit comments

Comments
 (0)
0