src/HOL/BNF/BNF.thy
author wenzelm
Fri, 11 Oct 2013 20:45:21 +0200
changeset 54325 2c4155003352
parent 54026 82d9b2701a03
child 54539 bbab2ebda234
permissions -rw-r--r--
clarified Editor.current_command: allow outdated snapshot; more accurate Document_View.perspective based on current_command for proper state output (see also 88c6e630c15f and ef62204a126b);

(*  Title:      HOL/BNF/BNF.thy
    Author:     Dmitriy Traytel, TU Muenchen
    Author:     Andrei Popescu, TU Muenchen
    Author:     Jasmin Blanchette, TU Muenchen
    Copyright   2012

Bounded natural functors for (co)datatypes.
*)

header {* Bounded Natural Functors for (Co)datatypes *}

theory BNF
imports More_BNFs BNF_LFP BNF_GFP Coinduction
begin

hide_const (open) image2 image2p vimage2p Gr Grp collect fsts snds setl setr 
  convol thePull pick_middlep fstOp sndOp csquare inver
  image2 relImage relInvImage prefCl PrefCl Succ Shift shift

end