src/Doc/ProgProve/Bool_nat_list.thy
changeset 54508 4bc48d713602
parent 54467 663a927fdc88
child 55317 834a84553e02
--- a/src/Doc/ProgProve/Bool_nat_list.thy	Tue Nov 19 22:20:01 2013 +0100
+++ b/src/Doc/ProgProve/Bool_nat_list.thy	Wed Nov 20 08:56:54 2013 +0100
@@ -99,10 +99,10 @@
   For example, given the goal @{text"x + 0 = x"}, there is nothing to indicate
   that you are talking about natural numbers. Hence Isabelle can only infer
   that @{term x} is of some arbitrary type where @{text 0} and @{text"+"}
-  exist. As a consequence, you will be unable to prove the
-  goal. To alert you to such pitfalls, Isabelle flags numerals without a
-  fixed type in its output: @{prop"x+0 = x"}.  In this particular example,
-  you need to include
+  exist. As a consequence, you will be unable to prove the goal.
+%  To alert you to such pitfalls, Isabelle flags numerals without a
+%  fixed type in its output: @ {prop"x+0 = x"}.
+  In this particular example, you need to include
   an explicit type constraint, for example @{text"x+0 = (x::nat)"}. If there
   is enough contextual information this may not be necessary: @{prop"Suc x =
   x"} automatically implies @{text"x::nat"} because @{term Suc} is not