src/HOL/HOL.thy
changeset 2393 651fce76c86c
parent 2372 a2999e19703b
child 2552 470bc495373e
--- a/src/HOL/HOL.thy	Fri Dec 13 18:32:07 1996 +0100
+++ b/src/HOL/HOL.thy	Fri Dec 13 18:40:50 1996 +0100
@@ -174,9 +174,6 @@
   o_def         "(f::'b=>'c) o g == (%(x::'a). f(g(x)))"
   if_def        "If P x y == @z::'a. (P=True --> z=x) & (P=False --> z=y)"
 
-(* start 8bit 1 *)
-(* end 8bit 1 *)
-
 end
 
 
@@ -198,6 +195,3 @@
 
 val print_ast_translation =
   map alt_ast_tr' [("! ", "*All"), ("? ", "*Ex"), ("?! ", "*Ex1")];
-
-(* start 8bit 2 *)
-(* end 8bit 2 *)