src/HOL/ex/Records.thy
changeset 11701 3d51fbf81c17
parent 10357 0d0cac129618
child 11704 3c50a2cd6f00
--- a/src/HOL/ex/Records.thy	Fri Oct 05 21:50:37 2001 +0200
+++ b/src/HOL/ex/Records.thy	Fri Oct 05 21:52:39 2001 +0200
@@ -182,7 +182,7 @@
 
 constdefs
   foo10 :: nat
-  "foo10 == getX (| x = 2, y = 0, colour = Blue |)"
+  "foo10 == getX (| x = # 2, y = 0, colour = Blue |)"
 
 
 subsubsection {* Non-coercive structural subtyping *}
@@ -194,7 +194,7 @@
 
 constdefs
   foo11 :: cpoint
-  "foo11 == setX (| x = 2, y = 0, colour = Blue |) 0"
+  "foo11 == setX (| x = # 2, y = 0, colour = Blue |) 0"
 
 
 subsection {* Other features *}
@@ -207,7 +207,7 @@
 
 text {*
  \noindent May not apply @{term getX} to 
- @{term [source] "(| x' = 2, y' = 0 |)"}.
+ @{term [source] "(| x' = # 2, y' = 0 |)"}.
 *}
 
 text {* \medskip Polymorphic records. *}