src/HOL/Hoare/Examples.thy
author clasohm
Wed, 29 Nov 1995 17:01:41 +0100
changeset 1374 5e407f2a3323
parent 1335 5e1c0540f285
child 1476 608483c2122a
permissions -rw-r--r--
removed quotes from consts and syntax sections

(*  Title: 	HOL/Hoare/Examples.thy
    ID:         $Id$
    Author: 	Norbert Galm
    Copyright   1995 TUM

Various arithmetic examples.
*)

Examples = Hoare + Arith2 +

syntax
  "@1"	:: nat	("1")
  "@2"	:: nat	("2")

translations
  "1" == "Suc(0)"
  "2" == "Suc(Suc(0))"
end