src/HOL/BNF_Examples/Derivation_Trees/Prelim.thy
changeset 55075 b3d0a02a756d
parent 55074 2b0b6f69b148
child 55091 c43394c2e5ec
equal deleted inserted replaced
55074:2b0b6f69b148 55075:b3d0a02a756d
     1 (*  Title:      HOL/BNF/Examples/Derivation_Trees/Prelim.thy
     1 (*  Title:      HOL/BNF_Examples/Derivation_Trees/Prelim.thy
     2     Author:     Andrei Popescu, TU Muenchen
     2     Author:     Andrei Popescu, TU Muenchen
     3     Copyright   2012
     3     Copyright   2012
     4 
     4 
     5 Preliminaries.
     5 Preliminaries.
     6 *)
     6 *)
     7 
     7 
     8 header {* Preliminaries *}
     8 header {* Preliminaries *}
     9 
     9 
    10 theory Prelim
    10 theory Prelim
    11 imports "../../BNF/More_BNFs"
    11 imports "~~/src/HOL/Library/More_BNFs"
    12 begin
    12 begin
    13 
    13 
    14 declare fset_to_fset[simp]
    14 declare fset_to_fset[simp]
    15 
    15 
    16 lemma fst_snd_convol_o[simp]: "<fst o s, snd o s> = s"
    16 lemma fst_snd_convol_o[simp]: "<fst o s, snd o s> = s"