src/HOLCF/IOA/NTP/Packet.ML
author wenzelm
Fri, 05 May 2006 21:59:47 +0200
changeset 19579 b802d1804b77
parent 17244 0b2ff9541727
permissions -rw-r--r--
replaced Sorts.DOMAIN by general Sorts.CLASS_ERROR; add_types etc.: reject qualified dummy types -- prevents users from messing up some internal conventions;

(*  Title:      HOL/IOA/NTP/Packet.ML
    ID:         $Id$
    Author:     Tobias Nipkow & Konrad Slind

Packets.
*)

(* Instantiation of a tautology? *)
Goal "!x. x = packet --> hdr(x) = hdr(packet)";
 by (simp_tac (simpset() addsimps [hdr_def]) 1);
qed "eq_packet_imp_eq_hdr"; 

Addsimps [hdr_def,msg_def];