doc-src/TutorialI/Types/Numbers.thy
changeset 22097 7ee0529c5674
parent 16585 02cf78f0afce
child 23498 4db8aa43076c
equal deleted inserted replaced
22096:fed088a475f9 22097:7ee0529c5674
     1 (* ID:         $Id$ *)
     1 (* ID:         $Id$ *)
     2 theory Numbers imports Real begin
     2 theory Numbers imports Real begin
     3 
     3 
     4 ML "Pretty.setmargin 64"
     4 ML "Pretty.setmargin 64"
     5 ML "IsarOutput.indent := 0"  (*we don't want 5 for listing theorems*)
     5 ML "ThyOutput.indent := 0"  (*we don't want 5 for listing theorems*)
     6 
     6 
     7 text{*
     7 text{*
     8 
     8 
     9 numeric literals; default simprules; can re-orient
     9 numeric literals; default simprules; can re-orient
    10 *}
    10 *}