src/Doc/Isar_Ref/Synopsis.thy
changeset 58310 91ea607a34d8
parent 58305 57752a91eec4
child 58618 782f0b662cae
equal deleted inserted replaced
58309:a09ec6daaa19 58310:91ea607a34d8
  1066 text {*
  1066 text {*
  1067   Isabelle/HOL specification mechanisms (datatype, inductive, etc.)
  1067   Isabelle/HOL specification mechanisms (datatype, inductive, etc.)
  1068   provide suitable derived cases rules.
  1068   provide suitable derived cases rules.
  1069 *}
  1069 *}
  1070 
  1070 
  1071 datatype_new foo = Foo | Bar foo
  1071 datatype foo = Foo | Bar foo
  1072 
  1072 
  1073 notepad
  1073 notepad
  1074 begin
  1074 begin
  1075   fix x :: foo
  1075   fix x :: foo
  1076   have C
  1076   have C