src/HOL/Isar_examples/Hoare.thy
changeset 19363 667b5ea637dd
parent 19122 e1b6a5071348
child 20503 503ac4c5ef91
--- a/src/HOL/Isar_examples/Hoare.thy	Sat Apr 08 22:12:02 2006 +0200
+++ b/src/HOL/Isar_examples/Hoare.thy	Sat Apr 08 22:51:06 2006 +0200
@@ -31,7 +31,7 @@
   | Cond "'a bexp" "'a com" "'a com"
   | While "'a bexp" "'a assn" "'a com"
 
-abbreviation (output)
+abbreviation
   Skip  ("SKIP")
   "SKIP == Basic id"