CookBook/Package/Ind_Interface.thy
changeset 42 cd612b489504
parent 35 d5c090b9a2b1
child 53 0c3580c831a4
equal deleted inserted replaced
41:b11653b11bd3 42:cd612b489504
     1 theory Ind_Interface
     1 theory Ind_Interface
     2 imports Base Simple_Inductive_Package
     2 imports "../Base" Simple_Inductive_Package
     3 begin
     3 begin
     4 
     4 
     5 (*<*)
     5 (*<*)
     6 ML {*
     6 ML {*
     7 structure SIP = SimpleInductivePackage
     7 structure SIP = SimpleInductivePackage
   112     [Const (\"all\", \<dots>) $ Abs (\"x\", TFree (\"'a\", \<dots>),
   112     [Const (\"all\", \<dots>) $ Abs (\"x\", TFree (\"'a\", \<dots>),
   113        Const (\"all\", \<dots>) $ Abs (\"y\", TFree (\"'a\", \<dots>),
   113        Const (\"all\", \<dots>) $ Abs (\"y\", TFree (\"'a\", \<dots>),
   114          Const (\"all\", \<dots>) $ Abs (\"z\", TFree (\"'a\", \<dots>),
   114          Const (\"all\", \<dots>) $ Abs (\"z\", TFree (\"'a\", \<dots>),
   115            Const (\"==>\", \<dots>) $
   115            Const (\"==>\", \<dots>) $
   116              (Const (\"Trueprop\", \<dots>) $
   116              (Const (\"Trueprop\", \<dots>) $
   117                 (Free (\"trcl\", \<dots>) $ Free (\"r\", \<dots>) $ Bound 2 $ Bound 1)) $
   117                (Free (\"trcl\", \<dots>) $ Free (\"r\", \<dots>) $ Bound 2 $ Bound 1)) $
   118              (Const (\"==>\", \<dots>) $ \<dots> $ \<dots>))))])]),
   118              (Const (\"==>\", \<dots>) $ \<dots> $ \<dots>))))])]),
   119  \<dots>)
   119  \<dots>)
   120 : (((Name.binding * typ) * mixfix) list *
   120 : (((Name.binding * typ) * mixfix) list *
   121    (Attrib.binding * term list) list) * local_theory"}
   121    (Attrib.binding * term list) list) * local_theory"}
   122 In the list of variables passed to @{ML_open read_specification (Specification)}, we have
   122 In the list of variables passed to @{ML_open read_specification (Specification)}, we have