diff -r 4939494ed791 -r ce654b0e6d69 src/HOL/HOLCF/IOA/NTP/Packet.thy --- a/src/HOL/HOLCF/IOA/NTP/Packet.thy Tue Feb 13 14:24:50 2018 +0100 +++ b/src/HOL/HOLCF/IOA/NTP/Packet.thy Thu Feb 15 12:11:00 2018 +0100 @@ -10,16 +10,16 @@ 'msg packet = "bool * 'msg" definition - hdr :: "'msg packet => bool" where - "hdr == fst" + hdr :: "'msg packet \ bool" where + "hdr \ fst" definition - msg :: "'msg packet => 'msg" where - "msg == snd" + msg :: "'msg packet \ 'msg" where + "msg \ snd" text \Instantiation of a tautology?\ -lemma eq_packet_imp_eq_hdr: "!x. x = packet --> hdr(x) = hdr(packet)" +lemma eq_packet_imp_eq_hdr: "\x. x = packet \ hdr(x) = hdr(packet)" by simp declare hdr_def [simp] msg_def [simp]