src/HOL/Integ/NatBin.thy
changeset 19380 b808efaa5828
parent 18984 4301eb0f051f
child 19601 299d4cd2ef51
--- a/src/HOL/Integ/NatBin.thy	Sun Apr 09 18:51:11 2006 +0200
+++ b/src/HOL/Integ/NatBin.thy	Sun Apr 09 18:51:13 2006 +0200
@@ -18,7 +18,19 @@
 
 defs (overloaded)
   nat_number_of_def:
-     "(number_of::bin => nat) v == nat ((number_of :: bin => int) v)"
+  "(number_of::bin => nat) v == nat ((number_of :: bin => int) v)"
+
+abbreviation (xsymbols)
+  square :: "'a::power => 'a"  ("(_\<twosuperior>)" [1000] 999)
+  "x\<twosuperior> == x^2"
+
+abbreviation (latex output)
+  square1  ("(_\<twosuperior>)" [1000] 999)
+  "square1 x == x^2"
+
+abbreviation (HTML output)
+  square2  ("(_\<twosuperior>)" [1000] 999)
+  "square2 x == x^2"
 
 
 subsection{*Function @{term nat}: Coercion from Type @{typ int} to @{typ nat}*}