src/HOL/ex/Points.thy
changeset 6744 9727e83f0578
parent 6737 03f0ff7ee029
child 6746 cf6ad8d22793
--- a/src/HOL/ex/Points.thy	Thu May 27 20:47:30 1999 +0200
+++ b/src/HOL/ex/Points.thy	Thu May 27 20:49:10 1999 +0200
@@ -15,7 +15,7 @@
   x :: nat
   y :: nat;
 
-text {|
+text {*
   Apart many other things, above record declaration produces the
   following theorems:
 
@@ -25,16 +25,16 @@
 
   The set of theorems "point.simps" is added automatically to the
   standard simpset, "point.iffs" is added to the claset and simpset.
-|};
+*};
 
-text {|
+text {*
   Record declarations define new type abbreviations:
 
     point = "(| x :: nat, y :: nat |)"
     'a point_scheme = "(| x :: nat, y :: nat, ... :: 'a |)"
 
   Extensions `...' must be in type class `more'!
-|};
+*};
 
 consts foo1 :: point;
 consts foo2 :: "(| x :: nat, y :: nat |)";
@@ -137,12 +137,12 @@
   colour :: colour;
 
 
-text {|
+text {*
   The record declaration defines new type constructors:
 
     cpoint = (| x :: nat, y :: nat, colour :: colour |)
     'a cpoint_scheme = (| x :: nat, y :: nat, colour :: colour, ... :: 'a |)
-|};
+*};
 
 consts foo6 :: cpoint;
 consts foo7 :: "(| x :: nat, y :: nat, colour :: colour |)";
@@ -178,7 +178,7 @@
 consts
   foo12 :: nat;
 
-text {| Definition @{term "foo12 == getX (| x' = 2, y' = 0 |)"} is invalid |};
+text {* Definition @{term "foo12 == getX (| x' = 2, y' = 0 |)"} is invalid *};
 
 
 text "polymorphic records";